src/HOL/HOLCF/IOA/CompoExecs.thy
changeset 67613 ce654b0e6d69
parent 63549 b0d31c7def86
--- a/src/HOL/HOLCF/IOA/CompoExecs.thy	Tue Feb 13 14:24:50 2018 +0100
+++ b/src/HOL/HOLCF/IOA/CompoExecs.thy	Thu Feb 15 12:11:00 2018 +0100
@@ -213,8 +213,8 @@
 
 theorem compositionality_ex:
   "ex \<in> executions (A \<parallel> B) \<longleftrightarrow>
-    Filter_ex (asig_of A) (ProjA ex) : executions A \<and>
-    Filter_ex (asig_of B) (ProjB ex) : executions B \<and>
+    Filter_ex (asig_of A) (ProjA ex) \<in> executions A \<and>
+    Filter_ex (asig_of B) (ProjB ex) \<in> executions B \<and>
     stutter (asig_of A) (ProjA ex) \<and>
     stutter (asig_of B) (ProjB ex) \<and>
     Forall (\<lambda>x. fst x \<in> act (A \<parallel> B)) (snd ex)"