src/Doc/Tutorial/Types/Setup.thy
author wenzelm
Tue, 28 Aug 2012 18:57:32 +0200
changeset 48985 5386df44a037
parent 48891 doc-src/TutorialI/Types/Setup.thy@c0eafbd55de3
child 56059 2390391584c2
permissions -rw-r--r--
renamed doc-src to src/Doc; renamed TutorialI to Tutorial;

theory Setup
imports Main
begin

ML_file "../../antiquote_setup.ML"
ML_file "../../more_antiquote.ML"

setup {* Antiquote_Setup.setup #> More_Antiquote.setup *}

end