aboutsummaryrefslogtreecommitdiffstats
path: root/backend/ForwardMoves.v
diff options
context:
space:
mode:
authorDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2020-01-09 08:02:36 +0100
committerDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2020-01-09 08:02:36 +0100
commita36948c2af873559e5df4a2d96fdbc5bbfcfaca8 (patch)
tree29f34dce4fde3af7073c6090fbc59faac24f1bdf /backend/ForwardMoves.v
parent5787da9e4d024dc3a3190bff0fe29385abbcece9 (diff)
downloadcompcert-kvx-a36948c2af873559e5df4a2d96fdbc5bbfcfaca8.tar.gz
compcert-kvx-a36948c2af873559e5df4a2d96fdbc5bbfcfaca8.zip
fix bug and forward in proofs
Diffstat (limited to 'backend/ForwardMoves.v')
-rw-r--r--backend/ForwardMoves.v3
1 files changed, 2 insertions, 1 deletions
diff --git a/backend/ForwardMoves.v b/backend/ForwardMoves.v
index 0e71b6b5..660d0458 100644
--- a/backend/ForwardMoves.v
+++ b/backend/ForwardMoves.v
@@ -250,13 +250,14 @@ Fixpoint kill_builtin_res (res : builtin_res reg) (rel : RELATION.t) :=
Definition apply_instr instr x :=
match instr with
| Inop _
+ | Icond _ _ _ _
| Istore _ _ _ _ _ => Some x
| Iop Omove (src :: nil) dst _ => Some (move src dst x)
| Iop _ _ dst _
| Iload _ _ _ _ dst _
| Icall _ _ _ dst _ => Some (kill dst x)
| Ibuiltin _ _ res _ => Some (kill_builtin_res res x)
- | Icond _ _ _ _ | Itailcall _ _ _ | Ijumptable _ _ | Ireturn _ => RB.bot
+ | Itailcall _ _ _ | Ijumptable _ _ | Ireturn _ => RB.bot
end.
Definition apply_instr' code (pc : node) (ro : RB.t) : RB.t :=