| author | kuncar | 
| Tue, 29 Nov 2011 15:52:51 +0100 | |
| changeset 45678 | 1a6206f538d4 | 
| 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: 
42651 
diff
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  |