aboutsummaryrefslogtreecommitdiff
path: root/src/Primitives/EdDSARepChange.v
diff options
context:
space:
mode:
authorGravatar Samuel Gruetter <samuel.gruetter@epfl.ch>2018-02-02 16:09:01 -0500
committerGravatar Jason Gross <jasongross9@gmail.com>2018-02-05 16:07:28 -0500
commit3fd5f652ba38a0b308b6e2e86783d82b861fb5bf (patch)
treefd3752dd3a4bb9b216bcc5eabeb320a8ed9ffba4 /src/Primitives/EdDSARepChange.v
parente11d6d06e6eda3cd5940765dbbea420416725832 (diff)
minor updates needed to make it compile with bbv
removing lemma wordToNat_wzero is ok because it's already in bbv
Diffstat (limited to 'src/Primitives/EdDSARepChange.v')
-rw-r--r--src/Primitives/EdDSARepChange.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/src/Primitives/EdDSARepChange.v b/src/Primitives/EdDSARepChange.v
index 9239b9c81..d867a62df 100644
--- a/src/Primitives/EdDSARepChange.v
+++ b/src/Primitives/EdDSARepChange.v
@@ -1,5 +1,5 @@
Require Import Crypto.Util.FixCoqMistakes.
-Require Import Crypto.Spec.EdDSA Bedrock.Word.
+Require Import Crypto.Spec.EdDSA bbv.WordScope.
Require Import Coq.Classes.Morphisms Coq.Relations.Relation_Definitions.
Require Import Crypto.Algebra.Monoid Crypto.Algebra.Group Crypto.Algebra.ScalarMult.
Require Import Crypto.Util.Decidable Crypto.Util.Option.