aboutsummaryrefslogtreecommitdiffstats
path: root/mppa_k1c/ValueAOp.v
diff options
context:
space:
mode:
authorDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2019-04-04 19:54:25 +0200
committerDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2019-04-04 19:54:25 +0200
commit7a69f306599498055a1420b16058572e3cbb0fc7 (patch)
tree3b37c60d6ad8ec56a8043b191ca7618bcf2ea848 /mppa_k1c/ValueAOp.v
parent7171888446d3d4b47765cc21d982eb2045cd00cd (diff)
downloadcompcert-kvx-7a69f306599498055a1420b16058572e3cbb0fc7.tar.gz
compcert-kvx-7a69f306599498055a1420b16058572e3cbb0fc7.zip
select_sound
Diffstat (limited to 'mppa_k1c/ValueAOp.v')
-rw-r--r--mppa_k1c/ValueAOp.v15
1 files changed, 0 insertions, 15 deletions
diff --git a/mppa_k1c/ValueAOp.v b/mppa_k1c/ValueAOp.v
index af685a5e..e791cc40 100644
--- a/mppa_k1c/ValueAOp.v
+++ b/mppa_k1c/ValueAOp.v
@@ -56,21 +56,6 @@ Definition eval_static_select (cond : condition0) (v0 v1 vselect : aval) : aval
| _ => Vtop
end.
-Definition eval_select2 (cond : condition0) (v0 : val) (v1 : val) (vselect : val) (m: mem) : val :=
- match (eval_condition0 cond vselect m), v0, v1 with
- | Some bval, Vint i0, Vint i1 => Vint (if bval then i1 else i0)
- | _,_,_ => Vundef
- end.
-
-Lemma eval_select_to2: forall cond v0 v1 vselect m,
- (eval_select cond v0 v1 vselect m) =
- (eval_select2 cond v0 v1 vselect m).
-Proof.
- intros.
- unfold eval_select2.
- destruct v0; destruct v1; simpl; destruct (eval_condition0 cond vselect m); simpl; reflexivity.
-Qed.
-
Definition eval_static_selectl (v0 v1 vselect : aval) : aval :=
match vselect with
| I iselect =>