Skip to content

Commit 21d80cf

Browse files
committed
Fix some code according to bump of bedrock2
1 parent c17edf4 commit 21d80cf

File tree

3 files changed

+8
-5
lines changed

3 files changed

+8
-5
lines changed

src/Bedrock/Field/Interface/Representation.v

+3-2
Original file line numberDiff line numberDiff line change
@@ -18,7 +18,8 @@ Require Import Crypto.Util.ZUtil.Tactics.ZeroBounds.
1818

1919
Section Representation.
2020
Context {p : Types.parameters} {field_parameters : FieldParameters}
21-
{p_ok : Types.ok}.
21+
{p_ok : Types.ok}
22+
(width_ge_32 : 32 <= Semantics.width).
2223
Context (n : nat) (weight : nat -> Z)
2324
(loose_bounds tight_bounds : list (option zrange))
2425
(relax_bounds :
@@ -73,7 +74,7 @@ Section Representation.
7374
{ match goal with
7475
| H : Array.array _ _ _ _ _ |- _ =>
7576
eapply Bignum_of_bytes with (n0:=n) in H;
76-
[ destruct H | nia ]
77+
[ destruct H | nia.. ]
7778
end.
7879
eexists; eauto. }
7980
{

src/Bedrock/Field/Synthesis/Generic/Bignum.v

+3-2
Original file line numberDiff line numberDiff line change
@@ -30,7 +30,8 @@ Section Bignum.
3030
sep (emp (length x = n_bytes)) (array ptsto (word.of_Z 1) px x).
3131

3232
Section Proofs.
33-
Context {ok : Types.ok}.
33+
Context {ok : Types.ok}
34+
(width_ge_32 : 32 <= Semantics.width).
3435
Existing Instance semantics_ok.
3536

3637
(* TODO: factor this proof into a more general form that says if subarrays
@@ -50,7 +51,7 @@ Section Bignum.
5051
cbn [array length] in *. sepsimpl; eauto. }
5152
{ rewrite <-(firstn_skipn (Z.to_nat word_size_in_bytes) bs).
5253
rewrite array_append.
53-
rewrite Scalars.scalar_of_bytes with (l:=List.firstn _ _).
54+
rewrite Scalars.scalar_of_bytes with (l:=List.firstn _ _); try assumption.
5455
2:{
5556
rewrite word_size_in_bytes_eq in *.
5657
etransitivity;

src/Bedrock/Field/Translation/Proofs/LoadStoreList.v

+2-1
Original file line numberDiff line numberDiff line change
@@ -297,7 +297,8 @@ Section LoadStoreList.
297297
{ cbv [Memory.load].
298298
erewrite load_Z_of_sep; [ reflexivity | ].
299299
ecancel_assumption. }
300-
{ rewrite Z.land_ones by auto with zarith.
300+
{ unfold truncate_Z.
301+
rewrite Z.land_ones by auto with zarith.
301302
rewrite Z.mod_small; [ reflexivity | ].
302303
rewrite <-hd_skipn_nth_default.
303304
match goal with H : base_access_sizes_good _ |- _ =>

0 commit comments

Comments
 (0)