| author | krauss | 
| Sun, 21 Aug 2011 22:13:04 +0200 | |
| changeset 44367 | 74c08021ab2e | 
| parent 43564 | 9864182c6bad | 
| child 48891 | c0eafbd55de3 | 
| permissions | -rw-r--r-- | 
| 42651 | 1 | theory Base | 
| 2 | imports Pure | |
| 3 | uses "../../antiquote_setup.ML" | |
| 4 | begin | |
| 5 | ||
| 6 | setup {*
 | |
| 43564 
9864182c6bad
document antiquotations are managed as theory data, with proper name space and entity markup;
 wenzelm parents: 
42651diff
changeset | 7 | Antiquote_Setup.setup #> | 
| 42651 | 8 | member (op =) (Session.id ()) "ZF" ? Pure_Thy.old_appl_syntax_setup | 
| 9 | *} | |
| 10 | ||
| 11 | declare [[thy_output_source]] | |
| 12 | ||
| 13 | end |