| author | bulwahn | 
| Wed, 19 Oct 2011 08:37:20 +0200 | |
| changeset 45174 | 10c3597f92f0 | 
| parent 43564 | 9864182c6bad | 
| child 48891 | c0eafbd55de3 | 
| permissions | -rw-r--r-- | 
| 43564 
9864182c6bad
document antiquotations are managed as theory data, with proper name space and entity markup;
 wenzelm parents: diff
changeset | 1 | theory Base | 
| 
9864182c6bad
document antiquotations are managed as theory data, with proper name space and entity markup;
 wenzelm parents: diff
changeset | 2 | imports Pure | 
| 
9864182c6bad
document antiquotations are managed as theory data, with proper name space and entity markup;
 wenzelm parents: diff
changeset | 3 | uses "../../antiquote_setup.ML" | 
| 
9864182c6bad
document antiquotations are managed as theory data, with proper name space and entity markup;
 wenzelm parents: diff
changeset | 4 | begin | 
| 
9864182c6bad
document antiquotations are managed as theory data, with proper name space and entity markup;
 wenzelm parents: diff
changeset | 5 | |
| 
9864182c6bad
document antiquotations are managed as theory data, with proper name space and entity markup;
 wenzelm parents: diff
changeset | 6 | setup {* Antiquote_Setup.setup *}
 | 
| 
9864182c6bad
document antiquotations are managed as theory data, with proper name space and entity markup;
 wenzelm parents: diff
changeset | 7 | |
| 
9864182c6bad
document antiquotations are managed as theory data, with proper name space and entity markup;
 wenzelm parents: diff
changeset | 8 | declare [[thy_output_source]] | 
| 
9864182c6bad
document antiquotations are managed as theory data, with proper name space and entity markup;
 wenzelm parents: diff
changeset | 9 | |
| 
9864182c6bad
document antiquotations are managed as theory data, with proper name space and entity markup;
 wenzelm parents: diff
changeset | 10 | end |