aboutsummaryrefslogtreecommitdiff
path: root/src/Specific/GF25519Reflective/Reified/CarrySub.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/Specific/GF25519Reflective/Reified/CarrySub.v')
-rw-r--r--src/Specific/GF25519Reflective/Reified/CarrySub.v4
1 files changed, 4 insertions, 0 deletions
diff --git a/src/Specific/GF25519Reflective/Reified/CarrySub.v b/src/Specific/GF25519Reflective/Reified/CarrySub.v
index ac70dec14..e7c2c53ab 100644
--- a/src/Specific/GF25519Reflective/Reified/CarrySub.v
+++ b/src/Specific/GF25519Reflective/Reified/CarrySub.v
@@ -4,3 +4,7 @@ Definition rcarry_subZ_sig : rexpr_binop_sig carry_sub. Proof. reify_sig. Define
Definition rcarry_subW := Eval vm_compute in rword_of_Z rcarry_subZ_sig.
Lemma rcarry_subW_correct_and_bounded_gen : correct_and_bounded_genT rcarry_subW rcarry_subZ_sig.
Proof. rexpr_correct. Qed.
+Definition rcarry_sub_output_bounds := Eval vm_compute in compute_bounds rcarry_subW ExprBinOp_bounds.
+
+Local Open Scope string_scope.
+Compute ("Carry_Sub", compute_bounds_for_display rcarry_subW ExprBinOp_bounds).