aboutsummaryrefslogtreecommitdiff
path: root/src/Assembly/GF25519.v
diff options
context:
space:
mode:
authorGravatar Jason Gross <jgross@mit.edu>2016-10-31 02:56:19 -0400
committerGravatar Jason Gross <jgross@mit.edu>2016-10-31 02:56:19 -0400
commitd25bba72f91c3617718ec0a5eaf69c6d506e2b74 (patch)
treeae8119c1665b82a1f0e045dc42a9706d4458c481 /src/Assembly/GF25519.v
parent6fb3a24a3600a588f63ef57850c5468e446b9fb5 (diff)
Silence a warning
Diffstat (limited to 'src/Assembly/GF25519.v')
-rw-r--r--src/Assembly/GF25519.v4
1 files changed, 3 insertions, 1 deletions
diff --git a/src/Assembly/GF25519.v b/src/Assembly/GF25519.v
index e1ecfdce0..a904f14b1 100644
--- a/src/Assembly/GF25519.v
+++ b/src/Assembly/GF25519.v
@@ -7,6 +7,8 @@ Require Import Crypto.ModularArithmetic.ModularBaseSystem.
Require Import Crypto.Specific.GF25519.
Require Import Crypto.Util.Tuple.
+Require InitialRing.
+
Module GF25519.
Definition bits: nat := 64.
Definition width: Width bits := W64.
@@ -226,7 +228,7 @@ Module GF25519.
Module Opp := Pipeline OppExpr.
Section Instantiation.
- Require Import InitialRing.
+ Import InitialRing.
Definition Binary : Type := NAry 20 (word bits) (@interp_type (word bits) FE).
Definition Unary : Type := NAry 10 (word bits) (@interp_type (word bits) FE).