Skip to content

Commit

Permalink
Bump dependencies
Browse files Browse the repository at this point in the history
  • Loading branch information
tchajed committed Mar 7, 2024
1 parent 10b8791 commit 772faf8
Show file tree
Hide file tree
Showing 12 changed files with 16 additions and 12 deletions.
2 changes: 1 addition & 1 deletion external/iris
Submodule iris updated from 06f499 to 9c192c
2 changes: 1 addition & 1 deletion external/stdpp
Submodule stdpp updated from cafd71 to 69984f
1 change: 1 addition & 0 deletions src/goose_lang/lib/slice/pred_slice.v
Original file line number Diff line number Diff line change
Expand Up @@ -62,6 +62,7 @@ Proof.
apply fmap_Some_2; eauto. }
iIntros "[Hs %Hty]".
iApply "HΦ"; iFrame.
iIntros "HΨ". iFrame. iApply ("Hxs" with "HΨ").
Qed.

Theorem wp_SliceAppend {stk E} s l v x :
Expand Down
2 changes: 1 addition & 1 deletion src/program_proof/buf/bufmap_proof.v
Original file line number Diff line number Diff line change
Expand Up @@ -166,7 +166,7 @@ Proof using.
iFrame.

iIntros "!>" (b') "Hbuf".
iExists _.
iExists _, _, _; iFrame.
iSplitR; first eauto.
replace (am) with (<[a:=v]> am) at 1 by ( apply insert_id; eauto ).
by iApply "Ham".
Expand Down
6 changes: 3 additions & 3 deletions src/program_proof/examples/async_mem_alloc_inode_proof.v
Original file line number Diff line number Diff line change
Expand Up @@ -71,7 +71,7 @@ Theorem is_inode_durable_read addr σ addrs :
Proof.
iNamed 1.
iExists _; iFrame "∗ %".
iIntros "!> $ $".
iIntros "!> Haddr Hdata". iExists _; iFrame "∗%".
Qed.

Definition inode_linv (l:loc) (addr:u64) σ : iProp Σ :=
Expand Down Expand Up @@ -312,7 +312,7 @@ Proof.
wp_loadField.
iApply "HΦ".
iFrame "∗ %".
iIntros "$".
iIntros "$". iFrame.
Qed.

Theorem wpc_Inode__UsedBlocks {l σ addr} :
Expand Down Expand Up @@ -914,7 +914,7 @@ Proof.
wpc_apply (wpc_Barrier1 with "[$Hhdr]").
iSplit.
{
iLeft in "Hfupd". iFrame. iIntros "$". by subst.
iLeft in "Hfupd". iFrame. iIntros "$". iFrame "∗%". by subst.
}
iNext. iIntros "[%Hfalso ?]". exfalso. congruence.
}
Expand Down
4 changes: 2 additions & 2 deletions src/program_proof/examples/inode_proof.v
Original file line number Diff line number Diff line change
Expand Up @@ -71,7 +71,7 @@ Theorem is_inode_durable_read addr σ addrs :
Proof.
iNamed 1.
iExists _; iFrame "∗ %".
iIntros "!> $ $".
iIntros "!> Haddr Hdata". iExists _; iFrame "∗%".
Qed.

Definition inode_linv (l:loc) (addr:u64) σ : iProp Σ :=
Expand Down Expand Up @@ -294,7 +294,7 @@ Proof.
wp_loadField.
iApply "HΦ".
iFrame "∗ %".
iIntros "$".
iIntros "$". iFrame.
Qed.

Theorem wpc_Inode__UsedBlocks {l σ addr} :
Expand Down
2 changes: 1 addition & 1 deletion src/program_proof/examples/replicated_block_proof.v
Original file line number Diff line number Diff line change
Expand Up @@ -226,7 +226,7 @@ Section goose.
wpc_apply (wpc_Read with "Haddr'").
iSplit; [ | iNext ].
{ iLeft in "HQ".
iFrame. iIntros.
iFrame. iIntros. iFrame "HP".
iApply rblock_linv_to_cinv; iFrame. iApply "Hlkinv". eauto. }
iIntros (s) "(Haddr'&Hb)".
iDestruct (own_slice_to_small with "Hb") as "Hb".
Expand Down
3 changes: 2 additions & 1 deletion src/program_proof/obj/commit_proof.v
Original file line number Diff line number Diff line change
Expand Up @@ -1275,14 +1275,15 @@ Proof.
iApply "HΦ". iModIntro. iFrame.
iSplitL.
2: { iIntros "%H". congruence. }
iIntros (H). iExists _; iFrame.
done.

* wp_pures.
wp_load.
iApply "HΦ". iModIntro. iFrame.
iSplitL.
2: { iIntros "%H". congruence. }
iIntros (??). intuition congruence.
iIntros (?). iExists _; iFrame. iIntros (?). intuition congruence.

+ wp_apply util_proof.wp_DPrintf.
wp_store.
Expand Down
2 changes: 1 addition & 1 deletion src/program_proof/obj/invariant.v
Original file line number Diff line number Diff line change
Expand Up @@ -192,7 +192,7 @@ Proof.
rewrite /pointsto_txn.
iIntros "H". iNamed "H".
iFrame.
iIntros (v') "$H".
iIntros (v') "$". iExists _; iFrame.
Qed.

Theorem pointsto_txn_cur_map {A} γ (m : gmap addr A) (f : A -> {K & bufDataT K}) (xform : A -> A):
Expand Down
1 change: 1 addition & 0 deletions src/program_proof/vrsm/replica/init_proof.v
Original file line number Diff line number Diff line change
Expand Up @@ -135,6 +135,7 @@ Proof.
iNamed "Hinit".
iFrame "∗ His_conf #".
iIntros.
iExists _. iFrame "His_conf_prop".
iPureIntro.
by apply elem_of_list_fmap_1.
Qed.
Expand Down
1 change: 1 addition & 0 deletions src/program_proof/wal/sliding_proof.v
Original file line number Diff line number Diff line change
Expand Up @@ -375,6 +375,7 @@ Proof.
iIntros "Hb"; iSpecialize ("Hlog" with "Hb").
iSpecialize ("Hlog_mutable" with "Hlog").
iSplit; auto.
iExists _, _; iFrame "∗#".
Qed.

Theorem addrPosMap_lookup_inv σ pos :
Expand Down

0 comments on commit 772faf8

Please sign in to comment.