1826
|
1 |
val thy = mk_base [Thy "Ord"] "Set2g" true;
|
|
2 |
|
|
3 |
structure Set2g =
|
|
4 |
struct
|
|
5 |
|
|
6 |
local
|
|
7 |
val parse_ast_translation = [];
|
|
8 |
val parse_translation = [];
|
|
9 |
val print_translation = [];
|
|
10 |
val print_ast_translation = [];
|
|
11 |
in
|
|
12 |
|
|
13 |
|
|
14 |
|
|
15 |
val thy = thy
|
|
16 |
|
|
17 |
|> add_trfuns
|
|
18 |
(parse_ast_translation, parse_translation, print_translation, print_ast_translation)
|
|
19 |
|
|
20 |
|> add_types
|
|
21 |
[("set", 1, NoSyn)]
|
|
22 |
|
|
23 |
|> add_tyabbrs
|
|
24 |
[]
|
|
25 |
|
|
26 |
|> add_consts
|
|
27 |
[("Ball", "'a set ë ('a ë bool) ë bool", NoSyn)]
|
|
28 |
|
|
29 |
|> add_syntax
|
|
30 |
[("GBall", "pttrn ë 'a set ë bool ë bool", Mixfix ("(3Â _ Î _ ./ _)", [], 10))]
|
|
31 |
|
|
32 |
|> add_trrules
|
|
33 |
[("logic", "Â x Î A . P") <-> ("logic", "Ball A (³x. P)")]
|
|
34 |
|
|
35 |
|> add_thyname "Set2g";
|
|
36 |
|
|
37 |
val _ = store_theory (thy, "Set2g");
|
|
38 |
|
|
39 |
|
|
40 |
|
|
41 |
|
|
42 |
end;
|
|
43 |
end;
|