diff -r 1bfdd19c1d47 -r ef006735bee8 doc-src/TutorialI/Misc/AdvancedInd.thy --- a/doc-src/TutorialI/Misc/AdvancedInd.thy Tue Nov 07 18:38:24 2000 +0100 +++ b/doc-src/TutorialI/Misc/AdvancedInd.thy Wed Nov 08 14:38:04 2000 +0100 @@ -51,23 +51,20 @@ (*<*)oops;(*>*) lemma hd_rev: "xs \ [] \ hd(rev xs) = last xs"; (*<*) -by(induct_tac xs, auto); +apply(induct_tac xs); (*>*) -text{*\noindent +txt{*\noindent This time, induction leaves us with the following base case -\begin{isabelle} -\ 1.\ []\ {\isasymnoteq}\ []\ {\isasymlongrightarrow}\ hd\ (rev\ [])\ =\ last\ [] -\end{isabelle} +@{subgoals[display,indent=0,goals_limit=1]} which is trivial, and @{text"auto"} finishes the whole proof. -If @{thm[source]hd_rev} is meant to be a simplification rule, you are +If @{text hd_rev} is meant to be a simplification rule, you are done. But if you really need the @{text"\"}-version of -@{thm[source]hd_rev}, for example because you want to apply it as an +@{text hd_rev}, for example because you want to apply it as an introduction rule, you need to derive it separately, by combining it with modus ponens: -*}; - +*}(*<*)by(auto);(*>*) lemmas hd_revI = hd_rev[THEN mp]; text{*\noindent