src/ZF/UNITY/AllocBase.thy
changeset 32960 69916a850301
parent 24893 b8ef7afe3a6b
child 41779 a68f503805ed
--- a/src/ZF/UNITY/AllocBase.thy	Sat Oct 17 01:05:59 2009 +0200
+++ b/src/ZF/UNITY/AllocBase.thy	Sat Oct 17 14:43:18 2009 +0200
@@ -1,8 +1,6 @@
 (*  Title:      ZF/UNITY/AllocBase.thy
-    ID:         $Id$
     Author:     Sidi O Ehmety, Cambridge University Computer Laboratory
     Copyright   2001  University of Cambridge
-
 *)
 
 header{*Common declarations for Chandy and Charpentier's Allocator*}
@@ -355,7 +353,7 @@
 
 lemma var_not_Finite: "~Finite(var)"
 apply (insert nat_not_Finite) 
-apply (blast intro: lepoll_Finite [OF 	nat_lepoll_var]) 
+apply (blast intro: lepoll_Finite [OF nat_lepoll_var]) 
 done
 
 lemma not_Finite_imp_exist: "~Finite(A) ==> \<exists>x. x\<in>A"