aboutsummaryrefslogtreecommitdiff
path: root/src/Specific/solinas32_2e468m17/fesub.v
diff options
context:
space:
mode:
authorGravatar Jason Gross <jgross@mit.edu>2017-11-02 04:37:37 -0400
committerGravatar Jason Gross <jgross@mit.edu>2017-11-02 04:37:37 -0400
commit631e3c7dca28f754f997f9d079d6900d76b8430e (patch)
treea587aae695cb8e27cbe63f10928c12ccf9c56799 /src/Specific/solinas32_2e468m17/fesub.v
parentc1a11d3b06cd984099e00a298b087f3a67855474 (diff)
python3 generate_parameters.py primes.txt; (cd src/Specific/CurveParameters/; ./remake_curves.sh -f)
Diffstat (limited to 'src/Specific/solinas32_2e468m17/fesub.v')
-rw-r--r--src/Specific/solinas32_2e468m17/fesub.v14
1 files changed, 14 insertions, 0 deletions
diff --git a/src/Specific/solinas32_2e468m17/fesub.v b/src/Specific/solinas32_2e468m17/fesub.v
new file mode 100644
index 000000000..e685ffab4
--- /dev/null
+++ b/src/Specific/solinas32_2e468m17/fesub.v
@@ -0,0 +1,14 @@
+Require Import Crypto.Arithmetic.PrimeFieldTheorems.
+Require Import Crypto.Specific.solinas32_2e468m17.Synthesis.
+
+(* TODO : change this to field once field isomorphism happens *)
+Definition sub :
+ { sub : feBW_tight -> feBW_tight -> feBW_loose
+ | forall a b, phiBW_loose (sub a b) = F.sub (phiBW_tight a) (phiBW_tight b) }.
+Proof.
+ Set Ltac Profiling.
+ Time synthesize_sub ().
+ Show Ltac Profile.
+Time Defined.
+
+Print Assumptions sub.