From eafbaf41e528cc9825a503c66739a66a92ca65a8 Mon Sep 17 00:00:00 2001 From: xleroy Date: Mon, 12 Aug 2013 13:09:20 +0000 Subject: Change interface of Kildall solvers to avoid precomputing the map pc -> list of successors. git-svn-id: https://yquem.inria.fr/compcert/svn/compcert/trunk@2305 fca1b0fc-160b-0410-b1d3-a4f43f01ea2e --- backend/Liveness.v | 3 +-- 1 file changed, 1 insertion(+), 2 deletions(-) (limited to 'backend/Liveness.v') diff --git a/backend/Liveness.v b/backend/Liveness.v index b97455fc..23faf41c 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 -- cgit