aboutsummaryrefslogtreecommitdiffstats
path: root/mppa_k1c/Asmvliw.v
diff options
context:
space:
mode:
authorDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2019-05-03 09:25:48 +0200
committerDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2019-05-03 09:25:48 +0200
commit92b48e2aa6d24d1ad487c1d2a3644a57966c765e (patch)
tree9ae13a1917a968992338a81a9a4a9fbb62df3222 /mppa_k1c/Asmvliw.v
parentc56f9a47fe1837b7afb73c2c24aed9228bc0db08 (diff)
downloadcompcert-kvx-92b48e2aa6d24d1ad487c1d2a3644a57966c765e.tar.gz
compcert-kvx-92b48e2aa6d24d1ad487c1d2a3644a57966c765e.zip
rm Ofslow (résidu du Risc-V, inutilisé et complique les preuves)
Diffstat (limited to 'mppa_k1c/Asmvliw.v')
-rw-r--r--mppa_k1c/Asmvliw.v14
1 files changed, 2 insertions, 12 deletions
diff --git a/mppa_k1c/Asmvliw.v b/mppa_k1c/Asmvliw.v
index e460727c..c25d4235 100644
--- a/mppa_k1c/Asmvliw.v
+++ b/mppa_k1c/Asmvliw.v
@@ -152,9 +152,7 @@ Inductive ftest: Type :=
(** Offsets for load and store instructions. An offset is either an
immediate integer or the low part of a symbol. *)
-Inductive offset : Type :=
- | Ofsimm (ofs: ptrofs)
- | Ofslow (id: ident) (ofs: ptrofs).
+Definition offset : Type := ptrofs.
(** We model a subset of the K1c instruction set. In particular, we do not
support floats yet.
@@ -1093,15 +1091,7 @@ Definition parexec_arith_instr (ai: ar_instruction) (rsr rsw: regset): regset :=
| PArithARRI64 n d s i => rsw#d <- (arith_eval_arri64 n rsr#d rsr#s i)
end.
-Definition eval_offset (ofs: offset) : res ptrofs :=
- match ofs with
- | Ofsimm n => OK n
- | Ofslow id delta =>
- match (Genv.symbol_address ge id delta) with
- | Vptr b ofs => OK ofs
- | _ => Error (msg "Asmblock.eval_offset")
- end
- end.
+Definition eval_offset (ofs: offset) : res ptrofs := OK ofs.
(** * load/store *)