Skip to content
Snippets Groups Projects
Commit e5840151 authored by Jonas Kastberg's avatar Jonas Kastberg
Browse files

Nits

parent 9f957e7c
No related branches found
No related tags found
1 merge request!8Algorithmic Typing Judgement
...@@ -103,7 +103,7 @@ Section Environment. ...@@ -103,7 +103,7 @@ Section Environment.
Qed. Qed.
Definition env_split (Γ Γ1 Γ2 : gmap string (lty Σ)) : iProp Σ := 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 Γ Γ. Lemma env_split_id_l Γ : env_split Γ Γ.
Proof. Proof.
...@@ -119,9 +119,7 @@ Section Environment. ...@@ -119,9 +119,7 @@ Section Environment.
Lemma env_split_empty : env_split ∅. Lemma env_split_empty : env_split ∅.
Proof. Proof.
iIntros "!>" (vs). iIntros "!>" (vs).
iSplit. iSplit; [iIntros "HΓ" | iIntros "[HΓ1 HΓ2]"]; auto.
- iIntros "HΓ". rewrite /env_ltyped. auto.
- iIntros "[HΓ1 HΓ2]". auto.
Qed. Qed.
(* TODO: Get rid of side condition that x does not appear in Γ1 *) (* TODO: Get rid of side condition that x does not appear in Γ1 *)
...@@ -183,7 +181,7 @@ Section Environment. ...@@ -183,7 +181,7 @@ Section Environment.
iApply "Hsplit". iFrame "HΓ1 HΓ2". iApply "Hsplit". iFrame "HΓ1 HΓ2".
Qed. Qed.
(* (* TODO: Prove lemmas about this *) *) (* TODO: Prove lemmas about this *)
Definition env_copy (Γ Γ' : gmap string (lty Σ)) : iProp Σ := Definition env_copy (Γ Γ' : gmap string (lty Σ)) : iProp Σ :=
vs, env_ltyped Γ vs -∗ env_ltyped Γ' vs. vs, env_ltyped Γ vs -∗ env_ltyped Γ' vs.
...@@ -223,8 +221,7 @@ Definition ltyped `{!heapG Σ} ...@@ -223,8 +221,7 @@ Definition ltyped `{!heapG Σ}
Notation "Γ ⊨ e : A ⫤ Γ'" := (ltyped Γ Γ' e A) Notation "Γ ⊨ e : A ⫤ Γ'" := (ltyped Γ Γ' e A)
(at level 100, e at next level, A at level 200). (at level 100, e at next level, A at level 200).
Notation "Γ ⊨ e : A" := (Γ e : A Γ)
Notation "Γ ⊨ e : A" := (ltyped Γ Γ e A)
(at level 100, e at next level, A at level 200). (at level 100, e at next level, A at level 200).
Lemma ltyped_frame `{!heapG Σ} (Γ Γ' Γ1 Γ1' Γ2 : gmap string (lty Σ)) e A : Lemma ltyped_frame `{!heapG Σ} (Γ Γ' Γ1 Γ1' Γ2 : gmap string (lty Σ)) e A :
......
...@@ -763,7 +763,7 @@ Section properties. ...@@ -763,7 +763,7 @@ Section properties.
Qed. Qed.
Lemma ltyped_recv Γ (x : string) A S : 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. Proof.
iIntros "!>" (vs) "HΓ"=> /=. iIntros "!>" (vs) "HΓ"=> /=.
iDestruct (env_ltyped_lookup with "HΓ") as (v' Heq) "[Hc HΓ]". iDestruct (env_ltyped_lookup with "HΓ") as (v' Heq) "[Hc HΓ]".
......
0% Loading or .
You are about to add 0 people to the discussion. Proceed with caution.
Finish editing this message first!
Please register or to comment