| author | Cezary Kaliszyk <kaliszyk@in.tum.de> | 
| Wed, 20 Jul 2011 16:14:49 +0200 | |
| changeset 43934 | 2108763f298d | 
| parent 43564 | 9864182c6bad | 
| child 46517 | 9d2e682a68eb | 
| permissions | -rw-r--r-- | 
| 28213 | 1 | theory Setup | 
| 39066 | 2 | imports | 
| 3 | Complex_Main | |
| 43271 | 4 | More_List RBT Dlist List_Cset Mapping | 
| 30227 | 5 | uses | 
| 6 | "../../antiquote_setup.ML" | |
| 7 | "../../more_antiquote.ML" | |
| 28213 | 8 | begin | 
| 9 | ||
| 38503 | 10 | setup {*
 | 
| 43564 
9864182c6bad
document antiquotations are managed as theory data, with proper name space and entity markup;
 wenzelm parents: 
43271diff
changeset | 11 | Antiquote_Setup.setup #> | 
| 
9864182c6bad
document antiquotations are managed as theory data, with proper name space and entity markup;
 wenzelm parents: 
43271diff
changeset | 12 | More_Antiquote.setup #> | 
| 38503 | 13 | let | 
| 14 | val typ = Simple_Syntax.read_typ; | |
| 15 | in | |
| 42293 
6cca0343ea48
renamed sprop "prop#" to "prop'" -- proper identifier;
 wenzelm parents: 
42288diff
changeset | 16 | Sign.del_modesyntax_i (Symbol.xsymbolsN, false) | 
| 
6cca0343ea48
renamed sprop "prop#" to "prop'" -- proper identifier;
 wenzelm parents: 
42288diff
changeset | 17 |    [("_constrain", typ "logic => type => logic", Mixfix ("_\<Colon>_", [4, 0], 3)),
 | 
| 
6cca0343ea48
renamed sprop "prop#" to "prop'" -- proper identifier;
 wenzelm parents: 
42288diff
changeset | 18 |     ("_constrain", typ "prop' => type => prop'", Mixfix ("_\<Colon>_", [4, 0], 3))] #>
 | 
| 
6cca0343ea48
renamed sprop "prop#" to "prop'" -- proper identifier;
 wenzelm parents: 
42288diff
changeset | 19 | Sign.add_modesyntax_i (Symbol.xsymbolsN, false) | 
| 
6cca0343ea48
renamed sprop "prop#" to "prop'" -- proper identifier;
 wenzelm parents: 
42288diff
changeset | 20 |    [("_constrain", typ "logic => type => logic", Mixfix ("_ \<Colon>  _", [4, 0], 3)),
 | 
| 
6cca0343ea48
renamed sprop "prop#" to "prop'" -- proper identifier;
 wenzelm parents: 
42288diff
changeset | 21 |     ("_constrain", typ "prop' => type => prop'", Mixfix ("_ \<Colon> _", [4, 0], 3))]
 | 
| 38503 | 22 | end | 
| 23 | *} | |
| 24 | ||
| 34071 | 25 | setup {* Code_Target.set_default_code_width 74 *}
 | 
| 26 | ||
| 42669 
04dfffda5671
more conventional naming scheme: names_long, names_short, names_unique;
 wenzelm parents: 
42358diff
changeset | 27 | declare [[names_unique = false]] | 
| 28213 | 28 | |
| 29 | end |