aboutsummaryrefslogtreecommitdiffstats
path: root/mppa_k1c/Asmblock.v
diff options
context:
space:
mode:
authorCyril SIX <cyril.six@kalray.eu>2018-09-28 17:02:56 +0200
committerCyril SIX <cyril.six@kalray.eu>2018-09-28 17:02:56 +0200
commit3482cce97fd40de8f2c34eaaf642a54a9f453b83 (patch)
tree9bea7a870bf50621400218d7624467f0c2d06134 /mppa_k1c/Asmblock.v
parent27045947a8934d90e1d880ddc37b79c6537ff523 (diff)
downloadcompcert-kvx-3482cce97fd40de8f2c34eaaf642a54a9f453b83.tar.gz
compcert-kvx-3482cce97fd40de8f2c34eaaf642a54a9f453b83.zip
Removed the bundle attempt
Diffstat (limited to 'mppa_k1c/Asmblock.v')
-rw-r--r--mppa_k1c/Asmblock.v54
1 files changed, 7 insertions, 47 deletions
diff --git a/mppa_k1c/Asmblock.v b/mppa_k1c/Asmblock.v
index 6411dca5..51010c43 100644
--- a/mppa_k1c/Asmblock.v
+++ b/mppa_k1c/Asmblock.v
@@ -1087,15 +1087,15 @@ Inductive state: Type :=
* Perhaps there is a way to avoid that ?
*)
-Inductive stepin: option bblock -> state -> trace -> state -> Prop :=
- | exec_stepin_internal:
+Inductive step: state -> trace -> state -> Prop :=
+ | exec_step_internal:
forall b ofs f bi rs m rs' m',
rs PC = Vptr b ofs ->
Genv.find_funct_ptr ge b = Some (Internal f) ->
find_bblock (Ptrofs.unsigned ofs) (fn_blocks f) = Some bi ->
exec_bblock f bi rs m = Next rs' m' ->
- stepin (Some bi) (State rs m) E0 (State rs' m')
- | exec_stepin_builtin:
+ step (State rs m) E0 (State rs' m')
+ | exec_step_builtin:
forall b ofs f ef args res rs m vargs t vres rs' m' bi,
rs PC = Vptr b ofs ->
Genv.find_funct_ptr ge b = Some (Internal f) ->
@@ -1107,57 +1107,17 @@ Inductive stepin: option bblock -> state -> trace -> state -> Prop :=
(set_res res vres
(undef_regs (map preg_of (destroyed_by_builtin ef))
(rs#GPR31 <- Vundef))) ->
- stepin (Some bi) (State rs m) t (State rs' m')
- | exec_stepin_external:
+ step (State rs m) t (State rs' m')
+ | exec_step_external:
forall b ef args res rs m t rs' m',
rs PC = Vptr b Ptrofs.zero ->
Genv.find_funct_ptr ge b = Some (External ef) ->
external_call ef ge args m t res m' ->
extcall_arguments rs m (ef_sig ef) args ->
rs' = (set_pair (loc_external_result (ef_sig ef) ) res rs)#PC <- (rs RA) ->
- stepin None (State rs m) t (State rs' m')
- .
-
-Definition step (s:state) (t:trace) (s':state): Prop := exists obi, stepin obi s t s'.
-
-(* original constructors *)
-Lemma exec_step_internal b ofs f bi rs m rs' m':
- rs PC = Vptr b ofs ->
- Genv.find_funct_ptr ge b = Some (Internal f) ->
- find_bblock (Ptrofs.unsigned ofs) (fn_blocks f) = Some bi ->
- exec_bblock f bi rs m = Next rs' m' ->
- step (State rs m) E0 (State rs' m').
-Proof.
- intros; eexists. eapply exec_stepin_internal; eauto.
-Qed.
-
-Lemma exec_step_builtin b ofs f ef args res rs m vargs t vres rs' m' bi:
- rs PC = Vptr b ofs ->
- Genv.find_funct_ptr ge b = Some (Internal f) ->
- find_bblock (Ptrofs.unsigned ofs) f.(fn_blocks) = Some bi ->
- exit bi = Some (PExpand (Pbuiltin ef args res)) ->
- eval_builtin_args ge rs (rs SP) m args vargs ->
- external_call ef ge vargs m t vres m' ->
- rs' = nextblock bi
- (set_res res vres
- (undef_regs (map preg_of (destroyed_by_builtin ef))
- (rs#GPR31 <- Vundef))) ->
- step (State rs m) t (State rs' m').
-Proof.
- intros; eexists. eapply exec_stepin_builtin; eauto.
-Qed.
-
-Lemma exec_step_external b ef args res rs m t rs' m':
- rs PC = Vptr b Ptrofs.zero ->
- Genv.find_funct_ptr ge b = Some (External ef) ->
- external_call ef ge args m t res m' ->
- extcall_arguments rs m (ef_sig ef) args ->
- rs' = (set_pair (loc_external_result (ef_sig ef) ) res rs)#PC <- (rs RA) ->
step (State rs m) t (State rs' m')
.
-Proof.
- intros; eexists. eapply exec_stepin_external; eauto.
-Qed.
+
End RELSEM.