aboutsummaryrefslogtreecommitdiffstats
path: root/mppa_k1c/Op.v
diff options
context:
space:
mode:
authorDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2019-05-10 23:53:02 +0200
committerDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2019-05-10 23:53:02 +0200
commit295058286407ec6c4182f2b12b27608fc7d28f95 (patch)
tree9f5583cf990eb9aaee259e13b0737cce27948fe2 /mppa_k1c/Op.v
parente2ea45f5ba656254fa11bf3f355da67292c11f06 (diff)
downloadcompcert-kvx-295058286407ec6c4182f2b12b27608fc7d28f95.tar.gz
compcert-kvx-295058286407ec6c4182f2b12b27608fc7d28f95.zip
use shift 1-4 in backend
Diffstat (limited to 'mppa_k1c/Op.v')
-rw-r--r--mppa_k1c/Op.v14
1 files changed, 0 insertions, 14 deletions
diff --git a/mppa_k1c/Op.v b/mppa_k1c/Op.v
index b93a9fc3..4abd104e 100644
--- a/mppa_k1c/Op.v
+++ b/mppa_k1c/Op.v
@@ -66,20 +66,6 @@ Definition arg_type_of_condition0 (cond: condition0) :=
(** Arithmetic and logical operations. In the descriptions, [rd] is the
result of the operation and [r1], [r2], etc, are the arguments. *)
-Inductive shift1_4 : Type :=
-| SHIFT1 | SHIFT2 | SHIFT3 | SHIFT4.
-
-Definition z_of_shift1_4 (x : shift1_4) :=
- match x with
- | SHIFT1 => 1
- | SHIFT2 => 2
- | SHIFT3 => 3
- | SHIFT4 => 4
- end.
-
-Definition int_of_shift1_4 (x : shift1_4) :=
- Int.repr (z_of_shift1_4 x).
-
Inductive operation : Type :=
| Omove (**r [rd = r1] *)
| Ointconst (n: int) (**r [rd] is set to the given integer constant *)