aboutsummaryrefslogtreecommitdiff
path: root/src/BoundsPipeline.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/BoundsPipeline.v
parentbe2789ada63a1a5a6710da1abc73430f9b676399 (diff)
sed s'/RewriterProofs/RewriterAll/g'
Diffstat (limited to 'src/BoundsPipeline.v')
-rw-r--r--src/BoundsPipeline.v6
1 files changed, 3 insertions, 3 deletions
diff --git a/src/BoundsPipeline.v b/src/BoundsPipeline.v
index f0c161dc2..6c21d7c64 100644
--- a/src/BoundsPipeline.v
+++ b/src/BoundsPipeline.v
@@ -29,7 +29,7 @@ Require Crypto.CStringification.
Require Crypto.LanguageWf.
Require Crypto.UnderLetsProofs.
Require Crypto.MiscCompilerPassesProofs.
-Require Crypto.RewriterProofs.
+Require Crypto.RewriterAll.
Require Crypto.AbstractInterpretationWf.
Require Crypto.AbstractInterpretationProofs.
Require Import Crypto.Util.Notations.
@@ -39,7 +39,7 @@ Import
Crypto.LanguageWf
Crypto.UnderLetsProofs
Crypto.MiscCompilerPassesProofs
- Crypto.RewriterProofs
+ Crypto.RewriterAll
Crypto.AbstractInterpretationWf
Crypto.AbstractInterpretationProofs
Crypto.Language
@@ -53,7 +53,7 @@ Import
LanguageWf.Compilers
UnderLetsProofs.Compilers
MiscCompilerPassesProofs.Compilers
- RewriterProofs.Compilers
+ RewriterAll.Compilers
AbstractInterpretationWf.Compilers
AbstractInterpretationProofs.Compilers
Language.Compilers