doc-src/Classes/Thy/Setup.thy
changeset 43564 9864182c6bad
parent 42224 578a51fae383
child 48891 c0eafbd55de3
--- a/doc-src/Classes/Thy/Setup.thy	Mon Jun 27 17:51:28 2011 +0200
+++ b/doc-src/Classes/Thy/Setup.thy	Mon Jun 27 22:20:49 2011 +0200
@@ -5,7 +5,11 @@
   "../../more_antiquote.ML"
 begin
 
-setup {* Code_Target.set_default_code_width 74 *}
+setup {*
+  Antiquote_Setup.setup #>
+  More_Antiquote.setup #>
+  Code_Target.set_default_code_width 74
+*}
 
 syntax
   "_alpha" :: "type"  ("\<alpha>")