| author | blanchet |
| Fri, 16 May 2014 19:13:50 +0200 | |
| changeset 56984 | d20f19f54789 |
| parent 56240 | 938c6c7e10eb |
| child 59324 | f5f9993a168d |
| 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" |
|
| 51162 | 7 |
"~~/src/HOL/Library/IArray" |
| 28213 | 8 |
begin |
9 |
||
|
48951
b9238cbcdd41
more standard document preparation within session context;
wenzelm
parents:
48891
diff
changeset
|
10 |
(* FIXME avoid writing into source directory *) |
|
b9238cbcdd41
more standard document preparation within session context;
wenzelm
parents:
48891
diff
changeset
|
11 |
ML {*
|
| 56208 | 12 |
Isabelle_System.mkdirs (Path.append (Resources.master_directory @{theory}) (Path.basic "examples"))
|
|
48951
b9238cbcdd41
more standard document preparation within session context;
wenzelm
parents:
48891
diff
changeset
|
13 |
*} |
|
b9238cbcdd41
more standard document preparation within session context;
wenzelm
parents:
48891
diff
changeset
|
14 |
|
|
b9238cbcdd41
more standard document preparation within session context;
wenzelm
parents:
48891
diff
changeset
|
15 |
ML_file "../antiquote_setup.ML" |
|
b9238cbcdd41
more standard document preparation within session context;
wenzelm
parents:
48891
diff
changeset
|
16 |
ML_file "../more_antiquote.ML" |
| 48891 | 17 |
|
| 38503 | 18 |
setup {*
|
19 |
let |
|
20 |
val typ = Simple_Syntax.read_typ; |
|
21 |
in |
|
| 56240 | 22 |
Sign.del_syntax (Symbol.xsymbolsN, false) |
|
42293
6cca0343ea48
renamed sprop "prop#" to "prop'" -- proper identifier;
wenzelm
parents:
42288
diff
changeset
|
23 |
[("_constrain", typ "logic => type => logic", Mixfix ("_\<Colon>_", [4, 0], 3)),
|
|
6cca0343ea48
renamed sprop "prop#" to "prop'" -- proper identifier;
wenzelm
parents:
42288
diff
changeset
|
24 |
("_constrain", typ "prop' => type => prop'", Mixfix ("_\<Colon>_", [4, 0], 3))] #>
|
| 56240 | 25 |
Sign.add_syntax (Symbol.xsymbolsN, false) |
|
42293
6cca0343ea48
renamed sprop "prop#" to "prop'" -- proper identifier;
wenzelm
parents:
42288
diff
changeset
|
26 |
[("_constrain", typ "logic => type => logic", Mixfix ("_ \<Colon> _", [4, 0], 3)),
|
|
6cca0343ea48
renamed sprop "prop#" to "prop'" -- proper identifier;
wenzelm
parents:
42288
diff
changeset
|
27 |
("_constrain", typ "prop' => type => prop'", Mixfix ("_ \<Colon> _", [4, 0], 3))]
|
| 38503 | 28 |
end |
29 |
*} |
|
30 |
||
| 34071 | 31 |
setup {* Code_Target.set_default_code_width 74 *}
|
32 |
||
|
42669
04dfffda5671
more conventional naming scheme: names_long, names_short, names_unique;
wenzelm
parents:
42358
diff
changeset
|
33 |
declare [[names_unique = false]] |
| 28213 | 34 |
|
35 |
end |
|
| 46517 | 36 |