From 0b03656ba15c354165ee14eda054de4489faeb9c Mon Sep 17 00:00:00 2001 From: Jason Gross Date: Sat, 14 Oct 2017 16:01:37 -0400 Subject: Run remake_curves.py --- src/Specific/solinas32_2e137m13/femul.v | 14 ++++++++++++++ 1 file changed, 14 insertions(+) create mode 100644 src/Specific/solinas32_2e137m13/femul.v (limited to 'src/Specific/solinas32_2e137m13/femul.v') diff --git a/src/Specific/solinas32_2e137m13/femul.v b/src/Specific/solinas32_2e137m13/femul.v new file mode 100644 index 000000000..9f1d4486a --- /dev/null +++ b/src/Specific/solinas32_2e137m13/femul.v @@ -0,0 +1,14 @@ +Require Import Crypto.Arithmetic.PrimeFieldTheorems. +Require Import Crypto.Specific.solinas32_2e137m13.Synthesis. + +(* TODO : change this to field once field isomorphism happens *) +Definition mul : + { mul : feBW -> feBW -> feBW + | forall a b, phiBW (mul a b) = F.mul (phiBW a) (phiBW b) }. +Proof. + Set Ltac Profiling. + Time synthesize_mul (). + Show Ltac Profile. +Time Defined. + +Print Assumptions mul. -- cgit v1.2.3