author | wenzelm |
Sun, 09 Feb 2025 17:04:14 +0100 | |
changeset 82129 | d2d8d00543b7 |
parent 72763 | 3cc73d00553c |
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 |
72763 | 6 |
|
69605 | 7 |
ML_file \<open>../antiquote_setup.ML\<close> |
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 |