aboutsummaryrefslogtreecommitdiffstats
path: root/src/hls/RTLPargen.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/hls/RTLPargen.v')
-rw-r--r--src/hls/RTLPargen.v10
1 files changed, 9 insertions, 1 deletions
diff --git a/src/hls/RTLPargen.v b/src/hls/RTLPargen.v
index 8ff701f..39c57df 100644
--- a/src/hls/RTLPargen.v
+++ b/src/hls/RTLPargen.v
@@ -683,7 +683,15 @@ Definition transl_function (f: RTLBlock.function) : Errors.res RTLPar.function :
else
Errors.Error (Errors.msg "RTLPargen: Could not prove the blocks equivalent.").
-Definition transl_fundef := transf_partial_fundef transl_function.
+Definition transl_function_temp (f: RTLBlock.function) : Errors.res RTLPar.function :=
+ let tfcode := fn_code (schedule f) in
+ Errors.OK (mkfunction f.(fn_sig)
+ f.(fn_params)
+ f.(fn_stacksize)
+ tfcode
+ f.(fn_entrypoint)).
+
+Definition transl_fundef := transf_partial_fundef transl_function_temp.
Definition transl_program (p : RTLBlock.program) : Errors.res RTLPar.program :=
transform_partial_program transl_fundef p.