Skip to content

Commit c2628b5

Browse files
committed
Tweak rlimit
This proof failed on the Mac build only, which is bizarre. We should isolate it and report the failure to Z3 (if we are indeed sending it the same query, which we should).
1 parent 3bb7a3c commit c2628b5

File tree

1 file changed

+2
-0
lines changed

1 file changed

+2
-0
lines changed

ulib/FStar.Math.Fermat.fst

Lines changed: 2 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -392,6 +392,7 @@ let binomial_prime p k =
392392
factorial_mod_prime p (p - k)
393393
end
394394

395+
#push-options "--z3rlimit 40"
395396
val freshman_aux (p:int{is_prime p}) (a b:int) (i:pos{i < p}): Lemma
396397
((binomial p i * pow a (p - i) * pow b i) % p == 0)
397398
let freshman_aux p a b i =
@@ -404,6 +405,7 @@ let freshman_aux p a b i =
404405
== { binomial_prime p i }
405406
0;
406407
}
408+
#pop-options
407409

408410
val freshman (p:int{is_prime p}) (a b:int) : Lemma
409411
(pow (a + b) p % p = (pow a p + pow b p) % p)

0 commit comments

Comments
 (0)