aboutsummaryrefslogtreecommitdiff
path: root/src/Specific/X25519/C64/ReificationTypes.v
blob: 0e999b2fc42b5d1ded0f505d80aa90826e1d7689 (plain)
1
2
3
4
5
6
7
8
9
10
11
12
Require Import Crypto.Specific.ReificationTypes.
Require Import Crypto.Specific.X25519.C64.ArithmeticSynthesisTest.

Module RP <: ReificationTypesPrePackage.
  Definition ReificationTypes_package' : { T : _ & T }.
  Proof. make_ReificationTypes_package wt sz bounds m wt_nonneg P.upper_bound_of_exponent. Defined.

  Definition ReificationTypes_package
    := Eval cbv [ReificationTypes_package' projT2] in projT2 ReificationTypes_package'.
End RP.

Module Export ReificationTypes := MakeReificationTypes RP.