Journal/Paper.thy
changeset 45 fc83f79009bd
parent 44 f676a68935a0
child 46 331137d43625
equal deleted inserted replaced
44:f676a68935a0 45:fc83f79009bd
  1155   precedence is computed in this more efficient manner, the selection
  1155   precedence is computed in this more efficient manner, the selection
  1156   of the thread with highest precedence from a set of ready threads is
  1156   of the thread with highest precedence from a set of ready threads is
  1157   a standard scheduling operation implemented in most operating
  1157   a standard scheduling operation implemented in most operating
  1158   systems.
  1158   systems.
  1159 
  1159 
  1160   \begin{proof}[of Lemma~\ref{childrenlem}]
  1160   %\begin{proof}[of Lemma~\ref{childrenlem}]
  1161   Test
  1161   %Test
  1162   \end{proof}
  1162   %\end{proof}
  1163 
  1163 
  1164   Of course the main work for implementing PIP involves the
  1164   Of course the main work for implementing PIP involves the
  1165   scheduler and coding how it should react to events.  Below we
  1165   scheduler and coding how it should react to events.  Below we
  1166   outline how our formalisation guides this implementation for each
  1166   outline how our formalisation guides this implementation for each
  1167   kind of events.\smallskip
  1167   kind of events.\smallskip