summaryrefslogtreecommitdiff
path: root/backend/Liveness.v
diff options
context:
space:
mode:
Diffstat (limited to 'backend/Liveness.v')
-rw-r--r--backend/Liveness.v3
1 files changed, 1 insertions, 2 deletions
diff --git a/backend/Liveness.v b/backend/Liveness.v
index b97455f..23faf41 100644
--- a/backend/Liveness.v
+++ b/backend/Liveness.v
@@ -110,7 +110,7 @@ Module RegsetLat := LFSet(Regset).
Module DS := Backward_Dataflow_Solver(RegsetLat)(NodeSetBackward).
Definition analyze (f: function): option (PMap.t Regset.t) :=
- DS.fixpoint (successors f) (transfer f) nil.
+ DS.fixpoint f.(fn_code) successors_instr (transfer f) nil.
(** Basic property of the liveness information computed by [analyze]. *)
@@ -122,7 +122,6 @@ Lemma analyze_solution:
Regset.Subset (transfer f s live!!s) live!!n.
Proof.
unfold analyze; intros. eapply DS.fixpoint_solution; eauto.
- unfold successors_list, successors. rewrite PTree.gmap1. rewrite H0. simpl. auto.
Qed.
(** Given an RTL function, compute (for every PC) the list of