aboutsummaryrefslogtreecommitdiff
path: root/src/Experiments/NewPipeline/Toplevel1.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/Experiments/NewPipeline/Toplevel1.v')
-rw-r--r--src/Experiments/NewPipeline/Toplevel1.v3
1 files changed, 3 insertions, 0 deletions
diff --git a/src/Experiments/NewPipeline/Toplevel1.v b/src/Experiments/NewPipeline/Toplevel1.v
index 437855405..3b8f81ac6 100644
--- a/src/Experiments/NewPipeline/Toplevel1.v
+++ b/src/Experiments/NewPipeline/Toplevel1.v
@@ -52,6 +52,7 @@ Require Crypto.Experiments.NewPipeline.LanguageWf.
Require Crypto.Experiments.NewPipeline.UnderLetsProofs.
Require Crypto.Experiments.NewPipeline.MiscCompilerPassesProofs.
Require Crypto.Experiments.NewPipeline.RewriterProofs.
+Require Crypto.Experiments.NewPipeline.AbstractInterpretationWf.
Require Crypto.Experiments.NewPipeline.AbstractInterpretationProofs.
Require Import Crypto.Util.Notations.
Import ListNotations. Local Open Scope Z_scope.
@@ -499,6 +500,7 @@ Import
Crypto.Experiments.NewPipeline.UnderLetsProofs
Crypto.Experiments.NewPipeline.MiscCompilerPassesProofs
Crypto.Experiments.NewPipeline.RewriterProofs
+ Crypto.Experiments.NewPipeline.AbstractInterpretationWf
Crypto.Experiments.NewPipeline.AbstractInterpretationProofs
Crypto.Experiments.NewPipeline.Language
Crypto.Experiments.NewPipeline.UnderLets
@@ -512,6 +514,7 @@ Import
UnderLetsProofs.Compilers
MiscCompilerPassesProofs.Compilers
RewriterProofs.Compilers
+ AbstractInterpretationWf.Compilers
AbstractInterpretationProofs.Compilers
Language.Compilers
UnderLets.Compilers