aboutsummaryrefslogtreecommitdiff
path: root/src/Specific/montgomery64_2e192m2e64m1_3limbs/fesub.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/Specific/montgomery64_2e192m2e64m1_3limbs/fesub.v')
-rw-r--r--src/Specific/montgomery64_2e192m2e64m1_3limbs/fesub.v14
1 files changed, 0 insertions, 14 deletions
diff --git a/src/Specific/montgomery64_2e192m2e64m1_3limbs/fesub.v b/src/Specific/montgomery64_2e192m2e64m1_3limbs/fesub.v
deleted file mode 100644
index 4e63c1baa..000000000
--- a/src/Specific/montgomery64_2e192m2e64m1_3limbs/fesub.v
+++ /dev/null
@@ -1,14 +0,0 @@
-Require Import Crypto.Arithmetic.PrimeFieldTheorems.
-Require Import Crypto.Specific.montgomery64_2e192m2e64m1_3limbs.Synthesis.
-
-(* TODO : change this to field once field isomorphism happens *)
-Definition sub :
- { sub : feBW_small -> feBW_small -> feBW_small
- | forall a b, phiM_small (sub a b) = F.sub (phiM_small a) (phiM_small b) }.
-Proof.
- Set Ltac Profiling.
- Time synthesize_sub ().
- Show Ltac Profile.
-Time Defined.
-
-Print Assumptions sub.