aboutsummaryrefslogtreecommitdiffstats
path: root/src/Compiler.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/Compiler.v')
-rw-r--r--src/Compiler.v7
1 files changed, 6 insertions, 1 deletions
diff --git a/src/Compiler.v b/src/Compiler.v
index a34b359..17d8921 100644
--- a/src/Compiler.v
+++ b/src/Compiler.v
@@ -48,7 +48,9 @@ From compcert.driver Require
From coqup Require
Verilog
Veriloggen
- HTLgen.
+ Veriloggenproof
+ HTLgen
+ HTLgenproof.
Parameter print_RTL: Z -> RTL.program -> unit.
Parameter print_HTL: HTL.program -> unit.
@@ -107,6 +109,9 @@ Definition CompCert's_passes :=
::: mkpass Cminorgenproof.match_prog
::: mkpass Selectionproof.match_prog
::: mkpass RTLgenproof.match_prog
+ ::: mkpass Inliningproof.match_prog
+ ::: mkpass HTLgenproof.match_prog
+ ::: mkpass Veriloggenproof.match_prog
::: pass_nil _.
Definition match_prog: Csyntax.program -> RTL.program -> Prop :=