aboutsummaryrefslogtreecommitdiff
path: root/src/Specific/montgomery64_2e152m17/fenz.v
diff options
context:
space:
mode:
authorGravatar Jason Gross <jgross@mit.edu>2017-10-14 16:01:37 -0400
committerGravatar Jason Gross <jasongross9@gmail.com>2017-10-18 23:01:29 -0400
commit0b03656ba15c354165ee14eda054de4489faeb9c (patch)
tree9c28e78ef48389a350fd8603d49f9eedc8f0c31f /src/Specific/montgomery64_2e152m17/fenz.v
parentd36702195ac82c2636b2f5842ae5fe210b7c415f (diff)
Run remake_curves.py
Diffstat (limited to 'src/Specific/montgomery64_2e152m17/fenz.v')
-rw-r--r--src/Specific/montgomery64_2e152m17/fenz.v16
1 files changed, 16 insertions, 0 deletions
diff --git a/src/Specific/montgomery64_2e152m17/fenz.v b/src/Specific/montgomery64_2e152m17/fenz.v
new file mode 100644
index 000000000..5fa15d88a
--- /dev/null
+++ b/src/Specific/montgomery64_2e152m17/fenz.v
@@ -0,0 +1,16 @@
+Require Import Coq.ZArith.ZArith.
+Require Import Crypto.Arithmetic.PrimeFieldTheorems.
+Require Import Crypto.Specific.montgomery64_2e152m17.Synthesis.
+Local Open Scope Z_scope.
+
+(* TODO : change this to field once field isomorphism happens *)
+Definition nonzero :
+ { nonzero : feBW_small -> BoundedWord.BoundedWord 1 adjusted_bitwidth bound1
+ | forall a, (BoundedWord.BoundedWordToZ _ _ _ (nonzero a) =? 0) = (if Decidable.dec (phiM_small a = F.of_Z m 0) then true else false) }.
+Proof.
+ Set Ltac Profiling.
+ Time synthesize_nonzero ().
+ Show Ltac Profile.
+Time Defined.
+
+Print Assumptions nonzero.