changeset 43564 | 9864182c6bad |
parent 42637 | 381fdcab0f36 |
child 48895 | 4cd4ef1ef4a4 |
--- 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 *}