Skip to content
Snippets Groups Projects
Commit 11c997df authored by Ralf Jung's avatar Ralf Jung
Browse files

fix remaining name mangling issues

parent 9ab7c2c7
No related branches found
No related tags found
No related merge requests found
Pipeline #52329 passed
...@@ -82,10 +82,10 @@ Section weak. ...@@ -82,10 +82,10 @@ Section weak.
Proof. Proof.
iIntros "#Hincl". iPoseProof "Hincl" as "(Hsz & #Hoincl & #Hsincl)". iIntros "#Hincl". iPoseProof "Hincl" as "(Hsz & #Hoincl & #Hsincl)".
iSplit; first done. iSplit; iModIntro. iSplit; first done. iSplit; iModIntro.
- iIntros "* Hvl". destruct vl as [|[[|vl|]|] [|]]; try done. - iIntros "%tid %vl Hvl". destruct vl as [|[[|vl|]|] [|]]; try done.
iDestruct "Hvl" as (γ ν) "(#Hpersist & Htok)". iDestruct "Hvl" as (γ ν) "(#Hpersist & Htok)".
iExists _, _. iFrame "Htok". by iApply rc_persist_type_incl. iExists _, _. iFrame "Htok". by iApply rc_persist_type_incl.
- iIntros "* #Hshr". iDestruct "Hshr" as (l') "[Hfrac Hshr]". iExists l'. - iIntros "%κ %tid %l #Hshr". iDestruct "Hshr" as (l') "[Hfrac Hshr]". iExists l'.
iIntros "{$Hfrac} !> * % Htok". iMod ("Hshr" with "[% //] Htok") as "{Hshr} H". iIntros "{$Hfrac} !> * % Htok". iMod ("Hshr" with "[% //] Htok") as "{Hshr} H".
iModIntro. iNext. iMod "H" as "[$ H]". iDestruct "H" as (γ ν) "(Hpersist & Hshr)". iModIntro. iNext. iMod "H" as "[$ H]". iDestruct "H" as (γ ν) "(Hpersist & Hshr)".
iExists _, _. iFrame "Hshr". by iApply rc_persist_type_incl. iExists _, _. iFrame "Hshr". by iApply rc_persist_type_incl.
...@@ -398,11 +398,11 @@ Section code. ...@@ -398,11 +398,11 @@ Section code.
iDestruct "Hrcproto" as ([st weakc]) "[>Hrc● Hrcst]". iDestruct "Hrcproto" as ([st weakc]) "[>Hrc● Hrcst]".
iDestruct (own_valid_2 with "Hrc● Hwtok") as iDestruct (own_valid_2 with "Hrc● Hwtok") as
%[[_ Hweak%nat_included]%prod_included [Hval _]]%auth_both_valid_discrete. %[[_ Hweak%nat_included]%prod_included [Hval _]]%auth_both_valid_discrete.
destruct weakc; first by simpl in *; lia. destruct weakc as [|weakc]; first by simpl in *; lia.
iMod (own_update_2 with "Hrc● Hwtok") as "Hrc●". iMod (own_update_2 with "Hrc● Hwtok") as "Hrc●".
{ apply auth_update_dealloc, prod_local_update_2, { apply auth_update_dealloc, prod_local_update_2,
(cancel_local_update_unit 1%nat), _. } (cancel_local_update_unit 1%nat), _. }
destruct st as [[[q'' strong]| |]|]; try done. destruct st as [[[q'' strong]| |]|]; [..|done|].
- iExists _. iDestruct "Hrcst" as (q0) "(Hlw & >$ & Hrcst)". iRight. - iExists _. iDestruct "Hrcst" as (q0) "(Hlw & >$ & Hrcst)". iRight.
iSplitR; first by auto with lia. iIntros "!>?". iApply "Hclose". iFrame. iSplitR; first by auto with lia. iIntros "!>?". iApply "Hclose". iFrame.
iExists _. iFrame. iExists _. iFrame. iExists _. iFrame. iExists _. iFrame.
......
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