aboutsummaryrefslogtreecommitdiff
path: root/src/Compilers/Z/HexNotationConstants.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/Compilers/Z/HexNotationConstants.v')
-rw-r--r--src/Compilers/Z/HexNotationConstants.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/src/Compilers/Z/HexNotationConstants.v b/src/Compilers/Z/HexNotationConstants.v
index fe08c9d1f..0e365d9f8 100644
--- a/src/Compilers/Z/HexNotationConstants.v
+++ b/src/Compilers/Z/HexNotationConstants.v
@@ -1,7 +1,7 @@
Require Import Coq.ZArith.ZArith.
Require Export Crypto.Compilers.Syntax.
Require Import Crypto.Compilers.Z.Syntax.
-Require Export Bedrock.Word.
+Require Export bbv.WordScope.
Require Export Crypto.Util.Notations.
Notation Const x := (Op (OpConst x) TT).
@@ -731,7 +731,7 @@ def header():
return (r"""Require Import Coq.ZArith.ZArith.
Require Export Crypto.Compilers.Syntax.
Require Import Crypto.Compilers.Z.Syntax.
-Require Export Bedrock.Word.
+Require Export bbv.WordScope.
Require Export Crypto.Util.Notations.
Notation Const x := (Op (OpConst x) TT).