| author | wenzelm | 
| Mon, 17 Dec 2012 14:07:34 +0100 | |
| changeset 50575 | ae1da46022d1 | 
| parent 48985 | 5386df44a037 | 
| child 51162 | 310b94ed1815 | 
| permissions | -rw-r--r-- | 
| 28213 | 1 | theory Setup | 
| 39066 | 2 | imports | 
| 3 | Complex_Main | |
| 46517 | 4 | "~~/src/HOL/Library/Dlist" | 
| 5 | "~~/src/HOL/Library/RBT" | |
| 6 | "~~/src/HOL/Library/Mapping" | |
| 28213 | 7 | begin | 
| 8 | ||
| 48951 
b9238cbcdd41
more standard document preparation within session context;
 wenzelm parents: 
48891diff
changeset | 9 | (* FIXME avoid writing into source directory *) | 
| 
b9238cbcdd41
more standard document preparation within session context;
 wenzelm parents: 
48891diff
changeset | 10 | ML {*
 | 
| 
b9238cbcdd41
more standard document preparation within session context;
 wenzelm parents: 
48891diff
changeset | 11 |   Isabelle_System.mkdirs (Path.append (Thy_Load.master_directory @{theory}) (Path.basic "examples"))
 | 
| 
b9238cbcdd41
more standard document preparation within session context;
 wenzelm parents: 
48891diff
changeset | 12 | *} | 
| 
b9238cbcdd41
more standard document preparation within session context;
 wenzelm parents: 
48891diff
changeset | 13 | |
| 
b9238cbcdd41
more standard document preparation within session context;
 wenzelm parents: 
48891diff
changeset | 14 | ML_file "../antiquote_setup.ML" | 
| 
b9238cbcdd41
more standard document preparation within session context;
 wenzelm parents: 
48891diff
changeset | 15 | ML_file "../more_antiquote.ML" | 
| 48891 | 16 | |
| 38503 | 17 | setup {*
 | 
| 43564 
9864182c6bad
document antiquotations are managed as theory data, with proper name space and entity markup;
 wenzelm parents: 
43271diff
changeset | 18 | Antiquote_Setup.setup #> | 
| 
9864182c6bad
document antiquotations are managed as theory data, with proper name space and entity markup;
 wenzelm parents: 
43271diff
changeset | 19 | More_Antiquote.setup #> | 
| 38503 | 20 | let | 
| 21 | val typ = Simple_Syntax.read_typ; | |
| 22 | in | |
| 42293 
6cca0343ea48
renamed sprop "prop#" to "prop'" -- proper identifier;
 wenzelm parents: 
42288diff
changeset | 23 | Sign.del_modesyntax_i (Symbol.xsymbolsN, false) | 
| 
6cca0343ea48
renamed sprop "prop#" to "prop'" -- proper identifier;
 wenzelm parents: 
42288diff
changeset | 24 |    [("_constrain", typ "logic => type => logic", Mixfix ("_\<Colon>_", [4, 0], 3)),
 | 
| 
6cca0343ea48
renamed sprop "prop#" to "prop'" -- proper identifier;
 wenzelm parents: 
42288diff
changeset | 25 |     ("_constrain", typ "prop' => type => prop'", Mixfix ("_\<Colon>_", [4, 0], 3))] #>
 | 
| 
6cca0343ea48
renamed sprop "prop#" to "prop'" -- proper identifier;
 wenzelm parents: 
42288diff
changeset | 26 | Sign.add_modesyntax_i (Symbol.xsymbolsN, false) | 
| 
6cca0343ea48
renamed sprop "prop#" to "prop'" -- proper identifier;
 wenzelm parents: 
42288diff
changeset | 27 |    [("_constrain", typ "logic => type => logic", Mixfix ("_ \<Colon>  _", [4, 0], 3)),
 | 
| 
6cca0343ea48
renamed sprop "prop#" to "prop'" -- proper identifier;
 wenzelm parents: 
42288diff
changeset | 28 |     ("_constrain", typ "prop' => type => prop'", Mixfix ("_ \<Colon> _", [4, 0], 3))]
 | 
| 38503 | 29 | end | 
| 30 | *} | |
| 31 | ||
| 34071 | 32 | setup {* Code_Target.set_default_code_width 74 *}
 | 
| 33 | ||
| 42669 
04dfffda5671
more conventional naming scheme: names_long, names_short, names_unique;
 wenzelm parents: 
42358diff
changeset | 34 | declare [[names_unique = false]] | 
| 28213 | 35 | |
| 36 | end | |
| 46517 | 37 |