aboutsummaryrefslogtreecommitdiff
path: root/src/Specific/montgomery32_2e291m19_10limbs/femul.v
diff options
context:
space:
mode:
authorGravatar Andres Erbsen <andreser@mit.edu>2019-01-08 04:21:38 -0500
committerGravatar Andres Erbsen <andreser@mit.edu>2019-01-09 22:49:02 -0500
commit3ca227f1137e6a3b65bc33f5689e1c230d591595 (patch)
treee1e5a2dd2a2f34f239d3276227ddbdc69eeeb667 /src/Specific/montgomery32_2e291m19_10limbs/femul.v
parent3ec21c64b3682465ca8e159a187689b207c71de4 (diff)
remove old pipeline
Diffstat (limited to 'src/Specific/montgomery32_2e291m19_10limbs/femul.v')
-rw-r--r--src/Specific/montgomery32_2e291m19_10limbs/femul.v14
1 files changed, 0 insertions, 14 deletions
diff --git a/src/Specific/montgomery32_2e291m19_10limbs/femul.v b/src/Specific/montgomery32_2e291m19_10limbs/femul.v
deleted file mode 100644
index 9f88a1ac7..000000000
--- a/src/Specific/montgomery32_2e291m19_10limbs/femul.v
+++ /dev/null
@@ -1,14 +0,0 @@
-Require Import Crypto.Arithmetic.PrimeFieldTheorems.
-Require Import Crypto.Specific.montgomery32_2e291m19_10limbs.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.