prio/PrioGDef.thy
changeset 295 8e4a5fff2eda
parent 294 bc5bf9e9ada2
child 298 f2e0d031a395
equal deleted inserted replaced
294:bc5bf9e9ada2 295:8e4a5fff2eda
   196 lemma 
   196 lemma 
   197   cpreced_def2:
   197   cpreced_def2:
   198   "cpreced wq s th \<equiv> Max ({preced th s} \<union> {preced th' s | th'. th' \<in> dependents wq th})"
   198   "cpreced wq s th \<equiv> Max ({preced th s} \<union> {preced th' s | th'. th' \<in> dependents wq th})"
   199   unfolding cpreced_def image_def
   199   unfolding cpreced_def image_def
   200   apply(rule eq_reflection)
   200   apply(rule eq_reflection)
   201   apply(rule arg_cong)
   201   apply(rule_tac f="Max" in arg_cong)
   202   back
       
   203   by (auto)
   202   by (auto)
   204 (*>*)
   203 (*>*)
   205 
   204 
   206 abbreviation
   205 abbreviation
   207   "all_unlocked \<equiv> \<lambda>_::cs. ([]::thread list)"
   206   "all_unlocked \<equiv> \<lambda>_::cs. ([]::thread list)"