doc-src/TutorialI/Misc/Itrev.thy
changeset 9644 6b0b6b471855
parent 9541 d17c0b34d5c8
child 9689 751fde5307e4
--- a/doc-src/TutorialI/Misc/Itrev.thy	Thu Aug 17 21:07:25 2000 +0200
+++ b/doc-src/TutorialI/Misc/Itrev.thy	Fri Aug 18 10:34:08 2000 +0200
@@ -84,6 +84,13 @@
 provability of the goal. Because it is not always required, and may even
 complicate matters in some cases, this heuristic is often not
 applied blindly.
+
+In general, if you have tried the above heuristics and still find your
+induction does not go through, and no obvious lemma suggests itself, you may
+need to generalize your proposition even further. This requires insight into
+the problem at hand and is beyond simple rules of thumb. In a nutshell: you
+will need to be creative. Additionally, you can read \S\ref{sec:advanced-ind}
+to learn about some advanced techniques for inductive proofs.
 *};
 
 (*<*)