aboutsummaryrefslogtreecommitdiff
path: root/src/CompilersTestCases.v
diff options
context:
space:
mode:
authorGravatar Jason Gross <jgross@mit.edu>2019-04-10 16:41:34 -0400
committerGravatar Jason Gross <jasongross9@gmail.com>2019-04-11 11:01:29 -0400
commit60520cd8d08f63337225c0a2938827e00a2c48a3 (patch)
treeaaf3a2a7b75aabc1dee784c49da868907f4a1b54 /src/CompilersTestCases.v
parentbe2789ada63a1a5a6710da1abc73430f9b676399 (diff)
sed s'/RewriterProofs/RewriterAll/g'
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 2ed149cdd..91fc3af1d 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.RewriterProofs.
+Require Import Crypto.RewriterAll.
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 RewriterProofs.Compilers.
+Import RewriterAll.Compilers.
Import MiscCompilerPasses.Compilers.
Import CStringification.Compilers.
Local Coercion Z.of_nat : nat >-> Z.