File tree 3 files changed +8
-5
lines changed
3 files changed +8
-5
lines changed Original file line number Diff line number Diff line change @@ -18,7 +18,8 @@ Require Import Crypto.Util.ZUtil.Tactics.ZeroBounds.
18
18
19
19
Section Representation.
20
20
Context {p : Types.parameters} {field_parameters : FieldParameters}
21
- {p_ok : Types.ok}.
21
+ {p_ok : Types.ok}
22
+ (width_ge_32 : 32 <= Semantics.width).
22
23
Context (n : nat) (weight : nat -> Z)
23
24
(loose_bounds tight_bounds : list (option zrange))
24
25
(relax_bounds :
@@ -73,7 +74,7 @@ Section Representation.
73
74
{ match goal with
74
75
| H : Array.array _ _ _ _ _ |- _ =>
75
76
eapply Bignum_of_bytes with (n0:=n) in H;
76
- [ destruct H | nia ]
77
+ [ destruct H | nia.. ]
77
78
end.
78
79
eexists; eauto. }
79
80
{
Original file line number Diff line number Diff line change @@ -30,7 +30,8 @@ Section Bignum.
30
30
sep (emp (length x = n_bytes)) (array ptsto (word.of_Z 1) px x).
31
31
32
32
Section Proofs.
33
- Context {ok : Types.ok}.
33
+ Context {ok : Types.ok}
34
+ (width_ge_32 : 32 <= Semantics.width).
34
35
Existing Instance semantics_ok.
35
36
36
37
(* TODO: factor this proof into a more general form that says if subarrays
@@ -50,7 +51,7 @@ Section Bignum.
50
51
cbn [array length] in *. sepsimpl; eauto. }
51
52
{ rewrite <-(firstn_skipn (Z.to_nat word_size_in_bytes) bs).
52
53
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 .
54
55
2:{
55
56
rewrite word_size_in_bytes_eq in *.
56
57
etransitivity;
Original file line number Diff line number Diff line change @@ -297,7 +297,8 @@ Section LoadStoreList.
297
297
{ cbv [Memory.load].
298
298
erewrite load_Z_of_sep; [ reflexivity | ].
299
299
ecancel_assumption. }
300
- { rewrite Z.land_ones by auto with zarith.
300
+ { unfold truncate_Z.
301
+ rewrite Z.land_ones by auto with zarith.
301
302
rewrite Z.mod_small; [ reflexivity | ].
302
303
rewrite <-hd_skipn_nth_default.
303
304
match goal with H : base_access_sizes_good _ |- _ =>
You can’t perform that action at this time.
0 commit comments