Skip to content

Commit

Permalink
use invGS_gen
Browse files Browse the repository at this point in the history
  • Loading branch information
tjhance committed Feb 12, 2025
1 parent 5eb5f70 commit 68d7971
Show file tree
Hide file tree
Showing 11 changed files with 14 additions and 14 deletions.
2 changes: 1 addition & 1 deletion src/examples/counting.v
Original file line number Diff line number Diff line change
Expand Up @@ -107,7 +107,7 @@ Section Counting.

Context {Σ: gFunctors}.
Context `{co_in_Σ: !@co_logicG Σ}.
Context `{!invGS Σ}.
Context `{!invGS_gen hlc Σ}.

Fixpoint sep_pow (n: nat) (P: iProp Σ) : iProp Σ :=
match n with
Expand Down
2 changes: 1 addition & 1 deletion src/examples/forever.v
Original file line number Diff line number Diff line change
Expand Up @@ -147,7 +147,7 @@ Section Forever.

Context {Σ: gFunctors}.
Context `{f_in_Σ: @forever_logicG Σ}.
Context `{!invGS Σ}.
Context `{!invGS_gen hlc Σ}.

Definition family (Q: iProp Σ) (e: Exc ()) : iProp Σ :=
match e with
Expand Down
2 changes: 1 addition & 1 deletion src/examples/fractional.v
Original file line number Diff line number Diff line change
Expand Up @@ -348,7 +348,7 @@ Proof. solve_inG. Qed.
Section Frac.
Context {Σ: gFunctors}.
Context `{@frac_logicG Σ}.
Context `{!invGS Σ}.
Context `{!invGS_gen hlc Σ}.

Definition sto_frac (γ: gname) (Q: iProp Σ) := sp_sto (sp_i := frac_sp_inG) γ (family Q).
Definition own_frac (γ: gname) (qp: Qp) := sp_own (sp_i := frac_sp_inG) γ (Some qp).
Expand Down
2 changes: 1 addition & 1 deletion src/examples/hash_table_logic.v
Original file line number Diff line number Diff line change
Expand Up @@ -66,7 +66,7 @@ Section HashTableLogic.

Context {Σ: gFunctors}.
Context {htl: ht_logicG Σ}.
Context `{!invGS Σ}.
Context `{!invGS_gen hlc Σ}.

Lemma ht_Init (n: nat) :
⊢ |==> (∃ γ , own γ (mseq n) ∗ own γ (sseq ht_fixed_size))%I.
Expand Down
2 changes: 1 addition & 1 deletion src/guarding/guard_later_pers.v
Original file line number Diff line number Diff line change
Expand Up @@ -72,7 +72,7 @@ Proof.
Qed.

Context {Σ: gFunctors}.
Context `{!invGS Σ}.
Context `{!invGS_gen hlc Σ}.

(* Later-Pers-Guard *)

Expand Down
2 changes: 1 addition & 1 deletion src/guarding/lib/cancellable.v
Original file line number Diff line number Diff line change
Expand Up @@ -29,7 +29,7 @@ Section CancellableInvariants.

Context {Σ: gFunctors}.
Context `{!ecInv_logicG Σ}.
Context `{!invGS Σ}.
Context `{!invGS_gen hlc Σ}.

Definition Active (γ: gname) : iProp Σ := own γ (Excl ()).

Expand Down
6 changes: 3 additions & 3 deletions src/guarding/lib/lifetime.v
Original file line number Diff line number Diff line change
Expand Up @@ -147,7 +147,7 @@ Qed.
Section LlftHelperResources.
Context {Σ: gFunctors}.
Context `{!llft_logicGpreS Σ}.
Context `{!invGS Σ}.
Context `{!invGS_gen hlc Σ}.

(* begin hide *)

Expand Down Expand Up @@ -538,7 +538,7 @@ End LlftHelperResources.
Section LlftLogic.
Context {Σ: gFunctors}.
Context `{!llft_logicGS Σ}.
Context `{!invGS Σ}.
Context `{!invGS_gen hlc Σ}.

(*** Lifetime logic ***)

Expand Down Expand Up @@ -867,7 +867,7 @@ Section LlftLogic.
Qed.
End LlftLogic.

Lemma llft_alloc {Σ: gFunctors} `{!llft_logicGpreS Σ} `{!invGS Σ} E
Lemma llft_alloc {Σ: gFunctors} `{!llft_logicGpreS Σ} `{!invGS_gen hlc Σ} E
: ⊢ |={E}=> ∃ _ : llft_logicGS Σ, llft_ctx.
Proof.
iIntros. iMod lt_alloc as (γ) "J".
Expand Down
2 changes: 1 addition & 1 deletion src/guarding/lib/non_atomic_map.v
Original file line number Diff line number Diff line change
Expand Up @@ -285,7 +285,7 @@ Section NonAtomicMap.

Context {Σ: gFunctors}.
Context `{!na_logicG L V Σ}.
Context `{!invGS Σ}.
Context `{!invGS_gen hlc Σ}.

Implicit Types (γ: gname) (l: L) (v: V).
Implicit Types (G: iProp Σ).
Expand Down
2 changes: 1 addition & 1 deletion src/guarding/lib/rwlock.v
Original file line number Diff line number Diff line change
Expand Up @@ -354,7 +354,7 @@ Context {eqdec: EqDecision S}.

Context {Σ: gFunctors}.
Context `{@rwlock_logicG S _ Σ}.
Context `{!invGS Σ}.
Context `{!invGS_gen hlc Σ}.

Definition fields γ (e: bool) (r: Z) (x: S) : iProp Σ
:= sp_own (sp_i := rwlock_sp_inG) γ (Central e r x).
Expand Down
2 changes: 1 addition & 1 deletion src/guarding/storage_protocol/protocol.v
Original file line number Diff line number Diff line change
Expand Up @@ -366,7 +366,7 @@ Section StorageLogic.

Context {Σ: gFunctors}.
Context `{sp_i: !sp_logicG storage_mixin Σ}.
Context `{!invGS Σ}.
Context `{!invGS_gen hlc Σ}.

Definition sp_sto (γ: gname) (f: B → iProp Σ) : iProp Σ :=
⌜ wf_prop_map f ⌝ ∗
Expand Down
4 changes: 2 additions & 2 deletions src/guarding/tactics.v
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@ From iris.prelude Require Import options.
Section TacticsHelpers.

Context {Σ: gFunctors}.
Context `{!invGS_gen hlc Σ}.
Context `{!invGS_gen hlc Σ}.

Local Lemma guard_weaken_helper_right (A B C : iProp Σ) (E: coPset) (n: nat)
: (A &&{E; n}&&> B) -∗ (B &&{E}&&> C) -∗ (A &&{E; n}&&> C).
Expand Down Expand Up @@ -133,7 +133,7 @@ Tactic Notation "leaf_open_laters" constr(g) "with" constr(sel) "as" constr(pat)
Section TacticsTests.

Context {Σ: gFunctors}.
Context `{!invGS Σ}.
Context `{!invGS_gen hlc Σ}.

Local Lemma test_leaf_hyp (A B C D : iProp Σ) E
: (A &&{∅ ; 3}&&> B ∗ C) ⊢ (A ∗ D &&{E ; 20}&&> B).
Expand Down

0 comments on commit 68d7971

Please sign in to comment.