author | huffman |
Fri, 26 Aug 2011 10:38:29 -0700 | |
changeset 44534 | 002b43117115 |
parent 43564 | 9864182c6bad |
child 48891 | c0eafbd55de3 |
permissions | -rw-r--r-- |
31678 | 1 |
theory Setup |
2 |
imports Main |
|
3 |
uses |
|
4 |
"../../antiquote_setup.ML" |
|
5 |
"../../more_antiquote.ML" |
|
6 |
begin |
|
7 |
||
43564
9864182c6bad
document antiquotations are managed as theory data, with proper name space and entity markup;
wenzelm
parents:
31678
diff
changeset
|
8 |
setup {* Antiquote_Setup.setup #> More_Antiquote.setup *} |
9864182c6bad
document antiquotations are managed as theory data, with proper name space and entity markup;
wenzelm
parents:
31678
diff
changeset
|
9 |
|
9864182c6bad
document antiquotations are managed as theory data, with proper name space and entity markup;
wenzelm
parents:
31678
diff
changeset
|
10 |
|
31678 | 11 |
end |