aboutsummaryrefslogtreecommitdiffstats
path: root/driver/Compiler.vexpand
diff options
context:
space:
mode:
Diffstat (limited to 'driver/Compiler.vexpand')
-rw-r--r--driver/Compiler.vexpand3
1 files changed, 2 insertions, 1 deletions
diff --git a/driver/Compiler.vexpand b/driver/Compiler.vexpand
index 0f59aab7..3acec956 100644
--- a/driver/Compiler.vexpand
+++ b/driver/Compiler.vexpand
@@ -35,6 +35,7 @@ Require Cshmgen.
Require Cminorgen.
Require Selection.
Require RTLgen.
+Require Import Duplicatepasses.
EXPAND_RTL_REQUIRE
Require Asmgen.
(** Proofs of semantic preservation. *)
@@ -53,7 +54,7 @@ Require Import Compopts.
Parameter print_Clight: Clight.program -> unit.
Parameter print_Cminor: Cminor.program -> unit.
Parameter print_RTL: Z -> RTL.program -> unit.
-Parameter print_LTL: LTL.program -> unit.
+Parameter print_LTL: Z -> LTL.program -> unit.
Parameter print_Mach: Mach.program -> unit.
Local Open Scope string_scope.