Skip to content

Commit

Permalink
state_update_inv_acc
Browse files Browse the repository at this point in the history
  • Loading branch information
hei411 committed Oct 31, 2024
1 parent 65c5d92 commit 836b0fb
Showing 1 changed file with 11 additions and 0 deletions.
11 changes: 11 additions & 0 deletions theories/coneris/wp_update.v
Original file line number Diff line number Diff line change
Expand Up @@ -559,6 +559,17 @@ Section state_update.
by iMod (inv_alloc with "[$]").
Qed.

Lemma state_update_inv_acc P E I N:
↑N ⊆ E -> inv N I -∗ (▷I -∗ state_update (E∖↑N) (P∗▷I)) -∗ state_update E P.
Proof.
iIntros (Hsubset) "#Hinv H".
iInv "Hinv" as "?" "Hclose".
iMod ("H" with "[$]") as "[??]".
iFrame. iMod ("Hclose" with "[$]") as "_".
iModIntro.
iApply fupd_mask_intro_subseteq; [set_solver|done].
Qed.

Context {A : cmra} `{i : inG Σ A}.
Lemma state_update_ra_alloc E (a:A):
✓ a -> ⊢ state_update E (∃ γ, own γ a).
Expand Down

0 comments on commit 836b0fb

Please sign in to comment.