Journal/Paper.thy
changeset 175 170e59f2d645
parent 174 1b72810a2d61
child 176 675416b1defd
equal deleted inserted replaced
174:1b72810a2d61 175:170e59f2d645
  1775 
  1775 
  1776   \noindent With this in place we can conclude our theorem.\hfill\qed
  1776   \noindent With this in place we can conclude our theorem.\hfill\qed
  1777   \end{proof}
  1777   \end{proof}
  1778 
  1778 
  1779   \noindent This theorem is the main conclusion we obtain for the
  1779   \noindent This theorem is the main conclusion we obtain for the
  1780   Priority Inheritance Protocol: it shows that set of @{text blockers}
  1780   Priority Inheritance Protocol: it shows that the set of @{text blockers}
  1781   is fixed at state @{text s} when @{text th} becomes the thread with
  1781   is fixed at state @{text s} when @{text th} becomes the thread with
  1782   highest priority. Then no additional blocker of @{text th} can
  1782   highest priority. Then no additional blocker of @{text th} can
  1783   appear after the state @{text s}. And in this way we can bound the
  1783   appear after the state @{text s}. And in this way we can bound the
  1784   number of states where the thread @{text th} with the highest
  1784   number of states where the thread @{text th} with the highest
  1785   priority is prevented from running.
  1785   priority is prevented from running.