aboutsummaryrefslogtreecommitdiff
path: root/src/Specific/GF25519Reflective/Reified/Mul.v
diff options
context:
space:
mode:
authorGravatar Jason Gross <jgross@mit.edu>2016-11-01 20:25:52 -0400
committerGravatar Jason Gross <jgross@mit.edu>2016-11-01 20:27:30 -0400
commite37f87b260b75bd5c9e3581b9e1e6cd278bf5820 (patch)
treefee5561d8023e5203d012b81b28e4b1f407864f3 /src/Specific/GF25519Reflective/Reified/Mul.v
parent9656c7d59727cef2266d611c41c4cb5dd79c19c6 (diff)
Print out the computed bounds on the various ops
Apparently some of them overflow (carry_opp, opp, sub, carry_sub) Also the bounds on ge_modulus are probably wrong, given that it's claiming that the function always returns 0. cc @andres-erbsen @jadep
Diffstat (limited to 'src/Specific/GF25519Reflective/Reified/Mul.v')
-rw-r--r--src/Specific/GF25519Reflective/Reified/Mul.v4
1 files changed, 4 insertions, 0 deletions
diff --git a/src/Specific/GF25519Reflective/Reified/Mul.v b/src/Specific/GF25519Reflective/Reified/Mul.v
index 2c19b8a5e..f1b775754 100644
--- a/src/Specific/GF25519Reflective/Reified/Mul.v
+++ b/src/Specific/GF25519Reflective/Reified/Mul.v
@@ -4,3 +4,7 @@ Definition rmulZ_sig : rexpr_binop_sig mul. Proof. reify_sig. Defined.
Definition rmulW := Eval vm_compute in rword_of_Z rmulZ_sig.
Lemma rmulW_correct_and_bounded_gen : correct_and_bounded_genT rmulW rmulZ_sig.
Proof. rexpr_correct. Qed.
+Definition rmul_output_bounds := Eval vm_compute in compute_bounds rmulW ExprBinOp_bounds.
+
+Local Open Scope string_scope.
+Compute ("Mul", compute_bounds_for_display rmulW ExprBinOp_bounds).