| author | wenzelm |
| Tue, 05 Apr 2016 20:03:24 +0200 | |
| changeset 62876 | 507c90523113 |
| 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 |