# HG changeset patch # User nipkow # Date 975339656 -3600 # Node ID 270b285d48ee48f3c9d921355f222530fb880cc6 # Parent 68105cf615fa7eeaac80a7ce9ffc3510688e27a3 *** empty log message *** diff -r 68105cf615fa -r 270b285d48ee doc-src/TutorialI/CTL/PDL.thy --- a/doc-src/TutorialI/CTL/PDL.thy Mon Nov 27 11:06:28 2000 +0100 +++ b/doc-src/TutorialI/CTL/PDL.thy Mon Nov 27 16:40:56 2000 +0100 @@ -96,7 +96,7 @@ apply(rule equalityI); apply(rule subsetI); - apply(simp) + apply(simp)(*<*)apply(rename_tac s)(*>*) txt{*\noindent Simplification leaves us with the following first subgoal diff -r 68105cf615fa -r 270b285d48ee doc-src/TutorialI/CTL/document/PDL.tex --- a/doc-src/TutorialI/CTL/document/PDL.tex Mon Nov 27 11:06:28 2000 +0100 +++ b/doc-src/TutorialI/CTL/document/PDL.tex Mon Nov 27 16:40:56 2000 +0100 @@ -98,7 +98,7 @@ \noindent Simplification leaves us with the following first subgoal \begin{isabelle}% -\ {\isadigit{1}}{\isachardot}\ {\isasymAnd}x{\isachardot}\ x\ {\isasymin}\ lfp\ {\isacharparenleft}{\isasymlambda}T{\isachardot}\ A\ {\isasymunion}\ M{\isasyminverse}\ {\isacharcircum}{\isacharcircum}\ T{\isacharparenright}\ {\isasymLongrightarrow}\ {\isasymexists}t{\isachardot}\ {\isacharparenleft}x{\isacharcomma}\ t{\isacharparenright}\ {\isasymin}\ M\isactrlsup {\isacharasterisk}\ {\isasymand}\ t\ {\isasymin}\ A% +\ {\isadigit{1}}{\isachardot}\ {\isasymAnd}s{\isachardot}\ s\ {\isasymin}\ lfp\ {\isacharparenleft}{\isasymlambda}T{\isachardot}\ A\ {\isasymunion}\ M{\isasyminverse}\ {\isacharcircum}{\isacharcircum}\ T{\isacharparenright}\ {\isasymLongrightarrow}\ {\isasymexists}t{\isachardot}\ {\isacharparenleft}s{\isacharcomma}\ t{\isacharparenright}\ {\isasymin}\ M\isactrlsup {\isacharasterisk}\ {\isasymand}\ t\ {\isasymin}\ A% \end{isabelle} which is proved by \isa{lfp}-induction:% \end{isamarkuptxt}% diff -r 68105cf615fa -r 270b285d48ee doc-src/TutorialI/proof.sty --- a/doc-src/TutorialI/proof.sty Mon Nov 27 11:06:28 2000 +0100 +++ /dev/null Thu Jan 01 00:00:00 1970 +0000 @@ -1,272 +0,0 @@ -\ProvidesPackage{proof}[1995/05/22] -% proof.sty (Proof Figure Macros) -% -% version 2.0 -% June 24, 1991 -% Copyright (C) 1990,1991 Makoto Tatsuta (tatsuta@riec.tohoku.ac.jp) -% -%Modified for LaTeX-2e by L. C. Paulson -% -% This program is free software; you can redistribute it or modify -% it under the terms of the GNU General Public License as published by -% the Free Software Foundation; either versions 1, or (at your option) -% any later version. -% -% This program is distributed in the hope that it will be useful -% but WITHOUT ANY WARRANTY; without even the implied warranty of -% MERCHANTABILITY or FITNESS FOR A PARTICULAR PURPOSE. See the -% GNU General Public License for more details. -% -% Usage: -% In \documentstyle, specify an optional style `proof', say, -% \documentstyle[proof]{article}. -% -% The following macros are available: -% -% In all the following macros, all the arguments such as -% and are processed in math mode. -% -% \infer -% draws an inference. -% -% Use & in to delimit upper formulae. -% consists more than 0 formulae. -% -% \infer returns \hbox{ ... } or \vbox{ ... } and -% sets \@LeftOffset and \@RightOffset globally. -% -% \infer[