aboutsummaryrefslogtreecommitdiffstats
path: root/powerpc/Op.v
diff options
context:
space:
mode:
authorBernhard Schommer <bernhardschommer@gmail.com>2015-04-02 16:25:25 +0200
committerBernhard Schommer <bernhardschommer@gmail.com>2015-04-02 16:25:25 +0200
commit170284b51766112e29d6bbfe519bad9f6da95269 (patch)
tree13a163ccee48cee0512a8af484b394623cdce030 /powerpc/Op.v
parent2e30ad9698a6f24a8a746f68b30c235913006392 (diff)
parent959432fa13a899290db5236f93575a8bfdc13bb5 (diff)
downloadcompcert-kvx-170284b51766112e29d6bbfe519bad9f6da95269.tar.gz
compcert-kvx-170284b51766112e29d6bbfe519bad9f6da95269.zip
Merge branch 'master' into dwarf
Diffstat (limited to 'powerpc/Op.v')
-rw-r--r--powerpc/Op.v5
1 files changed, 3 insertions, 2 deletions
diff --git a/powerpc/Op.v b/powerpc/Op.v
index 3d5b1fc5..4c1168cd 100644
--- a/powerpc/Op.v
+++ b/powerpc/Op.v
@@ -569,6 +569,7 @@ Definition is_trivial_op (op: operation) : bool :=
Definition op_depends_on_memory (op: operation) : bool :=
match op with
| Ocmp (Ccompu _) => true
+ | Ocmp (Ccompuimm _ _) => true
| _ => false
end.
@@ -577,8 +578,8 @@ Lemma op_depends_on_memory_correct:
op_depends_on_memory op = false ->
eval_operation ge sp op args m1 = eval_operation ge sp op args m2.
Proof.
- intros until m2. destruct op; simpl; try congruence.
- destruct c; simpl; auto; discriminate.
+ intros until m2. destruct op; simpl; try congruence. unfold eval_condition.
+ destruct c; simpl; auto; try discriminate.
Qed.
(** Global variables mentioned in an operation or addressing mode *)