aboutsummaryrefslogtreecommitdiff
path: root/src/Specific/GF25519Reflective/Reified/CarryAdd.v
blob: f3c65a02bf4b470fcc01022feef1fcc3451a39bb (plain)
1
2
3
Require Import Crypto.Specific.GF25519Reflective.Common.

Definition rcarry_addZ_sig : rexpr_binop_sig carry_add. Proof. reify_sig. Defined.