src/HOL/Hoare_Parallel/OG_Hoare.thy
changeset 32960 69916a850301
parent 32621 a073cb249a06
child 35416 d8d7d1b785af
--- a/src/HOL/Hoare_Parallel/OG_Hoare.thy	Sat Oct 17 01:05:59 2009 +0200
+++ b/src/HOL/Hoare_Parallel/OG_Hoare.thy	Sat Oct 17 14:43:18 2009 +0200
@@ -57,7 +57,7 @@
 
 
 | Parallel: "\<lbrakk> \<forall>i<length Ts. \<exists>c q. Ts!i = (Some c, q) \<and> \<turnstile> c q; interfree Ts \<rbrakk>
-	   \<Longrightarrow> \<parallel>- (\<Inter>i\<in>{i. i<length Ts}. pre(the(com(Ts!i)))) 
+           \<Longrightarrow> \<parallel>- (\<Inter>i\<in>{i. i<length Ts}. pre(the(com(Ts!i)))) 
                      Parallel Ts 
                   (\<Inter>i\<in>{i. i<length Ts}. post(Ts!i))"
 
@@ -70,7 +70,7 @@
 | While:  "\<lbrakk> \<parallel>- (p \<inter> b) c p \<rbrakk> \<Longrightarrow> \<parallel>- p (While b i c) (p \<inter> -b)"
 
 | Conseq: "\<lbrakk> p' \<subseteq> p; \<parallel>- p c q ; q \<subseteq> q' \<rbrakk> \<Longrightarrow> \<parallel>- p' c q'"
-					    
+
 section {* Soundness *}
 (* In the version Isabelle-10-Sep-1999: HOL: The THEN and ELSE
 parts of conditional expressions (if P then x else y) are no longer