aboutsummaryrefslogtreecommitdiff
path: root/src/Spec/MontgomeryCurve.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/Spec/MontgomeryCurve.v')
-rw-r--r--src/Spec/MontgomeryCurve.v131
1 files changed, 50 insertions, 81 deletions
diff --git a/src/Spec/MontgomeryCurve.v b/src/Spec/MontgomeryCurve.v
index 5f7246011..2717f6bbc 100644
--- a/src/Spec/MontgomeryCurve.v
+++ b/src/Spec/MontgomeryCurve.v
@@ -6,7 +6,7 @@ Require Import Crypto.Spec.WeierstrassCurve.
Module M.
Section MontgomeryCurve.
Import BinNat.
- Context {F Feq Fzero Fone Fopp Fadd Fsub Fmul Finv Fdiv} {field:@Algebra.field F Feq Fzero Fone Fopp Fadd Fsub Fmul Finv Fdiv} {Feq_dec:Decidable.DecidableRel Feq} {char_gt_2:@Ring.char_gt F Feq Fzero Fone Fopp Fadd Fsub Fmul (BinNat.N.succ_pos (BinNat.N.two))}.
+ Context {F Feq Fzero Fone Fopp Fadd Fsub Fmul Finv Fdiv} {field:@Algebra.field F Feq Fzero Fone Fopp Fadd Fsub Fmul Finv Fdiv} {Feq_dec:Decidable.DecidableRel Feq} {char_ge_3:@Ring.char_ge F Feq Fzero Fone Fopp Fadd Fsub Fmul (BinNat.N.succ_pos (BinNat.N.two))}.
Local Infix "=" := Feq : type_scope. Local Notation "a <> b" := (not (a = b)) : type_scope.
Local Infix "+" := Fadd. Local Infix "*" := Fmul.
Local Infix "-" := Fsub. Local Infix "/" := Fdiv.
@@ -28,20 +28,26 @@ Module M.
end }.
Definition coordinates (P:point) : (F*F + ∞) := proj1_sig P.
+ Definition eq (P1 P2:point) :=
+ match coordinates P1, coordinates P2 with
+ | (x1, y1), (x2, y2) => x1 = x2 /\ y1 = y2
+ | ∞, ∞ => True
+ | _, _ => False
+ end.
+
Import Crypto.Util.Tactics Crypto.Algebra.Field.
Ltac t :=
destruct_head' point; destruct_head' sum; destruct_head' prod;
break_match; simpl in *; break_match_hyps; trivial; try discriminate;
repeat match goal with
| |- _ /\ _ => split
- | [H:@eq (sum _ _ ) _ _ |- _] => symmetry in H; injection H; intros; clear H
- | [H:@eq (prod _ _ ) _ _ |- _] => symmetry in H; injection H; intros; clear H
+ | [H:@Logic.eq (sum _ _ ) _ _ |- _] => symmetry in H; injection H; intros; clear H
+ | [H:@Logic.eq (prod _ _ ) _ _ |- _] => symmetry in H; injection H; intros; clear H
end;
subst; try fsatz.
Program Definition add (P1 P2:point) : point :=
- exist _
- match coordinates P1, coordinates P2 return _ with
+ match coordinates P1, coordinates P2 return F*F+∞ with
(x1, y1), (x2, y2) =>
if Decidable.dec (x1 = x2)
then if Decidable.dec (y1 = - y2)
@@ -51,53 +57,39 @@ Module M.
| ∞, ∞ => ∞
| ∞, _ => coordinates P2
| _, ∞ => coordinates P1
- end _.
+ end.
Next Obligation. Proof. t. Qed.
Program Definition opp (P:point) : point :=
- exist _
- match P with
- | (x, y) => (x, -y)
- | ∞ => ∞
- end _.
- Next Obligation.
- Proof. t. Qed.
+ match P return F*F+∞ with
+ | (x, y) => (x, -y)
+ | ∞ => ∞
+ end.
+ Next Obligation. Proof. t. Qed.
Local Notation "4" := (1+3).
Local Notation "16" := (4*4).
Local Notation "9" := (3*3).
Local Notation "27" := (3*9).
- Context {char_gt_27:@Ring.char_gt F Feq Fzero Fone Fopp Fadd Fsub Fmul 27}.
+ Context {char_ge_28:@Ring.char_ge F Feq Fzero Fone Fopp Fadd Fsub Fmul 28}.
Let WeierstrassA := ((3-a^2)/(3*b^2)).
Let WeierstrassB := ((2*a^3-9*a)/(27*b^3)).
-
Local Notation Wpoint := (@W.point F Feq Fadd Fmul WeierstrassA WeierstrassB).
- Program Definition MontgomeryOfWeierstrass (P:Wpoint) : point :=
- exist
- _
- match W.coordinates P return _ with
- | (x,y) => (b*x-a/3, b*y)
- | _ => ∞
- end
- _.
- Next Obligation.
- Proof. subst WeierstrassA; subst WeierstrassB; destruct P; t. Qed.
+ Local Notation Wadd := (@W.add F Feq Fzero Fone Fopp Fadd Fsub Fmul Finv Fdiv field Feq_dec char_ge_3 WeierstrassA WeierstrassB).
- Definition eq (P1 P2:point) :=
- match coordinates P1, coordinates P2 with
- | (x1, y1), (x2, y2) => x1 = x2 /\ y1 = y2
- | ∞, ∞ => True
- | _, _ => False
+ Program Definition of_Weierstrass (P:Wpoint) : point :=
+ match W.coordinates P return F*F+∞ with
+ | (x,y) => (b*x-a/3, b*y)
+ | _ => ∞
end.
+ Next Obligation.
+ Proof. clear char_ge_3; subst WeierstrassA; subst WeierstrassB; destruct P; t. Qed.
- Local Notation Wadd := (@W.add F Feq Fzero Fone Fopp Fadd Fsub Fmul Finv Fdiv field Feq_dec char_gt_2 WeierstrassA WeierstrassB).
- Lemma MontgomeryOfWeierstrass_add P1 P2 :
- eq (MontgomeryOfWeierstrass (W.add P1 P2))
- (add (MontgomeryOfWeierstrass P1) (MontgomeryOfWeierstrass P2)).
- Proof.
- cbv [WeierstrassA WeierstrassB eq MontgomeryOfWeierstrass W.add add coordinates W.coordinates proj1_sig] in *; t.
- Qed.
+ Lemma of_Weierstrass_add P1 P2 :
+ eq (of_Weierstrass (W.add P1 P2))
+ (add (of_Weierstrass P1) (of_Weierstrass P2)).
+ Proof. cbv [WeierstrassA WeierstrassB eq of_Weierstrass W.add add coordinates W.coordinates proj1_sig] in *; clear char_ge_3; t. Qed.
Section AddX.
Lemma homogeneous_x_differential_addition_releations P1 P2 :
@@ -110,30 +102,20 @@ Module M.
end.
Proof. t. Qed.
- Definition onCurve xy := let 'pair x y := xy in b*y^2 = x^3 + a*x^2 + x.
- Definition xzpoint := { xz | let 'pair x z := xz in (z = 0 \/ exists y, onCurve (pair (x/z) y)) }.
- Definition xzcoordinates (P:xzpoint) : F*F := proj1_sig P.
- Program Definition toxz (P:point) : xzpoint :=
- exist _
- match coordinates P with
- | (x, y) => pair x 1
- | ∞ => pair 1 0
- end _.
- Next Obligation. t; [right; exists f0; t | left; reflexivity ]. Qed.
-
- Definition sig_pair_to_pair_sig {T T' I I'} (xy:{xy | let 'pair x y := xy in I x /\ I' y})
- : prod {x:T | I x} {y:T' | I' y}
- := let 'exist (pair x y) (conj pfx pfy) := xy in pair (exist _ x pfx) (exist _ y pfy).
+ Program Definition to_xz (P:point) : F*F :=
+ match coordinates P with
+ | (x, y) => pair x 1
+ | ∞ => pair 1 0
+ end.
(* From Explicit Formulas Database by Lange and Bernstein,
credited to 1987 Montgomery "Speeding the Pollard and elliptic curve
methods of factorization", page 261, fifth and sixth displays, plus
common-subexpression elimination, plus assumption Z1=1 *)
- Context {a24:F} {a24_correct:4*a24 = a+2}.
- Definition xzladderstep (X1:F) (P1 P2:xzpoint) : prod xzpoint xzpoint. refine (
- sig_pair_to_pair_sig (exist _
- match xzcoordinates P1, xzcoordinates P2 return _ with
+ Context {a24:F} {a24_correct:4*a24 = a+2}. (* TODO: +2 or -2 ? *)
+ Definition xzladderstep (X1:F) (P1 P2:F*F) : ((F*F)*(F*F)) :=
+ match P1, P2 with
pair X2 Z2, pair X3 Z3 =>
let A := X2+Z2 in
let AA := A^2 in
@@ -149,32 +131,19 @@ Module M.
let X4 := AA*BB in
let Z4 := E*(BB + a24*E) in
(pair (pair X4 Z4) (pair X5 Z5))
- end _) ).
- Proof.
- destruct P1, P2; cbv [onCurve xzcoordinates] in *. t; intuition idtac.
- { left. fsatz. }
- { left. fsatz. }
- admit.
- admit.
- admit.
- admit.
- { right.
- admit. (* the following used to work, but slowly:
- exists ((fun x1 y1 x2 y2 => (2*x1+x1+a)*(3*x1^2+2*a*x1+1)/(2*b*y1)-b*(3*x1^2+2*a*x1+1)^3/(2*b*y1)^3-y1) (f1/f2) x0 (f/f0) x).
- Algebra.common_denominator_in H.
- Algebra.common_denominator_in H0.
- Algebra.common_denominator.
- abstract Algebra.nsatz.
-
- idtac.
- admit.
- admit.
- admit.
- admit.
- admit. *) }
- { right.
- (* exists ((fun x1 y1 x2 y2 => (2*x1+x2+a)*(y2-y1)/(x2-x1)-b*(y2-y1)^3/(x2-x1)^3-y1) (f1/f2) x0 (f/f0) x). *)
- (* XXX: this case is probably not true -- there is not necessarily a guarantee that the output x/z is on curve if [X1] was not the x coordinate of the difference of input points as requored *)
+ end.
+
+ Require Import Crypto.Util.Tuple.
+
+ (* TODO: look up this lemma statement -- the current one may not be right *)
+ Lemma xzladderstep_to_xz X1 P1 P2
+ (HX1 : match coordinates (add P1 (opp P2)) with (x,y) => X1 = x | _ => False end)
+ : fieldwise (n:=2) (fieldwise (n:=2) Feq)
+ (xzladderstep X1 (to_xz P1) (to_xz P2))
+ (pair (to_xz (add P1 P2)) (to_xz (add P1 P1))).
+ destruct P1 as [[[??]|?]?], P2 as [[[??]|?]?];
+ cbv [fst snd xzladderstep to_xz add coordinates proj1_sig opp fieldwise fieldwise'] in *;
+ break_match_hyps; break_match; repeat split; try contradiction.
Abort.
End AddX.
End MontgomeryCurve.