aboutsummaryrefslogtreecommitdiff
path: root/src/Specific/NISTP256/AMD128/feadd.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/Specific/NISTP256/AMD128/feadd.v')
-rw-r--r--src/Specific/NISTP256/AMD128/feadd.v14
1 files changed, 14 insertions, 0 deletions
diff --git a/src/Specific/NISTP256/AMD128/feadd.v b/src/Specific/NISTP256/AMD128/feadd.v
new file mode 100644
index 000000000..5ee329e4e
--- /dev/null
+++ b/src/Specific/NISTP256/AMD128/feadd.v
@@ -0,0 +1,14 @@
+Require Import Crypto.Arithmetic.PrimeFieldTheorems.
+Require Import Crypto.Specific.NISTP256.AMD128.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.