aboutsummaryrefslogtreecommitdiff
path: root/src/CompilersTestCases.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/CompilersTestCases.v')
-rw-r--r--src/CompilersTestCases.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/src/CompilersTestCases.v b/src/CompilersTestCases.v
index 19fcf1588..2ed149cdd 100644
--- a/src/CompilersTestCases.v
+++ b/src/CompilersTestCases.v
@@ -5,7 +5,7 @@ Require Import Crypto.Util.LetIn.
Require Import Crypto.Language.
Require Import Crypto.UnderLets.
Require Import Crypto.AbstractInterpretation.
-Require Import Crypto.RewriterFull.
+Require Import Crypto.RewriterProofs.
Require Import Crypto.MiscCompilerPasses.
Require Import Crypto.CStringification.
Import ListNotations. Local Open Scope Z_scope.
@@ -13,7 +13,7 @@ Import ListNotations. Local Open Scope Z_scope.
Import Language.Compilers.
Import UnderLets.Compilers.
Import AbstractInterpretation.Compilers.
-Import RewriterFull.Compilers.
+Import RewriterProofs.Compilers.
Import MiscCompilerPasses.Compilers.
Import CStringification.Compilers.
Local Coercion Z.of_nat : nat >-> Z.