src/HOL/Hoare_Parallel/OG_Tran.thy
changeset 52141 eff000cab70f
parent 46362 b2878f059f91
child 58884 be4d203d35b3
--- a/src/HOL/Hoare_Parallel/OG_Tran.thy	Sat May 25 15:44:08 2013 +0200
+++ b/src/HOL/Hoare_Parallel/OG_Tran.thy	Sat May 25 15:44:29 2013 +0200
@@ -90,13 +90,13 @@
   "ann_sem c \<equiv> \<lambda>s. {t. (Some c, s) -*\<rightarrow> (None, t)}"
 
 definition ann_SEM :: "'a ann_com \<Rightarrow> 'a set \<Rightarrow> 'a set" where
-  "ann_SEM c S \<equiv> \<Union>ann_sem c ` S"  
+  "ann_SEM c S \<equiv> \<Union>(ann_sem c ` S)"
 
 definition sem :: "'a com \<Rightarrow> 'a \<Rightarrow> 'a set" where
   "sem c \<equiv> \<lambda>s. {t. \<exists>Ts. (c, s) -P*\<rightarrow> (Parallel Ts, t) \<and> All_None Ts}"
 
 definition SEM :: "'a com \<Rightarrow> 'a set \<Rightarrow> 'a set" where
-  "SEM c S \<equiv> \<Union>sem c ` S "
+  "SEM c S \<equiv> \<Union>(sem c ` S)"
 
 abbreviation Omega :: "'a com"    ("\<Omega>" 63)
   where "\<Omega> \<equiv> While UNIV UNIV (Basic id)"