aboutsummaryrefslogtreecommitdiff
path: root/src/Assembly/AlmostQhasm.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/Assembly/AlmostQhasm.v')
-rw-r--r--src/Assembly/AlmostQhasm.v6
1 files changed, 3 insertions, 3 deletions
diff --git a/src/Assembly/AlmostQhasm.v b/src/Assembly/AlmostQhasm.v
index f3ed925c7..e91e20843 100644
--- a/src/Assembly/AlmostQhasm.v
+++ b/src/Assembly/AlmostQhasm.v
@@ -1,6 +1,6 @@
-Require Import QhasmCommon QhasmEvalCommon.
-Require Import Language.
-Require Import List.
+Require Import Crypto.Assembly.QhasmCommon Crypto.Assembly.QhasmEvalCommon.
+Require Import Crypto.Assembly.Language.
+Require Import Coq.Lists.List.
Module AlmostQhasm <: Language.
Import QhasmEval.