aboutsummaryrefslogtreecommitdiff
path: root/src/Specific/GF25519.v
diff options
context:
space:
mode:
authorGravatar Andres Erbsen <andreser@mit.edu>2016-06-20 03:57:41 -0400
committerGravatar Andres Erbsen <andreser@mit.edu>2016-06-20 03:57:41 -0400
commitf9b01300a6f8233b967075a04103b64a773841dc (patch)
tree3544e79f752b70b8a9d75af3f80a482a3491b379 /src/Specific/GF25519.v
parent3febea4ed8fdb255c634acbeb3705c88baa89303 (diff)
GF25519: quiet
Diffstat (limited to 'src/Specific/GF25519.v')
-rw-r--r--src/Specific/GF25519.v6
1 files changed, 4 insertions, 2 deletions
diff --git a/src/Specific/GF25519.v b/src/Specific/GF25519.v
index 7e0e815e5..ff7bff8e1 100644
--- a/src/Specific/GF25519.v
+++ b/src/Specific/GF25519.v
@@ -57,8 +57,9 @@ Proof.
pose proof (carry_mul_opt_rep k_ c_ (eq_refl k_) c_subst _ _ _ _ Hf Hg) as Hfg.
compute_formula.
exact Hfg.
-Time Defined.
+(*Time*) Defined.
+(* Uncomment this to see a pretty-printed mulmod
Local Transparent Let_In.
Infix "<<" := Z.shiftr (at level 50).
Infix "&" := Z.land (at level 50).
@@ -68,6 +69,7 @@ Eval cbv beta iota delta [proj1_sig GF25519Base25Point5_mul_reduce_formula Let_I
GF25519Base25Point5_mul_reduce_formula f0 f1 f2 f3 f4 f5 f6 f7 f8 f9
g0 g1 g2 g3 g4 g5 g6 g7 g8 g9).
Local Opaque Let_In.
+*)
Extraction "/tmp/test.ml" GF25519Base25Point5_mul_reduce_formula.
@@ -169,7 +171,7 @@ Definition F25519Rep_mul (f g:F25519Rep) : F25519Rep.
clear r;
exact (r9, r8, r7, r6, r5, r4, r3, r2, r1, r0)
end.
-Time Defined.
+(*Time*) Defined.
Lemma F25519_mul_OK : RepBinOpOK F25519RepConversions ModularArithmetic.mul F25519Rep_mul.
cbv iota beta delta [RepBinOpOK F25519RepConversions F25519Rep_mul toRep unRep F25519toRep F25519unRep].