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

proof style nits

parent c6d98043
No related branches found
No related tags found
No related merge requests found
Pipeline #28213 passed
...@@ -98,7 +98,7 @@ Proof. ...@@ -98,7 +98,7 @@ Proof.
as %[EQB2%to_borUR_included _]%auth_both_valid. as %[EQB2%to_borUR_included _]%auth_both_valid.
iAssert j1 j2⌝%I with "[#]" as %Hj1j2. iAssert j1 j2⌝%I with "[#]" as %Hj1j2.
{ iDestruct (own_bor_valid_2 with "Hbor1 Hbor2") as %Hj1j2%auth_valid_discrete. { iDestruct (own_bor_valid_2 with "Hbor1 Hbor2") as %Hj1j2%auth_valid_discrete.
iPureIntro. iIntros (->). (* FIXME this used to work without iPureIntro. *) iIntros (->).
exfalso. revert Hj1j2. rewrite /= singleton_op singleton_valid. exfalso. revert Hj1j2. rewrite /= singleton_op singleton_valid.
by intros [[]]. } by intros [[]]. }
iMod (slice_combine _ _ true with "Hslice1 Hslice2 Hbox") iMod (slice_combine _ _ true with "Hslice1 Hslice2 Hbox")
......
...@@ -184,13 +184,13 @@ Section borrow. ...@@ -184,13 +184,13 @@ Section borrow.
{ iApply (lft_incl_glb with "Hincl []"). iApply lft_incl_refl. } { iApply (lft_incl_glb with "Hincl []"). iApply lft_incl_refl. }
iMod (lft_incl_acc with "Hincl' Htok2") as (q2) "[Htok2 Hclose'']"; first solve_ndisj. iMod (lft_incl_acc with "Hincl' Htok2") as (q2) "[Htok2 Hclose'']"; first solve_ndisj.
iApply (wp_step_fupd _ _ (_∖_) with "[Hown Htok2]"); try done. iApply (wp_step_fupd _ _ (_∖_) with "[Hown Htok2]"); try done.
- iApply ("Hown" with "[%] Htok2"); first solve_ndisj. { iApply ("Hown" with "[%] Htok2"); first solve_ndisj. }
- iApply wp_fupd. wp_read. iIntros "!>[#Hshr Htok2]". iApply wp_fupd. wp_read. iIntros "!>[#Hshr Htok2]".
iMod ("Hclose''" with "Htok2") as "Htok2". iMod ("Hclose''" with "Htok2") as "Htok2".
iMod ("Hclose'" with "[H↦]") as "Htok1"; first by auto. iMod ("Hclose'" with "[H↦]") as "Htok1"; first by auto.
iMod ("Hclose" with "[Htok1 Htok2]") as "($ & $)"; first by iFrame. iMod ("Hclose" with "[Htok1 Htok2]") as "($ & $)"; first by iFrame.
rewrite tctx_interp_singleton tctx_hasty_val' //. rewrite tctx_interp_singleton tctx_hasty_val' //.
by iApply (ty_shr_mono with "Hincl' Hshr"). by iApply (ty_shr_mono with "Hincl' Hshr").
Qed. Qed.
Lemma type_deref_shr_uniq {E L} κ κ' x p e ty C T T' : Lemma type_deref_shr_uniq {E L} κ κ' x p e ty C T T' :
......
0% Loading or .
You are about to add 0 people to the discussion. Proceed with caution.
Please register or to comment