Skip to content

Commit

Permalink
reflect fixes in 64-bit
Browse files Browse the repository at this point in the history
  • Loading branch information
mansky1 committed Apr 5, 2024
1 parent 3b4bb6c commit d132e3b
Show file tree
Hide file tree
Showing 2 changed files with 5 additions and 5 deletions.
2 changes: 1 addition & 1 deletion progs64/io_mem_dry.v
Original file line number Diff line number Diff line change
Expand Up @@ -93,7 +93,7 @@ Proof.
iPureIntro; repeat (split; first done).
subst; simpl.
rewrite Mem.loadbytes_empty //. }
rewrite split2_data_at_Tarray_app //.
erewrite split2_data_at_Tarray_app; [| done |].
iDestruct "Hbuf" as "(Hmsg & _)".
iDestruct (data_at_bytes with "[$Hz $Hmsg]") as %Hmsg; [done.. | |].
{ rewrite Forall_map Forall_forall //. }
Expand Down
8 changes: 4 additions & 4 deletions progs64/verif_strlib.v
Original file line number Diff line number Diff line change
Expand Up @@ -140,10 +140,10 @@ Qed.
Lemma split_data_at_app_tschar:
forall sh n (al bl: list val) p,
n = Zlength (al++bl) ->
data_at sh (tarray tschar n) (al++bl) p ⊣⊢
data_at sh (tarray tschar (Zlength al)) al p
* data_at sh (tarray tschar (n - Zlength al)) bl
(field_address0 (tarray tschar n) [ArraySubsc (Zlength al)] p).
data_at sh (tarray tschar n) (al++bl) p =
(data_at sh (tarray tschar (Zlength al)) al p
* data_at sh (tarray tschar (n - Zlength al)) bl
(field_address0 (tarray tschar n) [ArraySubsc (Zlength al)] p)).
Proof.
intros.
apply (split2_data_at_Tarray_app _ n sh tschar al bl); auto.
Expand Down

0 comments on commit d132e3b

Please sign in to comment.