| author | wenzelm |
| Sat, 03 Nov 2018 19:31:15 +0100 | |
| changeset 69223 | 44d68a00917c |
| parent 61656 | cfabbc083977 |
| child 69605 | a96320074298 |
| permissions | -rw-r--r-- |
| 61656 | 1 |
(*:maxLineLen=78:*) |
2 |
||
| 29755 | 3 |
theory Base |
| 39846 | 4 |
imports Main |
| 18537 | 5 |
begin |
| 30272 | 6 |
|
|
48938
d468d72a458f
more standard document preparation within session context;
wenzelm
parents:
48891
diff
changeset
|
7 |
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
|
8 |
|
| 18537 | 9 |
end |