From 3ca227f1137e6a3b65bc33f5689e1c230d591595 Mon Sep 17 00:00:00 2001 From: Andres Erbsen Date: Tue, 8 Jan 2019 04:21:38 -0500 Subject: remove old pipeline --- .../montgomery32_2e510m290x2e496m1_16limbs/fenz.v | 16 ---------------- 1 file changed, 16 deletions(-) delete mode 100644 src/Specific/montgomery32_2e510m290x2e496m1_16limbs/fenz.v (limited to 'src/Specific/montgomery32_2e510m290x2e496m1_16limbs/fenz.v') diff --git a/src/Specific/montgomery32_2e510m290x2e496m1_16limbs/fenz.v b/src/Specific/montgomery32_2e510m290x2e496m1_16limbs/fenz.v deleted file mode 100644 index f28b6235b..000000000 --- a/src/Specific/montgomery32_2e510m290x2e496m1_16limbs/fenz.v +++ /dev/null @@ -1,16 +0,0 @@ -Require Import Coq.ZArith.ZArith. -Require Import Crypto.Arithmetic.PrimeFieldTheorems. -Require Import Crypto.Specific.montgomery32_2e510m290x2e496m1_16limbs.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. -- cgit v1.2.3