aboutsummaryrefslogtreecommitdiffstats
path: root/src/hls/Pipeline.v
blob: ea0c32e9035af9f0ea3c705bd878a318c3896e98 (plain)
1
2
3
4
5
6
7
8
9
10
11
From compcert Require Import
     Maps
     AST
     RTL.

Parameter pipeline : function -> function.

Definition transf_fundef := transf_fundef pipeline.

Definition transf_program : program -> program :=
  transform_program transf_fundef.