aboutsummaryrefslogtreecommitdiff
path: root/src/Specific/X25519/C64/CurveParameters.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/Specific/X25519/C64/CurveParameters.v')
-rw-r--r--src/Specific/X25519/C64/CurveParameters.v7
1 files changed, 4 insertions, 3 deletions
diff --git a/src/Specific/X25519/C64/CurveParameters.v b/src/Specific/X25519/C64/CurveParameters.v
index 9a543b569..54c578a08 100644
--- a/src/Specific/X25519/C64/CurveParameters.v
+++ b/src/Specific/X25519/C64/CurveParameters.v
@@ -11,12 +11,13 @@ Module Curve <: CurveParameters.
Definition bitwidth : Z := 64.
Definition s : Z := 2^255.
Definition c : list limb := [(1, 19)].
- Definition carry_chain1 : option (list nat) := Eval vm_compute in Some (seq 0 (pred sz)).
- Definition carry_chain2 : option (list nat) := Eval vm_compute in Some [0; 1]%nat.
+ Definition carry_chains : option (list (list nat)) := Eval vm_compute in Some [seq 0 (pred sz); [0; 1]]%nat.
- Definition a24 : Z := 121665.
+ Definition a24 : option Z := Some 121665.
Definition coef_div_modulus : nat := 2%nat. (* add 2*modulus before subtracting *)
+ Definition goldilocks : bool := false.
+
Definition mul_code : option (Z^sz -> Z^sz -> Z^sz)
:= Some (fun a b =>
(* Micro-optimized form from curve25519-donna-c64 by Adam Langley (Google) and Daniel Bernstein. See <https://github.com/agl/curve25519-donna/blob/master/LICENSE.md>. *)