We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent 91e4186 commit 833860fCopy full SHA for 833860f
ulib/FStar.UInt128.fst
@@ -953,6 +953,7 @@ val u32_product_bound : a:nat{a < pow2 32} -> b:nat{b < pow2 32} ->
953
let u32_product_bound a b =
954
uint_product_bound #32 a b
955
956
+#push-options "--z3rlimit 15 --retry 5" // sporadically fails
957
let mul32 x y =
958
let x0 = u64_mod_32 x in
959
let x1 = U64.shift_right x u32_32 in
@@ -979,6 +980,7 @@ let mul32 x y =
979
980
mul32_digits (U64.v x) (U32.v y);
981
assert (U64.v x * U32.v y == U64.v x1y' * pow2 32 + U64.v x0y);
982
r
983
+#pop-options
984
985
let l32 (x: UInt.uint_t 64) : UInt.uint_t 32 = x % pow2 32
986
let h32 (x: UInt.uint_t 64) : UInt.uint_t 32 = x / pow2 32
0 commit comments