aboutsummaryrefslogtreecommitdiff
path: root/src/SpecificGen/GF25519_32Reflective/Reified/CarryOpp.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/SpecificGen/GF25519_32Reflective/Reified/CarryOpp.v')
-rw-r--r--src/SpecificGen/GF25519_32Reflective/Reified/CarryOpp.v17
1 files changed, 0 insertions, 17 deletions
diff --git a/src/SpecificGen/GF25519_32Reflective/Reified/CarryOpp.v b/src/SpecificGen/GF25519_32Reflective/Reified/CarryOpp.v
deleted file mode 100644
index 9a3eb5cb4..000000000
--- a/src/SpecificGen/GF25519_32Reflective/Reified/CarryOpp.v
+++ /dev/null
@@ -1,17 +0,0 @@
-Require Import Crypto.SpecificGen.GF25519_32Reflective.CommonUnOp.
-
-Definition rcarry_oppZ_sig : rexpr_unop_sig carry_opp. Proof. reify_sig. Defined.
-Definition rcarry_oppW := Eval vm_compute in rword_of_Z rcarry_oppZ_sig.
-Lemma rcarry_oppW_correct_and_bounded_gen : correct_and_bounded_genT rcarry_oppW rcarry_oppZ_sig.
-Proof. rexpr_correct. Qed.
-Definition rcarry_opp_output_bounds := Eval vm_compute in compute_bounds rcarry_oppW ExprUnOp_bounds.
-Local Obligation Tactic := intros; vm_compute; constructor.
-Program Definition rcarry_oppW_correct_and_bounded
- := ExprUnOp_correct_and_bounded
- rcarry_oppW carry_opp rcarry_oppZ_sig rcarry_oppW_correct_and_bounded_gen
- _ _.
-
-Local Open Scope string_scope.
-Compute ("Carry_Opp", compute_bounds_for_display rcarry_oppW ExprUnOp_bounds).
-Compute ("Carry_Opp overflows? ", sanity_compute rcarry_oppW ExprUnOp_bounds).
-Compute ("Carry_Opp overflows (error if it does)? ", sanity_check rcarry_oppW ExprUnOp_bounds).