# HG changeset patch # User Christian Urban # Date 1441794259 -3600 # Node ID fc83f79009bd019777566dc17e99655e4ba29253 # Parent f676a68935a05963eceab5d4ff5edd4066f716bb updated for Isabelle 2015 diff -r f676a68935a0 -r fc83f79009bd CpsG.thy --- a/CpsG.thy Tue Jul 15 17:25:53 2014 +0200 +++ b/CpsG.thy Wed Sep 09 11:24:19 2015 +0100 @@ -569,7 +569,7 @@ from tranclD[OF this] obtain z where "(Th th, z) \ RAG s'" by auto with rd_th show "False" - apply (case_tac z, auto simp:readys_def s_waiting_def s_RAG_def s_waiting_def cs_waiting_def) + apply (case_tac z, auto simp:readys_def s_RAG_def s_waiting_def cs_waiting_def) by (fold wq_def, blast) qed diff -r f676a68935a0 -r fc83f79009bd Journal/Paper.thy --- a/Journal/Paper.thy Tue Jul 15 17:25:53 2014 +0200 +++ b/Journal/Paper.thy Wed Sep 09 11:24:19 2015 +0100 @@ -1157,9 +1157,9 @@ a standard scheduling operation implemented in most operating systems. - \begin{proof}[of Lemma~\ref{childrenlem}] - Test - \end{proof} + %\begin{proof}[of Lemma~\ref{childrenlem}] + %Test + %\end{proof} Of course the main work for implementing PIP involves the scheduler and coding how it should react to events. Below we diff -r f676a68935a0 -r fc83f79009bd README --- a/README Tue Jul 15 17:25:53 2014 +0200 +++ b/README Wed Sep 09 11:24:19 2015 +0100 @@ -12,7 +12,7 @@ The repository can be checked using Isabelle 2013-2. - isabelle build -d . PIP + isabelle build -c -v -d . PIP Othe directories are: diff -r f676a68935a0 -r fc83f79009bd ROOT --- a/ROOT Tue Jul 15 17:25:53 2014 +0200 +++ b/ROOT Wed Sep 09 11:24:19 2015 +0100 @@ -2,7 +2,7 @@ theories [document = false] "CpsG" "ExtGG" - (* "Test" *) + "Test" session "Slides2" in "Slides" = PIP + options [document_variants="slides2"] diff -r f676a68935a0 -r fc83f79009bd Test.thy --- a/Test.thy Tue Jul 15 17:25:53 2014 +0200 +++ b/Test.thy Wed Sep 09 11:24:19 2015 +0100 @@ -749,10 +749,6 @@ - -done - - (* obtain th0 where th0_in: "th0 \ S1 \ th0 \ S2" and eq_f_th0: "preced th0 s = Max ((\th. preced th s) ` (S1 \ S2))" @@ -784,4 +780,6 @@ qed *) +thm waits_def waits2_def + end \ No newline at end of file diff -r f676a68935a0 -r fc83f79009bd journal.pdf Binary file journal.pdf has changed