Skip to content
Snippets Groups Projects
Commit 4c689e94 authored by Yusuke Matsushita's avatar Yusuke Matsushita
Browse files

Minor tweaks

parent 7ce083ee
No related branches found
No related tags found
No related merge requests found
Pipeline #63441 passed
...@@ -230,7 +230,7 @@ Notation "⟨ π , φ ⟩" := (proph_obs (λ π, φ%type%stdpp)) ...@@ -230,7 +230,7 @@ Notation "⟨ π , φ ⟩" := (proph_obs (λ π, φ%type%stdpp))
(** * Iris Lemmas *) (** * Iris Lemmas *)
Section lemmas. Section proph.
Context `{!invG Σ, !prophG Σ}. Context `{!invG Σ, !prophG Σ}.
(** Instances *) (** Instances *)
...@@ -419,7 +419,7 @@ Proof. ...@@ -419,7 +419,7 @@ Proof.
iMod (proph_obs_sat with "PROPH Obs") as %[? Ex]; [done|]. by apply Neg in Ex. iMod (proph_obs_sat with "PROPH Obs") as %[? Ex]; [done|]. by apply Neg in Ex.
Qed. Qed.
End lemmas. End proph.
Global Opaque proph_ctx proph_tok proph_obs. Global Opaque proph_ctx proph_tok proph_obs.
...@@ -430,7 +430,7 @@ Definition proph_eqz `{!invG Σ, !prophG Σ} {A} (uπ vπ: proph A) : iProp Σ : ...@@ -430,7 +430,7 @@ Definition proph_eqz `{!invG Σ, !prophG Σ} {A} (uπ vπ: proph A) : iProp Σ :
Notation "uπ :== vπ" := (proph_eqz ) (at level 70, format "uπ :== vπ") : bi_scope. Notation "uπ :== vπ" := (proph_eqz ) (at level 70, format "uπ :== vπ") : bi_scope.
Section lemmas. Section proph_eqz.
Context `{!invG Σ, !prophG Σ}. Context `{!invG Σ, !prophG Σ}.
(** ** Constructing Prophecy Equalizers *) (** ** Constructing Prophecy Equalizers *)
...@@ -499,4 +499,4 @@ Proof. ...@@ -499,4 +499,4 @@ Proof.
iIntros "Eqz". rewrite !vapply_insert_backmid. iIntros "Eqz". rewrite !vapply_insert_backmid.
iApply (proph_eqz_constr3 with "[] Eqz []"); iApply proph_eqz_refl. iApply (proph_eqz_constr3 with "[] Eqz []"); iApply proph_eqz_refl.
Qed. Qed.
End lemmas. End proph_eqz.
...@@ -5,7 +5,7 @@ Set Default Proof Using "Type". ...@@ -5,7 +5,7 @@ Set Default Proof Using "Type".
Implicit Type 𝔄: syn_type. Implicit Type 𝔄: syn_type.
Section lemmas. Section array_idx.
Context `{!typeG Σ}. Context `{!typeG Σ}.
(** * Owning Pointers *) (** * Owning Pointers *)
...@@ -267,7 +267,7 @@ Section lemmas. ...@@ -267,7 +267,7 @@ Section lemmas.
iApply type_let; [by apply type_idx_uniq_array_instr|solve_typing| |done]. iApply type_let; [by apply type_idx_uniq_array_instr|solve_typing| |done].
move: Ex=> [Htrx _]?. apply Htrx. by case=> [?[??]]. move: Ex=> [Htrx _]?. apply Htrx. by case=> [?[??]].
Qed. Qed.
End lemmas. End array_idx.
Global Hint Resolve tctx_extract_split_own_array Global Hint Resolve tctx_extract_split_own_array
tctx_extract_idx_shr_array tctx_extract_split_uniq_array | 5 : lrust_typing. tctx_extract_idx_shr_array tctx_extract_split_uniq_array | 5 : lrust_typing.
......
...@@ -133,7 +133,7 @@ End fix_defs. ...@@ -133,7 +133,7 @@ End fix_defs.
Import fix_defs. Import fix_defs.
Global Notation fix_ty := fix_ty. Global Notation fix_ty := fix_ty.
Section lemmas. Section fix_ty.
Context `{!typeG Σ}. Context `{!typeG Σ}.
Lemma fix_unfold_fold {𝔄} (T: type 𝔄 type 𝔄) {HT: TypeContractive T} E L : Lemma fix_unfold_fold {𝔄} (T: type 𝔄 type 𝔄) {HT: TypeContractive T} E L :
...@@ -244,9 +244,9 @@ Section lemmas. ...@@ -244,9 +244,9 @@ Section lemmas.
- move=> *. etrans; [apply conv_compl|]. - move=> *. etrans; [apply conv_compl|].
etrans; [|symmetry; apply conv_compl]. by apply Hne. etrans; [|symmetry; apply conv_compl]. by apply Hne.
Qed. Qed.
End lemmas. End fix_ty.
Section lemmas. Section fix_ty.
Context `{!typeG Σ} {𝔄} (T: type 𝔄 type 𝔄) {HT: TypeContractive T}. Context `{!typeG Σ} {𝔄} (T: type 𝔄 type 𝔄) {HT: TypeContractive T}.
Global Instance fix_copy : Global Instance fix_copy :
...@@ -302,9 +302,9 @@ Section lemmas. ...@@ -302,9 +302,9 @@ Section lemmas.
apply limit_preserving_entails; [done|]=> ??? Eq; apply limit_preserving_entails; [done|]=> ??? Eq;
do 3 f_equiv; [apply Eq|]; do 5 f_equiv); [|do 2 f_equiv]; apply Eq. do 3 f_equiv; [apply Eq|]; do 5 f_equiv); [|do 2 f_equiv]; apply Eq.
Qed. Qed.
End lemmas. End fix_ty.
Section subtyping. Section fix_subtyping.
Context `{!typeG Σ}. Context `{!typeG Σ}.
Local Lemma wand_forall P (Φ: nat iProp Σ) : (n, P -∗ Φ n) (P -∗ n, Φ n). Local Lemma wand_forall P (Φ: nat iProp Σ) : (n, P -∗ Φ n) (P -∗ n, Φ n).
...@@ -390,7 +390,7 @@ Section subtyping. ...@@ -390,7 +390,7 @@ Section subtyping.
Proof. Proof.
move=> ?. eapply (eqtype_trans _ _ _ id id); [|done]. apply fix_unfold_fold. move=> ?. eapply (eqtype_trans _ _ _ id id); [|done]. apply fix_unfold_fold.
Qed. Qed.
End subtyping. End fix_subtyping.
Global Hint Resolve fix_subtype_l fix_subtype_r fix_eqtype_l fix_eqtype_r | 100 Global Hint Resolve fix_subtype_l fix_subtype_r fix_eqtype_l fix_eqtype_r | 100
: lrust_typing. : lrust_typing.
0% Loading or .
You are about to add 0 people to the discussion. Proceed with caution.
Please register or to comment