diff --git a/theories/lifetime/frac_borrow.v b/theories/lifetime/frac_borrow.v index d144e141205355fe41afa0e7646d1d3222efd2ab..18e3a41fe22f6db52d8efa8eea379ddecdb6146d 100644 --- a/theories/lifetime/frac_borrow.v +++ b/theories/lifetime/frac_borrow.v @@ -26,11 +26,12 @@ Section frac_bor. Global Instance frac_bor_proper κ : Proper (pointwise_relation _ (⊣⊢) ==> (⊣⊢)) (frac_bor κ). Proof. solve_proper. Qed. - Lemma frac_bor_iff_proper κ φ' : + + Lemma frac_bor_iff κ φ' : ▷ □ (∀ q, φ q ↔ φ' q) -∗ &frac{κ} φ -∗ &frac{κ} φ'. Proof. iIntros "#Hφφ' H". iDestruct "H" as (γ κ') "[? Hφ]". iExists γ, κ'. iFrame. - iApply (shr_bor_iff_proper with "[Hφφ'] Hφ"). iNext. iAlways. + iApply (shr_bor_iff with "[Hφφ'] Hφ"). iNext. iAlways. iSplit; iIntros "H"; iDestruct "H" as (q) "[H ?]"; iExists q; iFrame; by iApply "Hφφ'". Qed. diff --git a/theories/lifetime/lifetime_sig.v b/theories/lifetime/lifetime_sig.v index 0da0470f90ccedc80cfc33e2d9fb6934eff12154..855e9a7f4d8168eee60e9ac8c4cb3a6da6e21504 100644 --- a/theories/lifetime/lifetime_sig.v +++ b/theories/lifetime/lifetime_sig.v @@ -67,11 +67,9 @@ Module Type lifetime_sig. Global Declare Instance bor_ne κ n : Proper (dist n ==> dist n) (bor κ). Global Declare Instance bor_contractive κ : Contractive (bor κ). Global Declare Instance bor_proper κ : Proper ((≡) ==> (≡)) (bor κ). - Parameter bor_iff_proper : ∀ κ P P', ▷ □ (P ↔ P') -∗ &{κ}P -∗ &{κ}P'. Global Declare Instance idx_bor_ne κ i n : Proper (dist n ==> dist n) (idx_bor κ i). Global Declare Instance idx_bor_contractive κ i : Contractive (idx_bor κ i). Global Declare Instance idx_bor_proper κ i : Proper ((≡) ==> (≡)) (idx_bor κ i). - Parameter idx_bor_iff_proper : ∀ κ i P P', ▷ □ (P ↔ P') -∗ &{κ,i}P -∗ &{κ,i}P'. Global Declare Instance lft_tok_fractional κ : Fractional (λ q, q.[κ])%I. Global Declare Instance lft_tok_as_fractional κ q : @@ -94,20 +92,24 @@ Module Type lifetime_sig. Parameter bor_fake : ∀ E κ P, ↑lftN ⊆ E → lft_ctx -∗ [†κ] ={E}=∗ &{κ}P. + Parameter bor_iff : ∀ κ P P', ▷ □ (P ↔ P') -∗ &{κ}P -∗ &{κ}P'. + Parameter bor_shorten : ∀ κ κ' P, κ ⊑ κ' -∗ &{κ'}P -∗ &{κ}P. + Parameter bor_sep : ∀ E κ P Q, ↑lftN ⊆ E → lft_ctx -∗ &{κ} (P ∗ Q) ={E}=∗ &{κ} P ∗ &{κ} Q. Parameter bor_combine : ∀ E κ P Q, ↑lftN ⊆ E → lft_ctx -∗ &{κ} P -∗ &{κ} Q ={E}=∗ &{κ} (P ∗ Q). - Parameter bor_unfold_idx : ∀ κ P, &{κ}P ⊣⊢ ∃ i, &{κ,i}P ∗ idx_bor_own 1 i. - Parameter bor_shorten : ∀ κ κ' P, κ ⊑ κ' -∗ &{κ'}P -∗ &{κ}P. - Parameter idx_bor_shorten : ∀ κ κ' i P, κ ⊑ κ' -∗ &{κ',i} P -∗ &{κ,i} P. - Parameter rebor : ∀ E κ κ' P, ↑lftN ⊆ E → lft_ctx -∗ κ' ⊑ κ -∗ &{κ}P ={E}=∗ &{κ'}P ∗ ([†κ'] ={E}=∗ &{κ}P). Parameter bor_unnest : ∀ E κ κ' P, ↑lftN ⊆ E → lft_ctx -∗ &{κ'} &{κ} P ={E, E∖↑lftN}▷=∗ &{κ ∪ κ'} P. + Parameter bor_unfold_idx : ∀ κ P, &{κ}P ⊣⊢ ∃ i, &{κ,i}P ∗ idx_bor_own 1 i. + + Parameter idx_bor_shorten : ∀ κ κ' i P, κ ⊑ κ' -∗ &{κ',i} P -∗ &{κ,i} P. + Parameter idx_bor_iff : ∀ κ i P P', ▷ □ (P ↔ P') -∗ &{κ,i}P -∗ &{κ,i}P'. + Parameter idx_bor_acc : ∀ E q κ i P, ↑lftN ⊆ E → lft_ctx -∗ &{κ,i}P -∗ idx_bor_own 1 i -∗ q.[κ] ={E}=∗ ▷ P ∗ (▷ P ={E}=∗ idx_bor_own 1 i ∗ q.[κ]). diff --git a/theories/lifetime/model/primitive.v b/theories/lifetime/model/primitive.v index b7e5bb904aeb2997c0b65321230259da640fc356..530324b135bfcad069f7716f1356c59c769b1e25 100644 --- a/theories/lifetime/model/primitive.v +++ b/theories/lifetime/model/primitive.v @@ -373,7 +373,7 @@ Lemma lft_incl_intro κ κ' : Proof. reflexivity. Qed. (** Basic rules about borrows *) -Lemma raw_bor_iff_proper i P P' : ▷ □ (P ↔ P') -∗ raw_bor i P -∗ raw_bor i P'. +Lemma raw_bor_iff i P P' : ▷ □ (P ↔ P') -∗ raw_bor i P -∗ raw_bor i P'. Proof. iIntros "#HPP' HP". unfold raw_bor. iDestruct "HP" as (s) "[HiP HP]". iExists s. iFrame. iDestruct "HP" as (P0) "[#Hiff ?]". iExists P0. iFrame. @@ -381,7 +381,7 @@ Proof. by iApply "HPP'"; iApply "Hiff". by iApply "Hiff"; iApply "HPP'". Qed. -Lemma idx_bor_iff_proper κ i P P' : ▷ □ (P ↔ P') -∗ &{κ,i}P -∗ &{κ,i}P'. +Lemma idx_bor_iff κ i P P' : ▷ □ (P ↔ P') -∗ &{κ,i}P -∗ &{κ,i}P'. Proof. unfold idx_bor. iIntros "#HPP' [$ HP]". iDestruct "HP" as (P0) "[#HP0P Hs]". iExists P0. iFrame. iNext. iAlways. iSplit; iIntros. @@ -397,10 +397,10 @@ Proof. iExists κ'. iFrame. iExists s. by iFrame. Qed. -Lemma bor_iff_proper κ P P' : ▷ □ (P ↔ P') -∗ &{κ}P -∗ &{κ}P'. +Lemma bor_iff κ P P' : ▷ □ (P ↔ P') -∗ &{κ}P -∗ &{κ}P'. Proof. rewrite !bor_unfold_idx. iIntros "#HPP' HP". iDestruct "HP" as (i) "[??]". - iExists i. iFrame. by iApply (idx_bor_iff_proper with "HPP'"). + iExists i. iFrame. by iApply (idx_bor_iff with "HPP'"). Qed. Lemma bor_shorten κ κ' P : κ ⊑ κ' -∗ &{κ'}P -∗ &{κ}P. diff --git a/theories/lifetime/model/raw_reborrow.v b/theories/lifetime/model/raw_reborrow.v index a3be4ed65b6f4395c5d219c2b6ece89ee92698e5..7f8c891cb6d8480dc34525300daf6755a4b6ad4b 100644 --- a/theories/lifetime/model/raw_reborrow.v +++ b/theories/lifetime/model/raw_reborrow.v @@ -133,7 +133,7 @@ Proof. iIntros "[$ [>? $]]". iModIntro. iNext. rewrite /raw_bor. iExists i. iFrame. iExists _. iFrame "#". } iExists Pb'. iModIntro. iFrame. iSplitL "Hclose Hκ". by iApply "Hclose". - by iApply (raw_bor_iff_proper with "HPP'"). + by iApply (raw_bor_iff with "HPP'"). Qed. Lemma raw_rebor E κ κ' P : @@ -171,7 +171,7 @@ Proof. with "[$HI $Hκ] Hi Hislice Hbor [Hvs]") as (Pb') "([HI Hκ] & HP' & Halive & Hvs)"; [solve_ndisj|done|done|..]. { iNext. by iApply lft_vs_frame. } - iDestruct (raw_bor_iff_proper with "HPP' HP'") as "$". + iDestruct (raw_bor_iff with "HPP' HP'") as "$". iDestruct ("Hκclose" with "Hκ") as "Hinv". iMod ("Hclose" with "[HA HI Hinv Halive Hinh Hvs]") as "_". { iNext. rewrite {2}/lfts_inv. iExists A, I. iFrame "HA HI". diff --git a/theories/lifetime/na_borrow.v b/theories/lifetime/na_borrow.v index 0c59478bce14d1d268c469c0e9ec3fae1081f832..78a7bb2dffa60292af019ad00c038d53e4305a00 100644 --- a/theories/lifetime/na_borrow.v +++ b/theories/lifetime/na_borrow.v @@ -20,11 +20,12 @@ Section na_bor. Proof. solve_contractive. Qed. Global Instance na_bor_proper κ : Proper ((⊣⊢) ==> (⊣⊢)) (na_bor κ tid N). Proof. solve_proper. Qed. - Lemma na_bor_iff_proper κ P' : + + Lemma na_bor_iff κ P' : ▷ □ (P ↔ P') -∗ &na{κ, tid, N} P -∗ &na{κ, tid, N} P'. Proof. iIntros "HPP' H". iDestruct "H" as (i) "[HP ?]". iExists i. iFrame. - iApply (idx_bor_iff_proper with "HPP' HP"). + iApply (idx_bor_iff with "HPP' HP"). Qed. Global Instance na_bor_persistent κ : PersistentP (&na{κ,tid,N} P) := _. diff --git a/theories/lifetime/shr_borrow.v b/theories/lifetime/shr_borrow.v index d4984e204b2f5e46cc6a09e6cf5307a41f350dfa..2f7020a53cc5a5e77217e459783d404d0d34e0a1 100644 --- a/theories/lifetime/shr_borrow.v +++ b/theories/lifetime/shr_borrow.v @@ -18,10 +18,11 @@ Section shared_bors. Proof. solve_contractive. Qed. Global Instance shr_bor_proper : Proper ((⊣⊢) ==> (⊣⊢)) (shr_bor κ). Proof. solve_proper. Qed. - Lemma shr_bor_iff_proper κ P' : ▷ □ (P ↔ P') -∗ &shr{κ} P -∗ &shr{κ} P'. + + Lemma shr_bor_iff κ P' : ▷ □ (P ↔ P') -∗ &shr{κ} P -∗ &shr{κ} P'. Proof. iIntros "HPP' H". iDestruct "H" as (i) "[HP ?]". iExists i. iFrame. - iApply (idx_bor_iff_proper with "HPP' HP"). + iApply (idx_bor_iff with "HPP' HP"). Qed. Global Instance shr_bor_persistent : PersistentP (&shr{κ} P) := _. diff --git a/theories/typing/uniq_bor.v b/theories/typing/uniq_bor.v index 8680f75dab080dddd3e4e7da492957397ee4aaef..8cf7c469864acc782cf3683b3350c7d51a69bd64 100644 --- a/theories/typing/uniq_bor.v +++ b/theories/typing/uniq_bor.v @@ -64,7 +64,7 @@ Section uniq_bor. iDestruct (Hty with "* [] [] []") as "(_ & #Ho & #Hs)"; [done..|clear Hty]. iDestruct (Hκ with "[] []") as "#Hκ"; [done..|]. iSplit; iAlways. - iIntros (? [|[[]|][]]) "H"; try iDestruct "H" as "[]". - iApply (bor_shorten with "Hκ"). iApply bor_iff_proper; last done. + iApply (bor_shorten with "Hκ"). iApply bor_iff; last done. iSplit; iIntros "!>!# H"; iDestruct "H" as (vl) "[??]"; iExists vl; iFrame; by iApply "Ho". - iIntros (κ ??) "H". iAssert (κ2 ∪ κ ⊑ κ1 ∪ κ)%I as "#Hincl'". @@ -96,7 +96,7 @@ Section uniq_bor. Send ty → Send (uniq_bor κ ty). Proof. iIntros (Hsend tid1 tid2 [|[[]|][]]) "H"; try iDestruct "H" as "[]". - iApply bor_iff_proper; last done. iNext. iAlways. iApply uPred.equiv_iff. + iApply bor_iff; last done. iNext. iAlways. iApply uPred.equiv_iff. do 3 f_equiv. iSplit; iIntros "."; by iApply Hsend. Qed. diff --git a/theories/typing/unsafe/cell.v b/theories/typing/unsafe/cell.v index 240459f647501f5e2765f8aba59c092db30168e2..f457b22178264ded0594d4b71b017bd9f5cfcd3f 100644 --- a/theories/typing/unsafe/cell.v +++ b/theories/typing/unsafe/cell.v @@ -34,7 +34,7 @@ Section cell. iDestruct (EQ with "LFT HE HL") as "(% & #Hown & #Hshr)". iSplit; [done|iSplit; iIntros "!# * H"]. - iApply ("Hown" with "H"). - - iApply na_bor_iff_proper; last done. iSplit; iIntros "!>!# H"; + - iApply na_bor_iff; last done. iSplit; iIntros "!>!# H"; iDestruct "H" as (vl) "[??]"; iExists vl; iFrame; by iApply "Hown". Qed. Lemma cell_mono' E L ty1 ty2 : eqtype E L ty1 ty2 → subtype E L (cell ty1) (cell ty2). diff --git a/theories/typing/unsafe/refcell.v b/theories/typing/unsafe/refcell.v index 52682739a07ceb2c642f7e89391d5cd2d6dff7c1..33f59031f53bc0ed9b33cc19762e3019850f3cdc 100644 --- a/theories/typing/unsafe/refcell.v +++ b/theories/typing/unsafe/refcell.v @@ -23,7 +23,7 @@ Definition reading_st (q : frac) (κ : lft) : refcell_stR := Some (Cinr (to_agree (κ : leibnizC lft), q, xH)). Definition writing_st : refcell_stR := Some (Cinl (Excl ())). -Definition refcellN := nroot .@ "refcell". +Definition refcellN := lrustN .@ "refcell". Definition refcell_invN := refcellN .@ "inv". Section refcell_inv. @@ -59,7 +59,7 @@ Section refcell_inv. iAssert (□ (&{α1} shift_loc l 1 ↦∗: ty_own ty1 tid -∗ &{α2} shift_loc l 1 ↦∗: ty_own ty2 tid))%I with "[]" as "#Hb". { iIntros "!# H". iApply (bor_shorten with "[]"). by iApply Hα. - iApply bor_iff_proper; last done. + iApply bor_iff; last done. iSplit; iIntros "!>!#H"; iDestruct "H" as (vl) "[Hf H]"; iExists vl; iFrame; by iApply "Hown". } iDestruct "H" as (st) "H"; iExists st; @@ -86,7 +86,7 @@ Section refcell. (∃ α γ, κ ⊑ α ∗ &na{α, tid, refcell_invN}(refcell_inv tid l γ α ty))%I |}. Next Obligation. iIntros (??[|[[]|]]); try iIntros "[]". rewrite ty_size_eq. - iIntros "[_ %]!%/=". congruence. + iIntros "[_ %] !% /=". congruence. Qed. Next Obligation. iIntros (ty E κ l tid q ?) "#LFT Hb Htok". @@ -154,7 +154,7 @@ Section refcell. - iPureIntro. simpl. congruence. - destruct vl as [|[[]|]]; try done. iDestruct "H" as "[$ H]". by iApply "Hown". - iDestruct "H" as (a γ) "[Ha H]". iExists a, γ. iFrame. - iApply na_bor_iff_proper; last done. + iApply na_bor_iff; last done. iSplit; iIntros "!>!# H"; by iApply refcell_inv_proper. Qed. Lemma refcell_mono' E L ty1 ty2 : @@ -360,7 +360,7 @@ Section refmut. - iIntros (tid [|[[]|][|[[]|][]]]); try iIntros "[]". iIntros "H". iDestruct "H" as (γ β ty') "(Hb & #H⊑ & #Hinv & Hown)". iExists γ, β, ty'. iFrame "∗#". iSplit. - + iApply bor_iff_proper; last done. + + iApply bor_iff; last done. iSplit; iIntros "!>!# H"; iDestruct "H" as (vl) "[??]"; iExists vl; iFrame; by iApply "Ho". + by iApply lft_incl_trans.