Skip to content

Commit

Permalink
Finish improvements to tutorial/kvservice/proof.v
Browse files Browse the repository at this point in the history
  • Loading branch information
upamanyus committed Nov 22, 2024
1 parent 5979dff commit fbb36a6
Show file tree
Hide file tree
Showing 5 changed files with 242 additions and 473 deletions.
2 changes: 1 addition & 1 deletion src/ShouldBuild.v
Original file line number Diff line number Diff line change
Expand Up @@ -99,7 +99,7 @@ From Perennial.program_proof.tutorial Require
basics.proof
queue.proof
kvservice.proof
(* kvservice.full_proof *).
kvservice.full_proof.

From Perennial.program_proof.cachekv Require proof.

Expand Down
16 changes: 7 additions & 9 deletions src/program_proof/tutorial/kvservice/bank_proof.v
Original file line number Diff line number Diff line change
Expand Up @@ -70,15 +70,13 @@ Proof.
iIntros (Φ) "(Hlck & #Hln1_islock & #Hln2_islock) Hpost".
wp_rec.
wp_pures.
destruct bool_decide; wp_pures.
{
wp_apply (wp_LockClerk__Lock with "[$Hlck $Hln1_islock]").
iIntros "[Hlck HP1]".
wp_pures.
wp_apply (wp_LockClerk__Lock with "[$Hlck $Hln2_islock]").
iIntros "[Hlck HP2]".
wp_pures.
iApply "Hpost". by iFrame.
wp_apply (wp_LockClerk__Lock with "[$Hlck]").
iIntros "[Hlck HP1]".
wp_pures.
wp_apply (wp_LockClerk__Lock with "[$Hlck $Hln2_islock]").
iIntros "[Hlck HP2]".
wp_pures.
iApply "Hpost". by iFrame.
}
{
wp_apply (wp_LockClerk__Lock with "[$Hlck $Hln2_islock]").
Expand Down
Loading

0 comments on commit fbb36a6

Please sign in to comment.