summaryrefslogtreecommitdiff
path: root/backend/CleanupLabelstyping.v
diff options
context:
space:
mode:
authorGravatar xleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2013-03-16 16:51:42 +0000
committerGravatar xleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2013-03-16 16:51:42 +0000
commit707b6a1ae9660b13cf6f68c7c0ce74017f5981c5 (patch)
tree166a21d507612d60db40737333ddec5003fc81aa /backend/CleanupLabelstyping.v
parente44df4563f1cb893ab25b2a8b25d5b83095205be (diff)
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
Diffstat (limited to 'backend/CleanupLabelstyping.v')
-rw-r--r--backend/CleanupLabelstyping.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/backend/CleanupLabelstyping.v b/backend/CleanupLabelstyping.v
index f58a910..11b516f 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.