aboutsummaryrefslogtreecommitdiff
path: root/src/Specific/montgomery32_2e189m25_6limbs/fenz.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/Specific/montgomery32_2e189m25_6limbs/fenz.v')
-rw-r--r--src/Specific/montgomery32_2e189m25_6limbs/fenz.v16
1 files changed, 0 insertions, 16 deletions
diff --git a/src/Specific/montgomery32_2e189m25_6limbs/fenz.v b/src/Specific/montgomery32_2e189m25_6limbs/fenz.v
deleted file mode 100644
index ab9fda2ab..000000000
--- a/src/Specific/montgomery32_2e189m25_6limbs/fenz.v
+++ /dev/null
@@ -1,16 +0,0 @@
-Require Import Coq.ZArith.ZArith.
-Require Import Crypto.Arithmetic.PrimeFieldTheorems.
-Require Import Crypto.Specific.montgomery32_2e189m25_6limbs.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.