aboutsummaryrefslogtreecommitdiffstats
path: root/scheduling/RTLtoBTL.v
diff options
context:
space:
mode:
Diffstat (limited to 'scheduling/RTLtoBTL.v')
-rw-r--r--scheduling/RTLtoBTL.v3
1 files changed, 2 insertions, 1 deletions
diff --git a/scheduling/RTLtoBTL.v b/scheduling/RTLtoBTL.v
index 507fc9d9..309c616e 100644
--- a/scheduling/RTLtoBTL.v
+++ b/scheduling/RTLtoBTL.v
@@ -1,7 +1,7 @@
Require Import Coqlib Maps.
Require Import AST Integers Values Events Memory Globalenvs Smallstep.
Require Import RTL Op Registers OptionMonad BTL.
-Require Export BTLmatchRTL.
+Require Export BTLmatchRTL BTL_Livecheck.
Require Import Errors Linking.
@@ -17,6 +17,7 @@ Definition transf_function (f: RTL.function) : res BTL.function :=
let (tc, te) := tcte in
let f' := BTL.mkfunction (RTL.fn_sig f) (RTL.fn_params f) (RTL.fn_stacksize f) tc te in
do u <- verify_function dupmap f' f;
+ do u <- liveness_checker f';
OK f'.
Definition transf_fundef (f: RTL.fundef) : res fundef :=