doc-src/TutorialI/Misc/AdvancedInd.thy
changeset 10242 028f54cd2cc9
parent 10241 e0428c2778f1
child 10281 9554ce1c2e54
--- a/doc-src/TutorialI/Misc/AdvancedInd.thy	Wed Oct 18 12:30:59 2000 +0200
+++ b/doc-src/TutorialI/Misc/AdvancedInd.thy	Wed Oct 18 17:19:18 2000 +0200
@@ -34,13 +34,14 @@
 \begin{isabelle}
 \ 1.\ xs\ {\isasymnoteq}\ []\ {\isasymLongrightarrow}\ hd\ []\ =\ last\ []
 \end{isabelle}
-We cannot prove this equality because we do not know what @{term"hd"} and
-@{term"last"} return when applied to @{term"[]"}.
+We cannot prove this equality because we do not know what @{term hd} and
+@{term last} return when applied to @{term"[]"}.
 
 The point is that we have violated the above warning. Because the induction
-formula is only the conclusion, the occurrence of @{term"xs"} in the premises is
+formula is only the conclusion, the occurrence of @{term xs} in the premises is
 not modified by induction. Thus the case that should have been trivial
-becomes unprovable. Fortunately, the solution is easy:
+becomes unprovable. Fortunately, the solution is easy:\footnote{A very similar
+heuristic applies to rule inductions; see \S\ref{sec:rtc}.}
 \begin{quote}
 \emph{Pull all occurrences of the induction variable into the conclusion
 using @{text"\<longrightarrow>"}.}