diff -r aeabb735883a -r 9864182c6bad doc-src/TutorialI/Inductive/Even.thy --- a/doc-src/TutorialI/Inductive/Even.thy Mon Jun 27 17:51:28 2011 +0200 +++ b/doc-src/TutorialI/Inductive/Even.thy Mon Jun 27 22:20:49 2011 +0200 @@ -1,4 +1,6 @@ -(*<*)theory Even imports Main uses "../../antiquote_setup.ML" begin(*>*) +(*<*)theory Even imports Main uses "../../antiquote_setup.ML" begin +setup {* Antiquote_Setup.setup *} +(*>*) section{* The Set of Even Numbers *}