aboutsummaryrefslogtreecommitdiff
path: root/src/Rep/ECRep.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/Rep/ECRep.v')
-rw-r--r--src/Rep/ECRep.v12
1 files changed, 5 insertions, 7 deletions
diff --git a/src/Rep/ECRep.v b/src/Rep/ECRep.v
index b42e1e067..60481fe72 100644
--- a/src/Rep/ECRep.v
+++ b/src/Rep/ECRep.v
@@ -1,18 +1,16 @@
-Require Export Crypto.Galois.Galois Crypto.Galois.GaloisTheory.
-Require Import Crypto.Galois.AbstractGaloisField.
+Require Export Crypto.Galois.GaloisField.
Module ECRep (M: Modulus).
- Module G := Galois M.
- Module F := AbstractGaloisField M.
- Import M G F.
+ Module F := GaloisField M.
+ Import F.
Local Open Scope GF_scope.
- Definition ECSig : ADTSig :=
+ (* Definition ECSig : ADTSig :=
ADTsignature {
Constructor "FromTwistedXY"
: GF x GF -> rep,
Method "Add"
: rep x rep -> rep,
- }.
+ }.*)
End ECRep.