From 707b6a1ae9660b13cf6f68c7c0ce74017f5981c5 Mon Sep 17 00:00:00 2001 From: xleroy Date: Sat, 16 Mar 2013 16:51:42 +0000 Subject: Assorted changes to reduce stack and heap requirements when compiling very big functions. git-svn-id: https://yquem.inria.fr/compcert/svn/compcert/trunk@2151 fca1b0fc-160b-0410-b1d3-a4f43f01ea2e --- backend/Allocproof.v | 10 +++++----- 1 file changed, 5 insertions(+), 5 deletions(-) (limited to 'backend/Allocproof.v') diff --git a/backend/Allocproof.v b/backend/Allocproof.v index 2011485..8dfa2d4 100644 --- a/backend/Allocproof.v +++ b/backend/Allocproof.v @@ -28,7 +28,9 @@ Require Import Op. Require Import Registers. Require Import RTL. Require Import RTLtyping. +Require Import Liveness. Require Import Locations. +Require Import LTL. Require Import Conventions. Require Import Coloring. Require Import Coloringproof. @@ -42,7 +44,7 @@ Require Import Allocation. Section REGALLOC_PROPERTIES. -Variable f: function. +Variable f: RTL.function. Variable env: regenv. Variable live: PMap.t Regset.t. Variable alloc: reg -> loc. @@ -145,7 +147,7 @@ Definition agree (live: Regset.t) (rs: regset) (ls: locset) : Prop := Lemma agree_increasing: forall live1 live2 rs ls, - RegsetLat.ge live1 live2 -> agree live1 rs ls -> + Regset.Subset live2 live1 -> agree live1 rs ls -> agree live2 rs ls. Proof. unfold agree; intros. @@ -162,9 +164,7 @@ Lemma agree_succ: Proof. intros. apply agree_increasing with (live!!n). - eapply DS.fixpoint_solution. unfold analyze in H; eauto. - unfold RTL.successors, Kildall.successors_list. - rewrite PTree.gmap1. rewrite H0. simpl. auto. + eapply Liveness.analyze_solution; eauto. auto. Qed. -- cgit v1.2.3