aboutsummaryrefslogtreecommitdiff
path: root/src/Experiments
diff options
context:
space:
mode:
authorGravatar jadep <jade.philipoom@gmail.com>2016-10-27 13:39:06 -0400
committerGravatar jadep <jade.philipoom@gmail.com>2016-10-27 13:39:21 -0400
commitcefea49230f2e2f4010e0b02a27bc55a48125f34 (patch)
tree57de6d8e876839c3536051a43fbebd4ed48b0e5f /src/Experiments
parent6730c30f7932c1170dbf249efd332dd21cb38f5f (diff)
removed now irrelevant commented-out code
Diffstat (limited to 'src/Experiments')
-rw-r--r--src/Experiments/Ed25519.v33
1 files changed, 0 insertions, 33 deletions
diff --git a/src/Experiments/Ed25519.v b/src/Experiments/Ed25519.v
index a25e7c73f..e8f7a8f04 100644
--- a/src/Experiments/Ed25519.v
+++ b/src/Experiments/Ed25519.v
@@ -534,39 +534,6 @@ Qed.
Lemma Proper_feEnc : Proper (GF25519BoundedCommon.eq ==> eq) feEnc.
Admitted.
-(*
-Lemma ext_to_coord_coord_to_ext : forall (P : GF25519BoundedCommon.fe25519 * GF25519BoundedCommon.fe25519)
- (pf : Pre.onCurve P),
- Tuple.fieldwise (n := 2)
- GF25519BoundedCommon.eq
- (extended_to_coord (coord_to_extended P pf))
- P.
-Proof.
- cbv [extended_to_coord coord_to_extended].
- intros.
- transitivity (CompleteEdwardsCurve.E.coordinates (exist _ P pf));
- [ | reflexivity].
- apply (CompleteEdwardsCurveTheorems.E.Proper_coordinates
- (field := GF25519Bounded.field25519) (a := a) (d := d)).
- apply ExtendedCoordinates.Extended.to_twisted_from_twisted.
-Qed.
- *)
-(*
-Lemma to_twist
- ed_from_twisted_coordinates_eq :
- forall pt : E,
- Tuple.fieldwise ModularBaseSystem.eq (n := 2)
- ((fun P0 : Erep =>
- CompleteEdwardsCurve.E.coordinates
- (ExtendedCoordinates.Extended.to_twisted (field := GF25519.field25519) P0))
- (ExtendedCoordinates.Extended.from_twisted (field := PrimeFieldTheorems.F.field_modulo GF25519.modulus) pt))
- (CompleteEdwardsCurve.E.coordinates pt).
-Proof.
- intros.
- pose proof ExtendedCoordinates.Extended.to_twisted_from_twisted.
- specialize (H0 pt).
-*)
-
Lemma ERepEnc_correct P : Eenc P = ERepEnc (EToRep P).
Proof.
cbv [Eenc ERepEnc EToRep sign Fencode].