aboutsummaryrefslogtreecommitdiffstats
path: root/kvx/Peephole.v
diff options
context:
space:
mode:
Diffstat (limited to 'kvx/Peephole.v')
-rw-r--r--kvx/Peephole.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/kvx/Peephole.v b/kvx/Peephole.v
index 35f4bbd9..5adb823b 100644
--- a/kvx/Peephole.v
+++ b/kvx/Peephole.v
@@ -153,6 +153,6 @@ Program Definition optimize_bblock (bb : bblock) :=
exit := exit bb |}.
Next Obligation.
destruct (wf_bblockb (optimize_body (body bb))) eqn:Rwf.
- - rewrite Rwf. simpl. trivial.
+ - rewrite Rwf. cbn. trivial.
- exact (correct bb).
Qed.