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/CleanupLabelstyping.v | 4 ++-- 1 file changed, 2 insertions(+), 2 deletions(-) (limited to 'backend/CleanupLabelstyping.v') diff --git a/backend/CleanupLabelstyping.v b/backend/CleanupLabelstyping.v index f58a910f..11b516fe 100644 --- a/backend/CleanupLabelstyping.v +++ b/backend/CleanupLabelstyping.v @@ -24,9 +24,9 @@ Require Import LTLintyping. Lemma in_remove_unused_labels: forall bto i c, In i (remove_unused_labels bto c) -> In i c. Proof. - induction c; simpl. + unfold remove_unused_labels, remove_unused. induction c; simpl. auto. - destruct a; simpl; intuition. + rewrite list_fold_right_eq. destruct a; simpl; intuition. destruct (Labelset.mem l bto); simpl in H; intuition. Qed. -- cgit