src/HOL/UNITY/Comp/Alloc.thy
changeset 69313 b021008c5397
parent 67717 5a1b299fe4af
child 69325 4b6ddc5989fc
equal deleted inserted replaced
69312:e0f68a507683 69313:b021008c5397
   161 definition
   161 definition
   162   \<comment> \<open>environmental constraints\<close>
   162   \<comment> \<open>environmental constraints\<close>
   163   alloc_allowed_acts :: "'a allocState_d program set"
   163   alloc_allowed_acts :: "'a allocState_d program set"
   164   where "alloc_allowed_acts =
   164   where "alloc_allowed_acts =
   165        {F. AllowedActs F =
   165        {F. AllowedActs F =
   166             insert Id (UNION (preserves allocGiv) Acts)}"
   166             insert Id (\<Union>(Acts ` (preserves allocGiv)))}"
   167 
   167 
   168 definition
   168 definition
   169   alloc_spec :: "'a allocState_d program set"
   169   alloc_spec :: "'a allocState_d program set"
   170   where "alloc_spec = alloc_increasing Int alloc_safety Int alloc_progress Int
   170   where "alloc_spec = alloc_increasing Int alloc_safety Int alloc_progress Int
   171                    alloc_allowed_acts Int alloc_preserves"
   171                    alloc_allowed_acts Int alloc_preserves"