aboutsummaryrefslogtreecommitdiffstats
path: root/src/hls/RTLBlockgen.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/hls/RTLBlockgen.v')
-rw-r--r--src/hls/RTLBlockgen.v15
1 files changed, 4 insertions, 11 deletions
diff --git a/src/hls/RTLBlockgen.v b/src/hls/RTLBlockgen.v
index 05f9a32..6b3e9c3 100644
--- a/src/hls/RTLBlockgen.v
+++ b/src/hls/RTLBlockgen.v
@@ -24,16 +24,9 @@ From compcert Require Import
From vericert Require Import
RTLBlock.
-Parameter partition : RTL.code -> code.
+Parameter partition : RTL.function -> Errors.res function.
-Definition transl_function (f : RTL.function) : function :=
- mkfunction f.(RTL.fn_sig)
- f.(RTL.fn_params)
- f.(RTL.fn_stacksize)
- (partition f.(RTL.fn_code))
- f.(RTL.fn_entrypoint).
+Definition transl_fundef := transf_partial_fundef partition.
-Definition transl_fundef := transf_fundef transl_function.
-
-Definition transl_program : RTL.program -> program :=
- transform_program transl_fundef.
+Definition transl_program : RTL.program -> Errors.res program :=
+ transform_partial_program transl_fundef.