src/ZF/UNITY/WFair.thy
changeset 32960 69916a850301
parent 24893 b8ef7afe3a6b
child 37936 1e4c5015a72e
--- a/src/ZF/UNITY/WFair.thy	Sat Oct 17 01:05:59 2009 +0200
+++ b/src/ZF/UNITY/WFair.thy	Sat Oct 17 14:43:18 2009 +0200
@@ -1,5 +1,4 @@
 (*  Title:      HOL/UNITY/WFair.thy
-    ID:         $Id$
     Author:     Sidi Ehmety, Computer Laboratory
     Copyright   1998  University of Cambridge
 *)
@@ -19,7 +18,7 @@
     is generic to all forms of fairness.*) 
   transient :: "i=>i"  where
   "transient(A) =={F:program. (EX act: Acts(F). A<=domain(act) &
-			       act``A <= state-A) & st_set(A)}"
+                               act``A <= state-A) & st_set(A)}"
 
 definition
   ensures :: "[i,i] => i"       (infixl "ensures" 60)  where
@@ -37,7 +36,7 @@
     Basis:  "[| F:A ensures B;  A:Pow(D); B:Pow(D) |] ==> <A,B>:leads(D, F)"
     Trans:  "[| <A,B> : leads(D, F); <B,C> : leads(D, F) |] ==>  <A,C>:leads(D, F)"
     Union:   "[| S:Pow({A:S. <A, B>:leads(D, F)}); B:Pow(D); S:Pow(Pow(D)) |] ==> 
-	      <Union(S),B>:leads(D, F)"
+              <Union(S),B>:leads(D, F)"
 
   monos        Pow_mono
   type_intros  Union_Pow_iff [THEN iffD2] UnionI PowI