author | haftmann |
Sat, 18 Feb 2012 20:07:26 +0100 | |
changeset 46517 | 9d2e682a68eb |
parent 43564 | 9864182c6bad |
child 48891 | c0eafbd55de3 |
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" |
|
30227 | 7 |
uses |
8 |
"../../antiquote_setup.ML" |
|
9 |
"../../more_antiquote.ML" |
|
28213 | 10 |
begin |
11 |
||
38503 | 12 |
setup {* |
43564
9864182c6bad
document antiquotations are managed as theory data, with proper name space and entity markup;
wenzelm
parents:
43271
diff
changeset
|
13 |
Antiquote_Setup.setup #> |
9864182c6bad
document antiquotations are managed as theory data, with proper name space and entity markup;
wenzelm
parents:
43271
diff
changeset
|
14 |
More_Antiquote.setup #> |
38503 | 15 |
let |
16 |
val typ = Simple_Syntax.read_typ; |
|
17 |
in |
|
42293
6cca0343ea48
renamed sprop "prop#" to "prop'" -- proper identifier;
wenzelm
parents:
42288
diff
changeset
|
18 |
Sign.del_modesyntax_i (Symbol.xsymbolsN, false) |
6cca0343ea48
renamed sprop "prop#" to "prop'" -- proper identifier;
wenzelm
parents:
42288
diff
changeset
|
19 |
[("_constrain", typ "logic => type => logic", Mixfix ("_\<Colon>_", [4, 0], 3)), |
6cca0343ea48
renamed sprop "prop#" to "prop'" -- proper identifier;
wenzelm
parents:
42288
diff
changeset
|
20 |
("_constrain", typ "prop' => type => prop'", Mixfix ("_\<Colon>_", [4, 0], 3))] #> |
6cca0343ea48
renamed sprop "prop#" to "prop'" -- proper identifier;
wenzelm
parents:
42288
diff
changeset
|
21 |
Sign.add_modesyntax_i (Symbol.xsymbolsN, false) |
6cca0343ea48
renamed sprop "prop#" to "prop'" -- proper identifier;
wenzelm
parents:
42288
diff
changeset
|
22 |
[("_constrain", typ "logic => type => logic", Mixfix ("_ \<Colon> _", [4, 0], 3)), |
6cca0343ea48
renamed sprop "prop#" to "prop'" -- proper identifier;
wenzelm
parents:
42288
diff
changeset
|
23 |
("_constrain", typ "prop' => type => prop'", Mixfix ("_ \<Colon> _", [4, 0], 3))] |
38503 | 24 |
end |
25 |
*} |
|
26 |
||
34071 | 27 |
setup {* Code_Target.set_default_code_width 74 *} |
28 |
||
42669
04dfffda5671
more conventional naming scheme: names_long, names_short, names_unique;
wenzelm
parents:
42358
diff
changeset
|
29 |
declare [[names_unique = false]] |
28213 | 30 |
|
31 |
end |
|
46517 | 32 |