aboutsummaryrefslogtreecommitdiff
path: root/src/Specific/X2448/Karatsuba/C64/Synthesis.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/Specific/X2448/Karatsuba/C64/Synthesis.v')
-rw-r--r--src/Specific/X2448/Karatsuba/C64/Synthesis.v9
1 files changed, 3 insertions, 6 deletions
diff --git a/src/Specific/X2448/Karatsuba/C64/Synthesis.v b/src/Specific/X2448/Karatsuba/C64/Synthesis.v
index 8ea8aa5c9..500671c90 100644
--- a/src/Specific/X2448/Karatsuba/C64/Synthesis.v
+++ b/src/Specific/X2448/Karatsuba/C64/Synthesis.v
@@ -3,12 +3,9 @@ Require Import Crypto.Specific.X2448.Karatsuba.C64.CurveParameters.
Module Import T := MakeSynthesisTactics Curve.
-Module P <: SynthesisPrePackage.
- Definition Synthesis_package' : Synthesis_package'_Type.
- Proof. make_synthesis_package (). Defined.
-
- Definition Synthesis_package
- := Eval cbv [Synthesis_package' projT2] in projT2 Synthesis_package'.
+Module P <: PrePackage.
+ Definition package : Tag.Context.
+ Proof. make_Synthesis_package (). Defined.
End P.
Module Export S := PackageSynthesis Curve P.