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

tune proofs a little

parent d0733ad8
No related branches found
No related tags found
No related merge requests found
...@@ -112,12 +112,9 @@ Proof. ...@@ -112,12 +112,9 @@ Proof.
iIntros {???} "[#Hvs1 [#Hvs2 #Hwp]] ! [HR HP]". iIntros {???} "[#Hvs1 [#Hvs2 #Hwp]] ! [HR HP]".
iApply (wp_frame_step_l E E1 E2); try done. iApply (wp_frame_step_l E E1 E2); try done.
iSplitL "HR". iSplitL "HR".
- (* TODO: Is there a way to do "apply Hvs1 in Hr"? *) - iPvs "Hvs1" "HR" as "HR"; first by set_solver.
iPvs "Hvs1" "HR"; first by set_solver. iPvsIntro. iNext. iPvs "Hvs2" "HR" as "HR"; first by set_solver.
(* TODO: iApply pvs_intro? *) iPvsIntro. iApply "HR".
rewrite -pvs_intro.
iNext. iPvs "Hvs2" "Hvs1"; first by set_solver.
rewrite -pvs_intro. done.
- iApply "Hwp". done. - iApply "Hwp". done.
Qed. Qed.
...@@ -126,10 +123,10 @@ Lemma ht_frame_step_r E E1 E2 P R1 R2 R3 e Φ : ...@@ -126,10 +123,10 @@ Lemma ht_frame_step_r E E1 E2 P R1 R2 R3 e Φ :
((R1 ={E1,E2}=> R2) (R2 ={E2,E1}=> R3) {{ P }} e @ E {{ Φ }}) ((R1 ={E1,E2}=> R2) (R2 ={E2,E1}=> R3) {{ P }} e @ E {{ Φ }})
{{ R1 P }} e @ (E E1) {{ λ v, Φ v R3 }}. {{ R1 P }} e @ (E E1) {{ λ v, Φ v R3 }}.
Proof. Proof.
iIntros {???} "[#Hvs1 [#Hvs2 #Hwp]]". iIntros {???} "[Hvs1 [Hvs2 Hwp]]".
setoid_rewrite (comm _ _ R3). setoid_rewrite (comm _ _ R3).
iApply ht_frame_step_l; try eassumption. iSplit; last iSplit; iApply ht_frame_step_l; try eassumption.
iIntros "!"; done. iSplit; last iSplit; done.
Qed. Qed.
Lemma ht_frame_step_l' E P R e Φ : Lemma ht_frame_step_l' E P R e Φ :
......
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