aboutsummaryrefslogtreecommitdiffstats
path: root/scheduling/RTLpathSE_impl.v
diff options
context:
space:
mode:
authorLéo Gourdin <leo.gourdin@univ-grenoble-alpes.fr>2021-02-23 18:10:29 +0100
committerLéo Gourdin <leo.gourdin@univ-grenoble-alpes.fr>2021-02-23 18:10:29 +0100
commit4192b5f46ff5dbe7a6ccc0929e2d339aaa0e7b71 (patch)
tree9ee80cf9ce0f3dc974f994d3aadb847f1636f302 /scheduling/RTLpathSE_impl.v
parent9cddf9110be0f088a62334e6eff74667110c5db8 (diff)
downloadcompcert-kvx-4192b5f46ff5dbe7a6ccc0929e2d339aaa0e7b71.tar.gz
compcert-kvx-4192b5f46ff5dbe7a6ccc0929e2d339aaa0e7b71.zip
Separate target_op_simplify for riscV
Diffstat (limited to 'scheduling/RTLpathSE_impl.v')
-rw-r--r--scheduling/RTLpathSE_impl.v21
1 files changed, 2 insertions, 19 deletions
diff --git a/scheduling/RTLpathSE_impl.v b/scheduling/RTLpathSE_impl.v
index bd7ae2ad..a7f1323d 100644
--- a/scheduling/RTLpathSE_impl.v
+++ b/scheduling/RTLpathSE_impl.v
@@ -6,7 +6,7 @@ Require Import Op Registers.
Require Import RTL RTLpath.
Require Import Errors.
Require Import RTLpathSE_theory RTLpathLivegenproof.
-Require Import Axioms RTLpathSE_simu_specs.
+Require Import Axioms RTLpathSE_simu_specs RTLpathSE_simplify.
Local Open Scope error_monad_scope.
Local Open Scope option_monad_scope.
@@ -695,23 +695,6 @@ Proof.
explore; try congruence.
Qed.
-
-(* TODO: This function could be defined in a specific file for each target *)
-Definition target_op_simplify (op: operation) (lr: list reg) (hst: hsistate_local): option hsval :=
- None. (* default implementation *)
-
-Lemma target_op_simplify_correct op lr hst fsv ge sp rs0 m0 st args m: forall
- (H: target_op_simplify op lr hst = Some fsv)
- (REF: hsilocal_refines ge sp rs0 m0 hst st)
- (OK0: hsok_local ge sp rs0 m0 hst)
- (OK1: seval_list_sval ge sp (list_sval_inj (map (si_sreg st) lr)) rs0 m0 = Some args)
- (OK2: seval_smem ge sp (si_smem st) rs0 m0 = Some m),
- seval_sval ge sp (hsval_proj fsv) rs0 m0 = eval_operation ge sp op args m.
-Proof.
- unfold target_op_simplify; simpl. congruence.
-Qed.
-Global Opaque target_op_simplify.
-
(** simplify a symbolic value before assignment to a register *)
Definition simplify (rsv: root_sval) (lr: list reg) (hst: hsistate_local): ?? hsval :=
match rsv with
@@ -1616,4 +1599,4 @@ Proof.
destruct (unsafe_coerce (aux_simu_check dm f tf)) as [[|]|] eqn:Hres; simpl; try discriminate.
intros; eapply aux_simu_check_correct; eauto.
eapply unsafe_coerce_not_really_correct; eauto.
-Qed. \ No newline at end of file
+Qed.