doc-src/TutorialI/Inductive/Advanced.thy
changeset 27167 a99747ccba87
parent 23842 9d87177f1f89
child 32891 d403b99287ff
--- a/doc-src/TutorialI/Inductive/Advanced.thy	Thu Jun 12 14:20:07 2008 +0200
+++ b/doc-src/TutorialI/Inductive/Advanced.thy	Thu Jun 12 14:20:25 2008 +0200
@@ -234,8 +234,8 @@
 apply (erule well_formed_gterm'.induct)
 (*>*)
 txt {*
-The proof script is identical, but the subgoal after applying induction may
-be surprising:
+The proof script is virtually identical,
+but the subgoal after applying induction may be surprising:
 @{subgoals[display,indent=0,margin=65]}
 The induction hypothesis contains an application of @{term lists}.  Using a
 monotone function in the inductive definition always has this effect.  The