doc-src/TutorialI/Misc/AdvancedInd.thy
changeset 12492 a4dd02e744e0
parent 11494 23a118849801
child 12699 deae80045527
--- a/doc-src/TutorialI/Misc/AdvancedInd.thy	Thu Dec 13 17:57:55 2001 +0100
+++ b/doc-src/TutorialI/Misc/AdvancedInd.thy	Thu Dec 13 19:05:10 2001 +0100
@@ -70,18 +70,7 @@
 which can yield a fairly complex conclusion.  However, @{text rule_format} 
 can remove any number of occurrences of @{text"\<forall>"} and
 @{text"\<longrightarrow>"}.
-*}
 
-(*<*)
-by auto;
-(*>*)
-(*
-Here is a simple example (which is proved by @{text"blast"}):
-lemma simple[rule_format]:  "\<forall>y. A y \<longrightarrow> B y \<longrightarrow> B y \<and> A y";
-by blast;
-*)
-
-text{*
 \index{induction!on a term}%
 A second reason why your proposition may not be amenable to induction is that
 you want to induct on a complex term, rather than a variable. In
@@ -122,6 +111,7 @@
 single theorem because it depends on the number of free variables in $t$ ---
 the notation $\overline{y}$ is merely an informal device.
 *}
+(*<*)by auto(*>*)
 
 subsection{*Beyond Structural and Recursion Induction*};