aboutsummaryrefslogtreecommitdiff
path: root/src/Specific/solinas32_2e216m2e108m1_10limbs/CurveParameters.v
diff options
context:
space:
mode:
authorGravatar jadep <jade.philipoom@gmail.com>2017-11-10 13:19:57 -0500
committerGravatar jadep <jade.philipoom@gmail.com>2017-11-12 15:01:59 -0500
commit795d24349b9aca1d9732c7b7fcaa505f24fa4bc6 (patch)
treef517d6c4e83f42e72a303e06567f779c0250fc2e /src/Specific/solinas32_2e216m2e108m1_10limbs/CurveParameters.v
parent7ad53a35ed68777cd21226998a88494e1d97c63e (diff)
new autogenerated files
Diffstat (limited to 'src/Specific/solinas32_2e216m2e108m1_10limbs/CurveParameters.v')
-rw-r--r--src/Specific/solinas32_2e216m2e108m1_10limbs/CurveParameters.v39
1 files changed, 39 insertions, 0 deletions
diff --git a/src/Specific/solinas32_2e216m2e108m1_10limbs/CurveParameters.v b/src/Specific/solinas32_2e216m2e108m1_10limbs/CurveParameters.v
new file mode 100644
index 000000000..bb4a23959
--- /dev/null
+++ b/src/Specific/solinas32_2e216m2e108m1_10limbs/CurveParameters.v
@@ -0,0 +1,39 @@
+Require Import Crypto.Specific.Framework.RawCurveParameters.
+Require Import Crypto.Util.LetIn.
+
+(***
+Modulus : 2^216 - 2^108 - 1
+Base: 21.6
+***)
+
+Definition curve : CurveParameters :=
+ {|
+ sz := 10%nat;
+ base := 21 + 3/5;
+ bitwidth := 32;
+ s := 2^216;
+ c := [(1, 1); (2^108, 1)];
+ carry_chains := Some [[4; 9]; [5; 0; 6; 1; 7; 2; 8; 3; 9; 4]; [5; 0]]%nat;
+
+ a24 := None;
+ coef_div_modulus := Some 2%nat;
+
+ goldilocks := Some true;
+ karatsuba := None;
+ montgomery := false;
+ freeze := Some true;
+ ladderstep := false;
+
+ mul_code := None;
+
+ square_code := None;
+
+ upper_bound_of_exponent_loose := None;
+ upper_bound_of_exponent_tight := None;
+ allowable_bit_widths := None;
+ freeze_extra_allowable_bit_widths := None;
+ modinv_fuel := None
+ |}.
+
+Ltac extra_prove_mul_eq _ := idtac.
+Ltac extra_prove_square_eq _ := idtac.