aboutsummaryrefslogtreecommitdiffstats
path: root/mppa_k1c/Peephole.v
diff options
context:
space:
mode:
authorDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2019-05-03 10:34:58 +0200
committerDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2019-05-03 10:34:58 +0200
commite1c864b670812eda55e0ee129855c69d32c8b84a (patch)
tree5e3154b90159293c2130e3615aa5fabed92e0fca /mppa_k1c/Peephole.v
parent676d1ae6324d3c2f13e20efdcff3fbda9aab1686 (diff)
downloadcompcert-kvx-e1c864b670812eda55e0ee129855c69d32c8b84a.tar.gz
compcert-kvx-e1c864b670812eda55e0ee129855c69d32c8b84a.zip
it compiles
Diffstat (limited to 'mppa_k1c/Peephole.v')
-rw-r--r--mppa_k1c/Peephole.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/mppa_k1c/Peephole.v b/mppa_k1c/Peephole.v
index 2c73bb63..91936ac6 100644
--- a/mppa_k1c/Peephole.v
+++ b/mppa_k1c/Peephole.v
@@ -34,8 +34,8 @@ Fixpoint optimize_body (insns : list basic) : list basic :=
match t0 with
| h1 :: t1 =>
match h0, h1 with
- | (PStoreRRO Psd_a rs0 ra0 (Ofsimm ofs0)),
- (PStoreRRO Psd_a rs1 ra1 (Ofsimm ofs1)) =>
+ | (PStoreRRO Psd_a rs0 ra0 ofs0),
+ (PStoreRRO Psd_a rs1 ra1 ofs1) =>
match gpreg_q_search rs0 rs1 with
| Some rs0rs1 =>
let zofs0 := Ptrofs.signed ofs0 in