src/HOL/UNITY/Comp/AllocImpl.thy
changeset 69313 b021008c5397
parent 65956 639eb3617a86
child 69325 4b6ddc5989fc
--- a/src/HOL/UNITY/Comp/AllocImpl.thy	Sun Nov 18 09:51:41 2018 +0100
+++ b/src/HOL/UNITY/Comp/AllocImpl.thy	Sun Nov 18 18:07:51 2018 +0000
@@ -116,7 +116,7 @@
 definition
   distr_allowed_acts :: "('a,'b) distr_d program set"
   where "distr_allowed_acts =
-       {D. AllowedActs D = insert Id (UNION (preserves distr.Out) Acts)}"
+       {D. AllowedActs D = insert Id (\<Union>(Acts ` (preserves distr.Out)))}"
 
 definition
   distr_spec :: "('a,'b) distr_d program set"
@@ -160,7 +160,7 @@
   (*environmental constraints*)
   alloc_allowed_acts :: "'a allocState_d program set"
   where "alloc_allowed_acts =
-       {F. AllowedActs F = insert Id (UNION (preserves giv) Acts)}"
+       {F. AllowedActs F = insert Id (\<Union>(Acts ` (preserves giv)))}"
 
 definition
   alloc_spec :: "'a allocState_d program set"