aboutsummaryrefslogtreecommitdiff
path: root/src/Specific/montgomery64_2e416m2e208m1_7limbs
diff options
context:
space:
mode:
Diffstat (limited to 'src/Specific/montgomery64_2e416m2e208m1_7limbs')
-rw-r--r--src/Specific/montgomery64_2e416m2e208m1_7limbs/CurveParameters.v39
-rw-r--r--src/Specific/montgomery64_2e416m2e208m1_7limbs/Synthesis.v9
-rwxr-xr-xsrc/Specific/montgomery64_2e416m2e208m1_7limbs/compiler.sh4
-rwxr-xr-xsrc/Specific/montgomery64_2e416m2e208m1_7limbs/compilerxx.sh4
-rw-r--r--src/Specific/montgomery64_2e416m2e208m1_7limbs/feadd.c46
-rw-r--r--src/Specific/montgomery64_2e416m2e208m1_7limbs/feadd.v14
-rw-r--r--src/Specific/montgomery64_2e416m2e208m1_7limbs/feaddDisplay.log29
-rw-r--r--src/Specific/montgomery64_2e416m2e208m1_7limbs/feaddDisplay.v4
-rw-r--r--src/Specific/montgomery64_2e416m2e208m1_7limbs/femul.v14
-rw-r--r--src/Specific/montgomery64_2e416m2e208m1_7limbs/femulDisplay.v4
-rw-r--r--src/Specific/montgomery64_2e416m2e208m1_7limbs/fenz.c17
-rw-r--r--src/Specific/montgomery64_2e416m2e208m1_7limbs/fenz.v16
-rw-r--r--src/Specific/montgomery64_2e416m2e208m1_7limbs/fenzDisplay.log13
-rw-r--r--src/Specific/montgomery64_2e416m2e208m1_7limbs/fenzDisplay.v4
-rw-r--r--src/Specific/montgomery64_2e416m2e208m1_7limbs/feopp.v14
-rw-r--r--src/Specific/montgomery64_2e416m2e208m1_7limbs/feoppDisplay.v4
-rw-r--r--src/Specific/montgomery64_2e416m2e208m1_7limbs/fesquare.c5
-rw-r--r--src/Specific/montgomery64_2e416m2e208m1_7limbs/fesub.v14
-rw-r--r--src/Specific/montgomery64_2e416m2e208m1_7limbs/fesubDisplay.v4
-rwxr-xr-xsrc/Specific/montgomery64_2e416m2e208m1_7limbs/py_interpreter.sh4
20 files changed, 0 insertions, 262 deletions
diff --git a/src/Specific/montgomery64_2e416m2e208m1_7limbs/CurveParameters.v b/src/Specific/montgomery64_2e416m2e208m1_7limbs/CurveParameters.v
deleted file mode 100644
index 15fb68dac..000000000
--- a/src/Specific/montgomery64_2e416m2e208m1_7limbs/CurveParameters.v
+++ /dev/null
@@ -1,39 +0,0 @@
-Require Import Crypto.Specific.Framework.RawCurveParameters.
-Require Import Crypto.Util.LetIn.
-
-(***
-Modulus : 2^416 - 2^208 - 1
-Base: 64
-***)
-
-Definition curve : CurveParameters :=
- {|
- sz := 7%nat;
- base := 64;
- bitwidth := 64;
- s := 2^416;
- c := [(1, 1); (2^208, 1)];
- carry_chains := None;
-
- a24 := None;
- coef_div_modulus := None;
-
- goldilocks := None;
- karatsuba := None;
- montgomery := true;
- freeze := Some false;
- ladderstep := false;
-
- mul_code := None;
-
- square_code := None;
-
- upper_bound_of_exponent_loose := None;
- upper_bound_of_exponent_tight := None;
- allowable_bit_widths := None;
- freeze_extra_allowable_bit_widths := None;
- modinv_fuel := None
- |}.
-
-Ltac extra_prove_mul_eq _ := idtac.
-Ltac extra_prove_square_eq _ := idtac.
diff --git a/src/Specific/montgomery64_2e416m2e208m1_7limbs/Synthesis.v b/src/Specific/montgomery64_2e416m2e208m1_7limbs/Synthesis.v
deleted file mode 100644
index 07c0c68cb..000000000
--- a/src/Specific/montgomery64_2e416m2e208m1_7limbs/Synthesis.v
+++ /dev/null
@@ -1,9 +0,0 @@
-Require Import Crypto.Specific.Framework.SynthesisFramework.
-Require Import Crypto.Specific.montgomery64_2e416m2e208m1_7limbs.CurveParameters.
-
-Module P <: PrePackage.
- Definition package : Tag.Context.
- Proof. make_Synthesis_package curve extra_prove_mul_eq extra_prove_square_eq. Defined.
-End P.
-
-Module Export S := PackageSynthesis P.
diff --git a/src/Specific/montgomery64_2e416m2e208m1_7limbs/compiler.sh b/src/Specific/montgomery64_2e416m2e208m1_7limbs/compiler.sh
deleted file mode 100755
index 85011ccfc..000000000
--- a/src/Specific/montgomery64_2e416m2e208m1_7limbs/compiler.sh
+++ /dev/null
@@ -1,4 +0,0 @@
-#!/bin/sh
-set -eu
-
-clang -fbracket-depth=999999 -march=native -mbmi2 -mtune=native -std=gnu11 -O3 -flto -fuse-ld=lld -fomit-frame-pointer -fwrapv -Wno-attributes -fno-strict-aliasing -Da24_hex='0x3039' -Da24_val='12345' -Da_minus_two_over_four_array='{0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x30,0x39}' -Dbitwidth='64' -Dlimb_weight_gaps_array='{64,64,64,64,64,64,64}' -Dmodulus_array='{0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xfe,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff}' -Dmodulus_bytes_val='52' -Dmodulus_limbs='7' -Dq_mpz='(1_mpz<<416) - (1_mpz<<208) - 1' "$@"
diff --git a/src/Specific/montgomery64_2e416m2e208m1_7limbs/compilerxx.sh b/src/Specific/montgomery64_2e416m2e208m1_7limbs/compilerxx.sh
deleted file mode 100755
index 80a407e51..000000000
--- a/src/Specific/montgomery64_2e416m2e208m1_7limbs/compilerxx.sh
+++ /dev/null
@@ -1,4 +0,0 @@
-#!/bin/sh
-set -eu
-
-clang++ -fbracket-depth=999999 -march=native -mbmi2 -mtune=native -std=gnu++11 -O3 -flto -fuse-ld=lld -fomit-frame-pointer -fwrapv -Wno-attributes -fno-strict-aliasing -Da24_hex='0x3039' -Da24_val='12345' -Da_minus_two_over_four_array='{0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x00,0x30,0x39}' -Dbitwidth='64' -Dlimb_weight_gaps_array='{64,64,64,64,64,64,64}' -Dmodulus_array='{0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xfe,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff,0xff}' -Dmodulus_bytes_val='52' -Dmodulus_limbs='7' -Dq_mpz='(1_mpz<<416) - (1_mpz<<208) - 1' "$@"
diff --git a/src/Specific/montgomery64_2e416m2e208m1_7limbs/feadd.c b/src/Specific/montgomery64_2e416m2e208m1_7limbs/feadd.c
deleted file mode 100644
index 753e03d78..000000000
--- a/src/Specific/montgomery64_2e416m2e208m1_7limbs/feadd.c
+++ /dev/null
@@ -1,46 +0,0 @@
-static void feadd(uint64_t out[7], const uint64_t in1[7], const uint64_t in2[7]) {
- { const uint64_t x14 = in1[6];
- { const uint64_t x15 = in1[5];
- { const uint64_t x13 = in1[4];
- { const uint64_t x11 = in1[3];
- { const uint64_t x9 = in1[2];
- { const uint64_t x7 = in1[1];
- { const uint64_t x5 = in1[0];
- { const uint64_t x26 = in2[6];
- { const uint64_t x27 = in2[5];
- { const uint64_t x25 = in2[4];
- { const uint64_t x23 = in2[3];
- { const uint64_t x21 = in2[2];
- { const uint64_t x19 = in2[1];
- { const uint64_t x17 = in2[0];
- { uint64_t x29; uint8_t x30 = _addcarryx_u64(0x0, x5, x17, &x29);
- { uint64_t x32; uint8_t x33 = _addcarryx_u64(x30, x7, x19, &x32);
- { uint64_t x35; uint8_t x36 = _addcarryx_u64(x33, x9, x21, &x35);
- { uint64_t x38; uint8_t x39 = _addcarryx_u64(x36, x11, x23, &x38);
- { uint64_t x41; uint8_t x42 = _addcarryx_u64(x39, x13, x25, &x41);
- { uint64_t x44; uint8_t x45 = _addcarryx_u64(x42, x15, x27, &x44);
- { uint64_t x47; uint8_t x48 = _addcarryx_u64(x45, x14, x26, &x47);
- { uint64_t x50; uint8_t x51 = _subborrow_u64(0x0, x29, 0xffffffffffffffffL, &x50);
- { uint64_t x53; uint8_t x54 = _subborrow_u64(x51, x32, 0xffffffffffffffffL, &x53);
- { uint64_t x56; uint8_t x57 = _subborrow_u64(x54, x35, 0xffffffffffffffffL, &x56);
- { uint64_t x59; uint8_t x60 = _subborrow_u64(x57, x38, 0xfffffffffffeffffL, &x59);
- { uint64_t x62; uint8_t x63 = _subborrow_u64(x60, x41, 0xffffffffffffffffL, &x62);
- { uint64_t x65; uint8_t x66 = _subborrow_u64(x63, x44, 0xffffffffffffffffL, &x65);
- { uint64_t x68; uint8_t x69 = _subborrow_u64(x66, x47, 0xffffffff, &x68);
- { uint64_t _; uint8_t x72 = _subborrow_u64(x69, x48, 0x0, &_);
- { uint64_t x73 = cmovznz64(x72, x68, x47);
- { uint64_t x74 = cmovznz64(x72, x65, x44);
- { uint64_t x75 = cmovznz64(x72, x62, x41);
- { uint64_t x76 = cmovznz64(x72, x59, x38);
- { uint64_t x77 = cmovznz64(x72, x56, x35);
- { uint64_t x78 = cmovznz64(x72, x53, x32);
- { uint64_t x79 = cmovznz64(x72, x50, x29);
- out[0] = x79;
- out[1] = x78;
- out[2] = x77;
- out[3] = x76;
- out[4] = x75;
- out[5] = x74;
- out[6] = x73;
- }}}}}}}}}}}}}}}}}}}}}}}}}}}}}}}}}}}}
-}
diff --git a/src/Specific/montgomery64_2e416m2e208m1_7limbs/feadd.v b/src/Specific/montgomery64_2e416m2e208m1_7limbs/feadd.v
deleted file mode 100644
index 039a4b8df..000000000
--- a/src/Specific/montgomery64_2e416m2e208m1_7limbs/feadd.v
+++ /dev/null
@@ -1,14 +0,0 @@
-Require Import Crypto.Arithmetic.PrimeFieldTheorems.
-Require Import Crypto.Specific.montgomery64_2e416m2e208m1_7limbs.Synthesis.
-
-(* TODO : change this to field once field isomorphism happens *)
-Definition add :
- { add : feBW_small -> feBW_small -> feBW_small
- | forall a b, phiM_small (add a b) = F.add (phiM_small a) (phiM_small b) }.
-Proof.
- Set Ltac Profiling.
- Time synthesize_add ().
- Show Ltac Profile.
-Time Defined.
-
-Print Assumptions add.
diff --git a/src/Specific/montgomery64_2e416m2e208m1_7limbs/feaddDisplay.log b/src/Specific/montgomery64_2e416m2e208m1_7limbs/feaddDisplay.log
deleted file mode 100644
index bdac118e2..000000000
--- a/src/Specific/montgomery64_2e416m2e208m1_7limbs/feaddDisplay.log
+++ /dev/null
@@ -1,29 +0,0 @@
-λ x x0 : word64 * word64 * word64 * word64 * word64 * word64 * word64,
-Interp-η
-(λ var : Syntax.base_type → Type,
- λ '(x14, x15, x13, x11, x9, x7, x5, (x26, x27, x25, x23, x21, x19, x17))%core,
- uint64_t x29, uint8_t x30 = addcarryx_u64(0x0, x5, x17);
- uint64_t x32, uint8_t x33 = addcarryx_u64(x30, x7, x19);
- uint64_t x35, uint8_t x36 = addcarryx_u64(x33, x9, x21);
- uint64_t x38, uint8_t x39 = addcarryx_u64(x36, x11, x23);
- uint64_t x41, uint8_t x42 = addcarryx_u64(x39, x13, x25);
- uint64_t x44, uint8_t x45 = addcarryx_u64(x42, x15, x27);
- uint64_t x47, uint8_t x48 = addcarryx_u64(x45, x14, x26);
- uint64_t x50, uint8_t x51 = subborrow_u64(0x0, x29, 0xffffffffffffffffL);
- uint64_t x53, uint8_t x54 = subborrow_u64(x51, x32, 0xffffffffffffffffL);
- uint64_t x56, uint8_t x57 = subborrow_u64(x54, x35, 0xffffffffffffffffL);
- uint64_t x59, uint8_t x60 = subborrow_u64(x57, x38, 0xfffffffffffeffffL);
- uint64_t x62, uint8_t x63 = subborrow_u64(x60, x41, 0xffffffffffffffffL);
- uint64_t x65, uint8_t x66 = subborrow_u64(x63, x44, 0xffffffffffffffffL);
- uint64_t x68, uint8_t x69 = subborrow_u64(x66, x47, 0xffffffff);
- uint64_t _, uint8_t x72 = subborrow_u64(x69, x48, 0x0);
- uint64_t x73 = cmovznz64(x72, x68, x47);
- uint64_t x74 = cmovznz64(x72, x65, x44);
- uint64_t x75 = cmovznz64(x72, x62, x41);
- uint64_t x76 = cmovznz64(x72, x59, x38);
- uint64_t x77 = cmovznz64(x72, x56, x35);
- uint64_t x78 = cmovznz64(x72, x53, x32);
- uint64_t x79 = cmovznz64(x72, x50, x29);
- return (x73, x74, x75, x76, x77, x78, x79))
-(x, x0)%core
- : word64 * word64 * word64 * word64 * word64 * word64 * word64 → word64 * word64 * word64 * word64 * word64 * word64 * word64 → ReturnType (uint64_t * uint64_t * uint64_t * uint64_t * uint64_t * uint64_t * uint64_t)
diff --git a/src/Specific/montgomery64_2e416m2e208m1_7limbs/feaddDisplay.v b/src/Specific/montgomery64_2e416m2e208m1_7limbs/feaddDisplay.v
deleted file mode 100644
index d02523bdd..000000000
--- a/src/Specific/montgomery64_2e416m2e208m1_7limbs/feaddDisplay.v
+++ /dev/null
@@ -1,4 +0,0 @@
-Require Import Crypto.Specific.montgomery64_2e416m2e208m1_7limbs.feadd.
-Require Import Crypto.Specific.Framework.IntegrationTestDisplayCommon.
-
-Check display add.
diff --git a/src/Specific/montgomery64_2e416m2e208m1_7limbs/femul.v b/src/Specific/montgomery64_2e416m2e208m1_7limbs/femul.v
deleted file mode 100644
index 6f9353567..000000000
--- a/src/Specific/montgomery64_2e416m2e208m1_7limbs/femul.v
+++ /dev/null
@@ -1,14 +0,0 @@
-Require Import Crypto.Arithmetic.PrimeFieldTheorems.
-Require Import Crypto.Specific.montgomery64_2e416m2e208m1_7limbs.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.
diff --git a/src/Specific/montgomery64_2e416m2e208m1_7limbs/femulDisplay.v b/src/Specific/montgomery64_2e416m2e208m1_7limbs/femulDisplay.v
deleted file mode 100644
index f72f3649b..000000000
--- a/src/Specific/montgomery64_2e416m2e208m1_7limbs/femulDisplay.v
+++ /dev/null
@@ -1,4 +0,0 @@
-Require Import Crypto.Specific.montgomery64_2e416m2e208m1_7limbs.femul.
-Require Import Crypto.Specific.Framework.IntegrationTestDisplayCommon.
-
-Check display mul.
diff --git a/src/Specific/montgomery64_2e416m2e208m1_7limbs/fenz.c b/src/Specific/montgomery64_2e416m2e208m1_7limbs/fenz.c
deleted file mode 100644
index d09ab7ff5..000000000
--- a/src/Specific/montgomery64_2e416m2e208m1_7limbs/fenz.c
+++ /dev/null
@@ -1,17 +0,0 @@
-static void fenz(ReturnType uint64_t out[1], const uint64_t in1[7]) {
- { const uint64_t x11 = in1[6];
- { const uint64_t x12 = in1[5];
- { const uint64_t x10 = in1[4];
- { const uint64_t x8 = in1[3];
- { const uint64_t x6 = in1[2];
- { const uint64_t x4 = in1[1];
- { const uint64_t x2 = in1[0];
- { uint64_t x13 = (x12 | x11);
- { uint64_t x14 = (x10 | x13);
- { uint64_t x15 = (x8 | x14);
- { uint64_t x16 = (x6 | x15);
- { uint64_t x17 = (x4 | x16);
- { uint64_t x18 = (x2 | x17);
- out[0] = x18;
- }}}}}}}}}}}}}
-}
diff --git a/src/Specific/montgomery64_2e416m2e208m1_7limbs/fenz.v b/src/Specific/montgomery64_2e416m2e208m1_7limbs/fenz.v
deleted file mode 100644
index 26142d172..000000000
--- a/src/Specific/montgomery64_2e416m2e208m1_7limbs/fenz.v
+++ /dev/null
@@ -1,16 +0,0 @@
-Require Import Coq.ZArith.ZArith.
-Require Import Crypto.Arithmetic.PrimeFieldTheorems.
-Require Import Crypto.Specific.montgomery64_2e416m2e208m1_7limbs.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.
diff --git a/src/Specific/montgomery64_2e416m2e208m1_7limbs/fenzDisplay.log b/src/Specific/montgomery64_2e416m2e208m1_7limbs/fenzDisplay.log
deleted file mode 100644
index 28baa6eea..000000000
--- a/src/Specific/montgomery64_2e416m2e208m1_7limbs/fenzDisplay.log
+++ /dev/null
@@ -1,13 +0,0 @@
-λ x : word64 * word64 * word64 * word64 * word64 * word64 * word64,
-Interp-η
-(λ var : Syntax.base_type → Type,
- λ '(x11, x12, x10, x8, x6, x4, x2)%core,
- uint64_t x13 = (x12 | x11);
- uint64_t x14 = (x10 | x13);
- uint64_t x15 = (x8 | x14);
- uint64_t x16 = (x6 | x15);
- uint64_t x17 = (x4 | x16);
- uint64_t x18 = (x2 | x17);
- return x18)
-x
- : word64 * word64 * word64 * word64 * word64 * word64 * word64 → ReturnType uint64_t
diff --git a/src/Specific/montgomery64_2e416m2e208m1_7limbs/fenzDisplay.v b/src/Specific/montgomery64_2e416m2e208m1_7limbs/fenzDisplay.v
deleted file mode 100644
index c1834cf24..000000000
--- a/src/Specific/montgomery64_2e416m2e208m1_7limbs/fenzDisplay.v
+++ /dev/null
@@ -1,4 +0,0 @@
-Require Import Crypto.Specific.montgomery64_2e416m2e208m1_7limbs.fenz.
-Require Import Crypto.Specific.Framework.IntegrationTestDisplayCommon.
-
-Check display nonzero.
diff --git a/src/Specific/montgomery64_2e416m2e208m1_7limbs/feopp.v b/src/Specific/montgomery64_2e416m2e208m1_7limbs/feopp.v
deleted file mode 100644
index c02f8857d..000000000
--- a/src/Specific/montgomery64_2e416m2e208m1_7limbs/feopp.v
+++ /dev/null
@@ -1,14 +0,0 @@
-Require Import Crypto.Arithmetic.PrimeFieldTheorems.
-Require Import Crypto.Specific.montgomery64_2e416m2e208m1_7limbs.Synthesis.
-
-(* TODO : change this to field once field isomorphism happens *)
-Definition opp :
- { opp : feBW_small -> feBW_small
- | forall a, phiM_small (opp a) = F.opp (phiM_small a) }.
-Proof.
- Set Ltac Profiling.
- Time synthesize_opp ().
- Show Ltac Profile.
-Time Defined.
-
-Print Assumptions opp.
diff --git a/src/Specific/montgomery64_2e416m2e208m1_7limbs/feoppDisplay.v b/src/Specific/montgomery64_2e416m2e208m1_7limbs/feoppDisplay.v
deleted file mode 100644
index 89cad0fde..000000000
--- a/src/Specific/montgomery64_2e416m2e208m1_7limbs/feoppDisplay.v
+++ /dev/null
@@ -1,4 +0,0 @@
-Require Import Crypto.Specific.montgomery64_2e416m2e208m1_7limbs.feopp.
-Require Import Crypto.Specific.Framework.IntegrationTestDisplayCommon.
-
-Check display opp.
diff --git a/src/Specific/montgomery64_2e416m2e208m1_7limbs/fesquare.c b/src/Specific/montgomery64_2e416m2e208m1_7limbs/fesquare.c
deleted file mode 100644
index 7bd8db166..000000000
--- a/src/Specific/montgomery64_2e416m2e208m1_7limbs/fesquare.c
+++ /dev/null
@@ -1,5 +0,0 @@
-/* WARNING: This file was copied from Specific/CurveParameters/montgomery64/fesquare.c.
- If you edit it here, changes will be erased the next time remake_curves.sh is run. */
-static void fesquare(uint64_t *out, const uint64_t *in) {
- femul(out, in, in);
-}
diff --git a/src/Specific/montgomery64_2e416m2e208m1_7limbs/fesub.v b/src/Specific/montgomery64_2e416m2e208m1_7limbs/fesub.v
deleted file mode 100644
index 381ee1bdb..000000000
--- a/src/Specific/montgomery64_2e416m2e208m1_7limbs/fesub.v
+++ /dev/null
@@ -1,14 +0,0 @@
-Require Import Crypto.Arithmetic.PrimeFieldTheorems.
-Require Import Crypto.Specific.montgomery64_2e416m2e208m1_7limbs.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.
diff --git a/src/Specific/montgomery64_2e416m2e208m1_7limbs/fesubDisplay.v b/src/Specific/montgomery64_2e416m2e208m1_7limbs/fesubDisplay.v
deleted file mode 100644
index 5ad930b75..000000000
--- a/src/Specific/montgomery64_2e416m2e208m1_7limbs/fesubDisplay.v
+++ /dev/null
@@ -1,4 +0,0 @@
-Require Import Crypto.Specific.montgomery64_2e416m2e208m1_7limbs.fesub.
-Require Import Crypto.Specific.Framework.IntegrationTestDisplayCommon.
-
-Check display sub.
diff --git a/src/Specific/montgomery64_2e416m2e208m1_7limbs/py_interpreter.sh b/src/Specific/montgomery64_2e416m2e208m1_7limbs/py_interpreter.sh
deleted file mode 100755
index 6495749c9..000000000
--- a/src/Specific/montgomery64_2e416m2e208m1_7limbs/py_interpreter.sh
+++ /dev/null
@@ -1,4 +0,0 @@
-#!/bin/sh
-set -eu
-
-/usr/bin/env python3 "$@" -Dq='2**416 - 2**208 - 1' -Dmodulus_bytes='64' -Da24='121665'