diff --git a/theories/logrel/ltyping.v b/theories/logrel/ltyping.v
index 152a30191e1ef9646f51f7f2c484b7b07344a921..ba5810713f167f6d257a2960b5d5d3cde097698a 100755
--- a/theories/logrel/ltyping.v
+++ b/theories/logrel/ltyping.v
@@ -103,7 +103,7 @@ Section Environment.
   Qed.
 
   Definition env_split (Γ Γ1 Γ2 : gmap string (lty Σ)) : iProp Σ :=
-    □ ∀ vs, (env_ltyped Γ vs ∗-∗ (env_ltyped Γ1 vs ∗ env_ltyped Γ2 vs)).
+    □ ∀ vs, env_ltyped Γ vs ∗-∗ (env_ltyped Γ1 vs ∗ env_ltyped Γ2 vs).
 
   Lemma env_split_id_l Γ : ⊢ env_split Γ ∅ Γ.
   Proof.
@@ -119,9 +119,7 @@ Section Environment.
   Lemma env_split_empty : ⊢ env_split ∅ ∅ ∅.
   Proof.
     iIntros "!>" (vs).
-    iSplit.
-    - iIntros "HΓ". rewrite /env_ltyped. auto.
-    - iIntros "[HΓ1 HΓ2]". auto.
+    iSplit; [iIntros "HΓ" | iIntros "[HΓ1 HΓ2]"]; auto.
   Qed.
 
   (* TODO: Get rid of side condition that x does not appear in Γ1 *)
@@ -183,7 +181,7 @@ Section Environment.
       iApply "Hsplit". iFrame "HΓ1 HΓ2".
   Qed.
 
-  (* (* TODO: Prove lemmas about this *) *)
+  (* TODO: Prove lemmas about this *)
   Definition env_copy (Γ Γ' : gmap string (lty Σ)) : iProp Σ :=
     □ ∀ vs, env_ltyped Γ vs -∗ □ env_ltyped Γ' vs.
 
@@ -223,8 +221,7 @@ Definition ltyped `{!heapG Σ}
 
 Notation "Γ ⊨ e : A ⫤ Γ'" := (ltyped Γ Γ' e A)
   (at level 100, e at next level, A at level 200).
-
-Notation "Γ ⊨ e : A" := (ltyped Γ Γ e A)
+Notation "Γ ⊨ e : A" := (Γ ⊨ e : A ⫤ Γ)
   (at level 100, e at next level, A at level 200).
 
 Lemma ltyped_frame `{!heapG Σ} (Γ Γ' Γ1 Γ1' Γ2 : gmap string (lty Σ)) e A :
diff --git a/theories/logrel/types.v b/theories/logrel/types.v
index 880cedc91780049248901f41c77c90e4a5698ece..41c4c543e24cdf9632ca636729ad6d48da260aa3 100644
--- a/theories/logrel/types.v
+++ b/theories/logrel/types.v
@@ -763,7 +763,7 @@ Section properties.
     Qed.
 
     Lemma ltyped_recv Γ (x : string) A S :
-      ⊢ <[x := (chan (<??> A; S))%lty]>Γ ⊨ recv x : A ⫤ <[x:=(chan S)%lty]> Γ.
+      ⊢ <[x := (chan (<??> A; S))%lty]> Γ ⊨ recv x : A ⫤ <[x:=(chan S)%lty]> Γ.
     Proof.
       iIntros "!>" (vs) "HΓ"=> /=.
       iDestruct (env_ltyped_lookup with "HΓ") as (v' Heq) "[Hc HΓ]".