aboutsummaryrefslogtreecommitdiff
path: root/src/Specific/montgomery64_2e384m79x2e376m1/femul.v
diff options
context:
space:
mode:
authorGravatar Jason Gross <jgross@mit.edu>2017-10-16 01:16:24 -0400
committerGravatar Jason Gross <jasongross9@gmail.com>2017-10-18 23:01:29 -0400
commit3963ad55fada5c6df6c52e82ee483da9a085c9a9 (patch)
tree50f5831e0608a6a48873ebdd9226460866cb9a86 /src/Specific/montgomery64_2e384m79x2e376m1/femul.v
parent228b9c35ae331ac30b5829689d9a9320612edb67 (diff)
Remake some curves
Diffstat (limited to 'src/Specific/montgomery64_2e384m79x2e376m1/femul.v')
-rw-r--r--src/Specific/montgomery64_2e384m79x2e376m1/femul.v14
1 files changed, 14 insertions, 0 deletions
diff --git a/src/Specific/montgomery64_2e384m79x2e376m1/femul.v b/src/Specific/montgomery64_2e384m79x2e376m1/femul.v
new file mode 100644
index 000000000..8523fc2d6
--- /dev/null
+++ b/src/Specific/montgomery64_2e384m79x2e376m1/femul.v
@@ -0,0 +1,14 @@
+Require Import Crypto.Arithmetic.PrimeFieldTheorems.
+Require Import Crypto.Specific.montgomery64_2e384m79x2e376m1.Synthesis.
+
+(* TODO : change this to field once field isomorphism happens *)
+Definition mul :
+ { mul : feBW_small -> feBW_small -> feBW_small
+ | forall a b, phiM_small (mul a b) = F.mul (phiM_small a) (phiM_small b) }.
+Proof.
+ Set Ltac Profiling.
+ Time synthesize_mul ().
+ Show Ltac Profile.
+Time Defined.
+
+Print Assumptions mul.