aboutsummaryrefslogtreecommitdiff
path: root/src/Spec/EdDSA.v
diff options
context:
space:
mode:
authorGravatar Andres Erbsen <andreser@mit.edu>2016-04-22 15:27:42 -0400
committerGravatar Andres Erbsen <andreser@mit.edu>2016-04-22 15:27:42 -0400
commit2b43845eabdb5522162d52a86ecf6dfaf6dbc847 (patch)
tree00c193d89adbd22bac516072164b76f363241d9e /src/Spec/EdDSA.v
parent30ef733d1a5820456d5e5aac774270b51a9c9dde (diff)
point_eq_dec
Diffstat (limited to 'src/Spec/EdDSA.v')
-rw-r--r--src/Spec/EdDSA.v5
1 files changed, 4 insertions, 1 deletions
diff --git a/src/Spec/EdDSA.v b/src/Spec/EdDSA.v
index 3decae6a7..8a48f4dea 100644
--- a/src/Spec/EdDSA.v
+++ b/src/Spec/EdDSA.v
@@ -6,6 +6,7 @@ Require Import Crypto.Util.WordUtil.
Require Bedrock.Word.
Require Coq.ZArith.Znumtheory Coq.ZArith.BinInt.
Require Coq.Numbers.Natural.Peano.NPeano.
+Require Crypto.CompleteEdwardsCurve.CompleteEdwardsCurveTheorems.
Coercion Word.wordToNat : Word.word >-> nat.
@@ -54,6 +55,8 @@ Section EdDSA.
Notation secretkey := (Word.word b) (only parsing).
Notation publickey := (Word.word b) (only parsing).
Notation signature := (Word.word (b + b)) (only parsing).
+ Let point_eq_dec : forall P Q, {P = Q} + {P <> Q} := CompleteEdwardsCurveTheorems.point_eq_dec.
+ Local Infix "==" := point_eq_dec (at level 70) : E_scope .
(* TODO: proofread curveKey and definition of n *)
Definition curveKey (sk:secretkey) : nat :=
@@ -82,4 +85,4 @@ Section EdDSA.
end
end
end%E.
-End EdDSA.
+End EdDSA. \ No newline at end of file