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