Skip to content

Commit 833860f

Browse files
committed
Tweak flaky proof
1 parent 91e4186 commit 833860f

File tree

1 file changed

+2
-0
lines changed

1 file changed

+2
-0
lines changed

ulib/FStar.UInt128.fst

Lines changed: 2 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -953,6 +953,7 @@ val u32_product_bound : a:nat{a < pow2 32} -> b:nat{b < pow2 32} ->
953953
let u32_product_bound a b =
954954
uint_product_bound #32 a b
955955

956+
#push-options "--z3rlimit 15 --retry 5" // sporadically fails
956957
let mul32 x y =
957958
let x0 = u64_mod_32 x in
958959
let x1 = U64.shift_right x u32_32 in
@@ -979,6 +980,7 @@ let mul32 x y =
979980
mul32_digits (U64.v x) (U32.v y);
980981
assert (U64.v x * U32.v y == U64.v x1y' * pow2 32 + U64.v x0y);
981982
r
983+
#pop-options
982984

983985
let l32 (x: UInt.uint_t 64) : UInt.uint_t 32 = x % pow2 32
984986
let h32 (x: UInt.uint_t 64) : UInt.uint_t 32 = x / pow2 32

0 commit comments

Comments
 (0)