1
(*:maxLineLen=78:*)
2
3
theory Setup
4
imports Main
5
begin
6
7
ML_file \<open>../antiquote_setup.ML\<close>
8
ML_file \<open>../more_antiquote.ML\<close>
9
10
end