aboutsummaryrefslogtreecommitdiffstats
path: root/src/hls/GibleSubPar.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/hls/GibleSubPar.v')
-rw-r--r--src/hls/GibleSubPar.v4
1 files changed, 1 insertions, 3 deletions
diff --git a/src/hls/GibleSubPar.v b/src/hls/GibleSubPar.v
index c867e1b..e69e71a 100644
--- a/src/hls/GibleSubPar.v
+++ b/src/hls/GibleSubPar.v
@@ -40,9 +40,7 @@ Module SubParBB <: BlockType.
Definition t := list (list instr).
Definition foldl (A: Type) (f: A -> instr -> A) (bb : t) (m : A): A :=
- fold_left
- (fun x l => fold_left f l x)
- bb m.
+ fold_left f (concat bb) m.
Definition length : t -> nat := @length (list instr).