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

Definition rsubZ_sig : rexpr_binop_sig sub. Proof. reify_sig. Defined.