From 60520cd8d08f63337225c0a2938827e00a2c48a3 Mon Sep 17 00:00:00 2001 From: Jason Gross Date: Wed, 10 Apr 2019 16:41:34 -0400 Subject: sed s'/RewriterProofs/RewriterAll/g' --- src/BoundsPipeline.v | 6 +++--- 1 file changed, 3 insertions(+), 3 deletions(-) (limited to 'src/BoundsPipeline.v') 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 -- cgit v1.2.3