doc-src/TutorialI/Inductive/Star.thy
changeset 32891 d403b99287ff
parent 27172 8236f13be95b
--- a/doc-src/TutorialI/Inductive/Star.thy	Wed Oct 07 16:57:56 2009 +0200
+++ b/doc-src/TutorialI/Inductive/Star.thy	Thu Oct 08 15:16:13 2009 +0200
@@ -54,7 +54,7 @@
 To prove transitivity, we need rule induction, i.e.\ theorem
 @{thm[source]rtc.induct}:
 @{thm[display]rtc.induct}
-It says that @{text"?P"} holds for an arbitrary pair @{thm_style prem1 rtc.induct}
+It says that @{text"?P"} holds for an arbitrary pair @{thm (prem 1) rtc.induct}
 if @{text"?P"} is preserved by all rules of the inductive definition,
 i.e.\ if @{text"?P"} holds for the conclusion provided it holds for the
 premises. In general, rule induction for an $n$-ary inductive relation $R$