| author | blanchet |
| Mon, 04 Nov 2013 10:52:41 +0100 | |
| changeset 54238 | 58742c759205 |
| parent 48985 | 5386df44a037 |
| child 56059 | 2390391584c2 |
| permissions | -rw-r--r-- |
| 29755 | 1 |
theory Base |
| 39846 | 2 |
imports Main |
| 18537 | 3 |
begin |
| 30272 | 4 |
|
|
48938
d468d72a458f
more standard document preparation within session context;
wenzelm
parents:
48891
diff
changeset
|
5 |
ML_file "../antiquote_setup.ML" |
|
43564
9864182c6bad
document antiquotations are managed as theory data, with proper name space and entity markup;
wenzelm
parents:
40110
diff
changeset
|
6 |
setup {* Antiquote_Setup.setup *}
|
|
9864182c6bad
document antiquotations are managed as theory data, with proper name space and entity markup;
wenzelm
parents:
40110
diff
changeset
|
7 |
|
| 18537 | 8 |
end |