author | wenzelm |
Fri, 13 Nov 2015 14:49:30 +0100 | |
changeset 61656 | cfabbc083977 |
parent 56059 | 2390391584c2 |
child 69605 | a96320074298 |
permissions | -rw-r--r-- |
61656 | 1 |
(*:maxLineLen=78:*) |
2 |
||
43564
9864182c6bad
document antiquotations are managed as theory data, with proper name space and entity markup;
wenzelm
parents:
diff
changeset
|
3 |
theory Base |
9864182c6bad
document antiquotations are managed as theory data, with proper name space and entity markup;
wenzelm
parents:
diff
changeset
|
4 |
imports Pure |
9864182c6bad
document antiquotations are managed as theory data, with proper name space and entity markup;
wenzelm
parents:
diff
changeset
|
5 |
begin |
9864182c6bad
document antiquotations are managed as theory data, with proper name space and entity markup;
wenzelm
parents:
diff
changeset
|
6 |
|
48937
e7418f8d49fe
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:
diff
changeset
|
8 |
|
9864182c6bad
document antiquotations are managed as theory data, with proper name space and entity markup;
wenzelm
parents:
diff
changeset
|
9 |
end |