doc-src/TutorialI/Inductive/Advanced.thy
changeset 32891 d403b99287ff
parent 27167 a99747ccba87
child 39795 9e59b4c11039
--- a/doc-src/TutorialI/Inductive/Advanced.thy	Wed Oct 07 16:57:56 2009 +0200
+++ b/doc-src/TutorialI/Inductive/Advanced.thy	Thu Oct 08 15:16:13 2009 +0200
@@ -185,7 +185,7 @@
 
 Even with its use of the function \isa{lists}, the premise of our
 introduction rule is positive:
-@{thm_style [display,indent=0] prem1 step [no_vars]}
+@{thm [display,indent=0] (prem 1) step [no_vars]}
 To apply the rule we construct a list @{term args} of previously
 constructed well-formed terms.  We obtain a
 new term, @{term "Apply f args"}.  Because @{term lists} is monotone,