equal
deleted
inserted
replaced
36 cp ("cprec") and |
36 cp ("cprec") and |
37 holdents ("resources") and |
37 holdents ("resources") and |
38 original_priority ("priority") and |
38 original_priority ("priority") and |
39 DUMMY ("\<^raw:\mbox{$\_\!\_$}>") |
39 DUMMY ("\<^raw:\mbox{$\_\!\_$}>") |
40 |
40 |
41 abbreviation |
41 (*abbreviation |
42 "detached s th \<equiv> cntP s th = cntV s th" |
42 "detached s th \<equiv> cntP s th = cntV s th" |
|
43 *) |
43 (*>*) |
44 (*>*) |
44 |
45 |
45 section {* Introduction *} |
46 section {* Introduction *} |
46 |
47 |
47 text {* |
48 text {* |
373 we must ensure that the resulting RAG is not circular. In practice, the |
374 we must ensure that the resulting RAG is not circular. In practice, the |
374 programmer has to ensure this. |
375 programmer has to ensure this. |
375 |
376 |
376 |
377 |
377 {\bf ??? define detached} |
378 {\bf ??? define detached} |
|
379 \begin{isabelle}\ \ \ \ \ %%% |
|
380 @{thm detached_def} |
|
381 \end{isabelle} |
|
382 |
378 |
383 |
379 |
384 |
380 Next we introduce the notion of the \emph{current precedence} of a thread @{text th} in a |
385 Next we introduce the notion of the \emph{current precedence} of a thread @{text th} in a |
381 state @{text s}. It is defined as |
386 state @{text s}. It is defined as |
382 |
387 |