aboutsummaryrefslogtreecommitdiffstats
path: root/src/hls/GiblePargen.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/hls/GiblePargen.v')
-rw-r--r--src/hls/GiblePargen.v8
1 files changed, 4 insertions, 4 deletions
diff --git a/src/hls/GiblePargen.v b/src/hls/GiblePargen.v
index 0ca7ead..af09ee6 100644
--- a/src/hls/GiblePargen.v
+++ b/src/hls/GiblePargen.v
@@ -241,10 +241,10 @@ Definition is_initial_pred (f: forest) (p: positive) :=
| _ => None
end.
-Definition update (fop : option (pred_op * forest)) (i : instr): option (pred_op * forest) :=
- do (pred, f) <- fop;
+Definition update (fop : pred_op * forest) (i : instr): option (pred_op * forest) :=
+ let (pred, f) := fop in
match i with
- | RBnop => fop
+ | RBnop => Some fop
| RBop p op rl r =>
do pruned <-
prune_predicated
@@ -298,7 +298,7 @@ Get a sequence from the basic block.
|*)
Definition abstract_sequence (b : list instr) : option forest :=
- Option.map snd (fold_left update b (Some (Ptrue, empty))).
+ Option.map snd (mfold_left update b (Some (Ptrue, empty))).
(*|
Check equivalence of control flow instructions. As none of the basic blocks