src/HOL/UNITY/Simple/Deadlock.thy
changeset 32960 69916a850301
parent 26824 32e612e77edb
child 37936 1e4c5015a72e
--- a/src/HOL/UNITY/Simple/Deadlock.thy	Sat Oct 17 01:05:59 2009 +0200
+++ b/src/HOL/UNITY/Simple/Deadlock.thy	Sat Oct 17 14:43:18 2009 +0200
@@ -1,5 +1,4 @@
-(*  Title:      HOL/UNITY/Deadlock
-    ID:         $Id$
+(*  Title:      HOL/UNITY/Deadlock.thy
     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     Copyright   1998  University of Cambridge
 
@@ -63,7 +62,7 @@
 lemma
   assumes zeroprem: "F \<in> (A 0 \<inter> A (Suc n)) co (A 0)"
       and allprem:
-	    "!!i. i \<in> atMost n ==> F \<in> (A(Suc i) \<inter> A i) co (-A i \<union> A(Suc i))"
+            "!!i. i \<in> atMost n ==> F \<in> (A(Suc i) \<inter> A i) co (-A i \<union> A(Suc i))"
   shows "F \<in> stable (\<Inter>i \<in> atMost (Suc n). A i)"
 apply (unfold stable_def) 
 apply (rule constrains_Int [THEN constrains_weaken])