diff -r 8ce9a432680b -r e6b13c7b9494 prio/PrioGDef.thy --- a/prio/PrioGDef.thy Mon Apr 23 08:01:37 2012 +0000 +++ b/prio/PrioGDef.thy Mon Apr 30 15:32:34 2012 +0000 @@ -361,7 +361,15 @@ @{text "th"} in state @{text "s"}. *} definition holdents :: "state \ thread \ cs set" - where "holdents s th \ {cs . (Cs cs, Th th) \ depend s}" + where "holdents s th \ {cs . holding s th cs}" + +lemma holdents_test: + "holdents s th = {cs . (Cs cs, Th th) \ depend s}" +unfolding holdents_def +unfolding s_depend_def +unfolding s_holding_abv +unfolding wq_def +by (simp) text {* \noindent @{text "cntCS s th"} returns the number of resources held by thread @{text "th"} in