aboutsummaryrefslogtreecommitdiffstats
path: root/scheduling/BTLtoRTL.v
diff options
context:
space:
mode:
authorSylvain Boulmé <sylvain.boulme@univ-grenoble-alpes.fr>2021-05-28 14:28:56 +0200
committerSylvain Boulmé <sylvain.boulme@univ-grenoble-alpes.fr>2021-05-28 14:28:56 +0200
commit25595a7b34b70011dcb77aae277ee1cdb8920c60 (patch)
tree6b8269b22eca57b51986593f8646f652d8598e09 /scheduling/BTLtoRTL.v
parent8752cea89f862d92d49183fe10d1918588143ab1 (diff)
downloadcompcert-kvx-25595a7b34b70011dcb77aae277ee1cdb8920c60.tar.gz
compcert-kvx-25595a7b34b70011dcb77aae277ee1cdb8920c60.zip
splitting BTL by introducing BTLmatchRTL
reduce also copy-paste between BTLtoRTLproof and RTLtoBTLproof sharing is done in BTLmatchRTL
Diffstat (limited to 'scheduling/BTLtoRTL.v')
-rw-r--r--scheduling/BTLtoRTL.v7
1 files changed, 4 insertions, 3 deletions
diff --git a/scheduling/BTLtoRTL.v b/scheduling/BTLtoRTL.v
index 1333b406..fc58533d 100644
--- a/scheduling/BTLtoRTL.v
+++ b/scheduling/BTLtoRTL.v
@@ -1,21 +1,22 @@
Require Import Coqlib Maps.
Require Import AST Integers Values Events Memory Globalenvs Smallstep.
Require Import RTL Op Registers OptionMonad BTL.
+Require Export BTLmatchRTL.
Require Import Errors Linking.
(** External oracle *)
-Axiom btl2rtl: function -> RTL.code * node * (PTree.t node).
+Axiom btl2rtl: BTL.function -> RTL.code * node * (PTree.t node).
Extract Constant btl2rtl => "BTLtoRTLaux.btl2rtl".
Local Open Scope error_monad_scope.
-Definition transf_function (f: function) : res RTL.function :=
+Definition transf_function (f: BTL.function) : res RTL.function :=
let (tcte, dupmap) := btl2rtl f in
let (tc, te) := tcte in
let f' := RTL.mkfunction (fn_sig f) (fn_params f) (fn_stacksize f) tc te in
- (*do u <- verify_function dupmap f f';*)
+ do u <- verify_function dupmap f f';
OK f'.
Definition transf_fundef (f: fundef) : res RTL.fundef :=