| author | Fabian Huch <huch@in.tum.de> |
| Mon, 10 Jun 2024 16:02:53 +0200 | |
| changeset 80337 | 02f8a35ed8e2 |
| parent 69605 | a96320074298 |
| permissions | -rw-r--r-- |
| 61656 | 1 |
(*:maxLineLen=78:*) |
2 |
||
| 29755 | 3 |
theory Base |
| 39846 | 4 |
imports Main |
| 18537 | 5 |
begin |
| 30272 | 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:
40110
diff
changeset
|
8 |
|
| 18537 | 9 |
end |