src/HOL/UNITY/Comp/AllocBase.thy
changeset 32960 69916a850301
parent 24147 edc90be09ac1
child 35274 1cb90bbbf45e
--- a/src/HOL/UNITY/Comp/AllocBase.thy	Sat Oct 17 01:05:59 2009 +0200
+++ b/src/HOL/UNITY/Comp/AllocBase.thy	Sat Oct 17 14:43:18 2009 +0200
@@ -1,8 +1,6 @@
-(*  Title:      HOL/UNITY/AllocBase.thy
-    ID:         $Id$
+(*  Title:      HOL/UNITY/Comp/AllocBase.thy
     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     Copyright   1998  University of Cambridge
-
 *)
 
 header{*Common Declarations for Chandy and Charpentier's Allocator*}
@@ -87,7 +85,7 @@
      "bag_of (sublist l (A Un B)) + bag_of (sublist l (A Int B)) =  
       bag_of (sublist l A) + bag_of (sublist l B)"
 apply (subgoal_tac "A Int B Int {..<length l} =
-	            (A Int {..<length l}) Int (B Int {..<length l}) ")
+                    (A Int {..<length l}) Int (B Int {..<length l}) ")
 apply (simp add: bag_of_sublist Int_Un_distrib2 setsum_Un_Int, blast)
 done