Skip to content

Commit

Permalink
document applyUpdates
Browse files Browse the repository at this point in the history
  • Loading branch information
sanjit-bhat committed Jul 30, 2024
1 parent c856fdf commit 20b4fb1
Showing 1 changed file with 6 additions and 1 deletion.
7 changes: 6 additions & 1 deletion src/program_proof/pav/server.v
Original file line number Diff line number Diff line change
Expand Up @@ -333,8 +333,13 @@ Proof.
wp_apply (wp_Tree_DeepCopy with "Hown_currTr");
iEval (rewrite /named); iIntros (ptr_nextTr) "[Hown_currTr Hown_nextTr]".
set (loopInv := λ (_ sl_mdone : gmap string Slice.t),
(∃ (mdone : gmap (list w8) (list w8)),
(∃ mdone,
let sl_mdone' := (kmap string_to_bytes sl_mdone) : gmap (list w8) Slice.t in
(* these first two properties 'characterize' the following:
[Definition map_filter_keyset m S :
filter (λ '(k,_), k ∈ S) m.]
using the characterization instead of the implementation makes it easier
to work with. no rewriting under filter preds. *)
"%Hdom" ∷ ⌜ dom mdone = dom sl_mdone' ⌝ ∗
"%Hsubset" ∷ ⌜ mdone ⊆ updates ⌝ ∗
"Hown_nextTr" ∷ own_Tree ptr_nextTr (mdone ∪ currTr))%I).
Expand Down

0 comments on commit 20b4fb1

Please sign in to comment.