aboutsummaryrefslogtreecommitdiffstats
path: root/backend/RTLtyping.v
diff options
context:
space:
mode:
authorDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2019-09-02 18:30:25 +0200
committerDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2019-09-02 18:30:25 +0200
commit71c58a8d494eafd847776446b0c246229b2bc9cf (patch)
tree7570087588f24b3b340baeed5871b398bf7fc390 /backend/RTLtyping.v
parentdc8b24fa2dd7ede561dd75458899cf42e9be09d2 (diff)
downloadcompcert-kvx-71c58a8d494eafd847776446b0c246229b2bc9cf.tar.gz
compcert-kvx-71c58a8d494eafd847776446b0c246229b2bc9cf.zip
avancement (il faut utiliser Vundef visiblement)
Diffstat (limited to 'backend/RTLtyping.v')
-rw-r--r--backend/RTLtyping.v12
1 files changed, 6 insertions, 6 deletions
diff --git a/backend/RTLtyping.v b/backend/RTLtyping.v
index 8336d1bf..6d27df28 100644
--- a/backend/RTLtyping.v
+++ b/backend/RTLtyping.v
@@ -104,11 +104,11 @@ Inductive wt_instr : instruction -> Prop :=
valid_successor s ->
wt_instr (Iop op args res s)
| wt_Iload:
- forall chunk addr args dst s,
+ forall trap chunk addr args dst s,
map env args = type_of_addressing addr ->
env dst = type_of_chunk chunk ->
valid_successor s ->
- wt_instr (Iload chunk addr args dst s)
+ wt_instr (Iload trap chunk addr args dst s)
| wt_Istore:
forall chunk addr args src s,
map env args = type_of_addressing addr ->
@@ -282,7 +282,7 @@ Definition type_instr (e: S.typenv) (i: instruction) : res S.typenv :=
else
(let (targs, tres) := type_of_operation op in
do e1 <- S.set_list e args targs; S.set e1 res tres)
- | Iload chunk addr args dst s =>
+ | Iload trap chunk addr args dst s =>
do x <- check_successor s;
do e1 <- S.set_list e args (type_of_addressing addr);
S.set e1 dst (type_of_chunk chunk)
@@ -841,14 +841,14 @@ Proof.
Qed.
Lemma wt_exec_Iload:
- forall env f chunk addr args dst s m a v rs,
- wt_instr f env (Iload chunk addr args dst s) ->
+ forall env f trap chunk addr args dst s m a v rs,
+ wt_instr f env (Iload trap chunk addr args dst s) ->
Mem.loadv chunk m a = Some v ->
wt_regset env rs ->
wt_regset env (rs#dst <- v).
Proof.
intros. destruct a; simpl in H0; try discriminate. inv H.
- eapply wt_regset_assign; eauto. rewrite H8; eapply Mem.load_type; eauto.
+ eapply wt_regset_assign; eauto. rewrite H9; eapply Mem.load_type; eauto.
Qed.
Lemma wt_exec_Ibuiltin: