aboutsummaryrefslogtreecommitdiff
path: root/src/Specific/GF25519ReflectiveAddCoordinates.v
diff options
context:
space:
mode:
authorGravatar Jason Gross <jgross@mit.edu>2017-01-11 21:02:50 -0500
committerGravatar Jason Gross <jasongross9@gmail.com>2017-03-01 11:45:47 -0500
commit6b3048c37ad348dc88ecc03ef892ecfb121bfa7f (patch)
tree351e5438c5664ab0caf08b9d5054f296ff4aa2ee /src/Specific/GF25519ReflectiveAddCoordinates.v
parent80dc66a34fbf031bfac1214ccbb3bb1dcdef3d39 (diff)
Switch to fully uncurried form for reflection
This will eventually make a number of proofs easier. Unfortunately, the correctness lemmas for AddCoordinates and LadderStep no longer work (because of different arities), and there's a proof in Experiments/Ed25519 that I've admitted. The correctness lemmas will be easy to re-add when we have a more general version that handle arbitrary type shapes.
Diffstat (limited to 'src/Specific/GF25519ReflectiveAddCoordinates.v')
-rw-r--r--src/Specific/GF25519ReflectiveAddCoordinates.v5
1 files changed, 3 insertions, 2 deletions
diff --git a/src/Specific/GF25519ReflectiveAddCoordinates.v b/src/Specific/GF25519ReflectiveAddCoordinates.v
index c4e88f2a7..c40c093ed 100644
--- a/src/Specific/GF25519ReflectiveAddCoordinates.v
+++ b/src/Specific/GF25519ReflectiveAddCoordinates.v
@@ -32,7 +32,7 @@ Import ListNotations.
Require Import Coq.ZArith.ZArith Coq.ZArith.Zpower Coq.ZArith.ZArith Coq.ZArith.Znumtheory.
Local Open Scope Z.
-Time Definition radd_coordinates : Expr9_4Op := Eval vm_compute in radd_coordinatesW.
+Time Definition radd_coordinates : Expr _ := Eval vm_compute in radd_coordinatesW.
Declare Reduction asm_interp_add_coordinates
:= cbv beta iota delta
@@ -57,7 +57,7 @@ Ltac asm_interp_add_coordinates
mapf_interp_flat_type WordW.interp_base_type word64ize
Interp interp interp_flat_type interpf interp_flat_type fst snd].
-
+(*
Time Definition interp_radd_coordinates : Specific.GF25519BoundedCommon.fe25519W
-> Specific.GF25519BoundedCommon.fe25519W
-> Specific.GF25519BoundedCommon.fe25519W
@@ -74,3 +74,4 @@ Time Definition interp_radd_coordinates_correct : interp_radd_coordinates = inte
Lemma radd_coordinates_correct_and_bounded : op9_4_correct_and_bounded radd_coordinates add_coordinates.
Proof. exact_no_check radd_coordinatesW_correct_and_bounded. Time Qed.
+*)