aboutsummaryrefslogtreecommitdiffstats
path: root/backend/CSE2.v
diff options
context:
space:
mode:
authorDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2020-01-27 20:27:20 +0100
committerDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2020-01-27 20:27:20 +0100
commit7dd2fce8926e3d9fa30ad2619dd38c5e2d535a5e (patch)
tree4f17ea2239dc4de3210d0060a2f992b978a7861e /backend/CSE2.v
parentbec3d3e29881590541130ef3f1116bd41df71a25 (diff)
downloadcompcert-kvx-7dd2fce8926e3d9fa30ad2619dd38c5e2d535a5e.tar.gz
compcert-kvx-7dd2fce8926e3d9fa30ad2619dd38c5e2d535a5e.zip
goes to the end but does not find available ops
Diffstat (limited to 'backend/CSE2.v')
-rw-r--r--backend/CSE2.v18
1 files changed, 5 insertions, 13 deletions
diff --git a/backend/CSE2.v b/backend/CSE2.v
index 36558033..d5412d73 100644
--- a/backend/CSE2.v
+++ b/backend/CSE2.v
@@ -621,23 +621,16 @@ Definition forward_map (f : RTL.function) := DS.fixpoint
(RTL.fn_code f) RTL.successors_instr
(apply_instr' (RTL.fn_code f)) (RTL.fn_entrypoint f) (Some RELATION.top).
-(*
-Definition get_r (rel : RELATION.t) (x : reg) :=
- match move_cases (PTree.get x rel) with
- | Move_case x' => x'
- | Other_case _ => x
- end.
-
-Definition get_rb (rb : RB.t) (x : reg) :=
+Definition forward_move_b (rb : RB.t) (x : reg) :=
match rb with
| None => x
- | Some rel => get_r rel x
+ | Some rel => forward_move rel x
end.
Definition subst_arg (fmap : option (PMap.t RB.t)) (pc : node) (x : reg) : reg :=
match fmap with
| None => x
- | Some inv => get_rb (PMap.get pc inv) x
+ | Some inv => forward_move_b (PMap.get pc inv) x
end.
Definition subst_args fmap pc := List.map (subst_arg fmap pc).
@@ -648,8 +641,8 @@ Definition transf_instr (fmap : option (PMap.t RB.t))
match instr with
| Iop op args dst s =>
Iop op (subst_args fmap pc args) dst s
- | Iload trap chunk addr args dst s =>
- Iload trap chunk addr (subst_args fmap pc args) dst s
+ | Iload chunk addr args dst s =>
+ Iload chunk addr (subst_args fmap pc args) dst s
| Istore chunk addr args src s =>
Istore chunk addr (subst_args fmap pc args) src s
| Icall sig ros args dst s =>
@@ -678,4 +671,3 @@ Definition transf_fundef (fd: fundef) : fundef :=
Definition transf_program (p: program) : program :=
transform_program transf_fundef p.
-*) \ No newline at end of file