src/HOL/UNITY/ProgressSets.thy
changeset 32960 69916a850301
parent 32693 6c6b1ba5e71e
child 35416 d8d7d1b785af
--- a/src/HOL/UNITY/ProgressSets.thy	Sat Oct 17 01:05:59 2009 +0200
+++ b/src/HOL/UNITY/ProgressSets.thy	Sat Oct 17 14:43:18 2009 +0200
@@ -1,4 +1,4 @@
-(*  Title:      HOL/UNITY/ProgressSets
+(*  Title:      HOL/UNITY/ProgressSets.thy
     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     Copyright   2003  University of Cambridge
 
@@ -23,7 +23,7 @@
   lattice :: "'a set set => bool"
    --{*Meier calls them closure sets, but they are just complete lattices*}
    "lattice L ==
-	 (\<forall>M. M \<subseteq> L --> \<Inter>M \<in> L) & (\<forall>M. M \<subseteq> L --> \<Union>M \<in> L)"
+         (\<forall>M. M \<subseteq> L --> \<Inter>M \<in> L) & (\<forall>M. M \<subseteq> L --> \<Union>M \<in> L)"
 
   cl :: "['a set set, 'a set] => 'a set"
    --{*short for ``closure''*}
@@ -197,14 +197,14 @@
               [OF _ lattice_awp_lemma [OF TXC BsubX latt TC BC clos, of r]
                     latt])
 apply (subgoal_tac
-	 "T \<inter> (B \<union> wp act X) \<inter> (T \<inter> (B \<union> awp F (X \<union> cl C (T\<inter>r)))) = 
-	  T \<inter> (B \<union> wp act X \<inter> awp F (X \<union> cl C (T\<inter>r)))") 
+         "T \<inter> (B \<union> wp act X) \<inter> (T \<inter> (B \<union> awp F (X \<union> cl C (T\<inter>r)))) = 
+          T \<inter> (B \<union> wp act X \<inter> awp F (X \<union> cl C (T\<inter>r)))") 
  prefer 2 apply blast 
 apply simp  
 apply (drule Un_in_lattice [OF _ TXC latt])  
 apply (subgoal_tac
-	 "T \<inter> (B \<union> wp act X \<inter> awp F (X \<union> cl C (T\<inter>r))) \<union> T\<inter>X = 
-	  T \<inter> (wp act X \<inter> awp F (X \<union> cl C (T\<inter>r)) \<union> X)")
+         "T \<inter> (B \<union> wp act X \<inter> awp F (X \<union> cl C (T\<inter>r))) \<union> T\<inter>X = 
+          T \<inter> (wp act X \<inter> awp F (X \<union> cl C (T\<inter>r)) \<union> X)")
  apply simp 
 apply (blast intro: BsubX [THEN subsetD]) 
 done
@@ -408,7 +408,7 @@
 constdefs
   decoupled :: "['a program, 'a program] => bool"
    "decoupled F G ==
-	\<forall>act \<in> Acts F. \<forall>B. G \<in> stable B --> G \<in> stable (wp act B)"
+        \<forall>act \<in> Acts F. \<forall>B. G \<in> stable B --> G \<in> stable (wp act B)"
 
 
 text{*Rao's Decoupling Theorem*}