author | haftmann |
Mon, 01 Jun 2015 18:59:20 +0200 | |
changeset 60344 | a40369ea3ba5 |
parent 59970 | e9f73d87d904 |
child 61246 | 077b88f9ec16 |
permissions | -rw-r--r-- |
35626 | 1 |
(* Title: Pure/Isar/typedecl.ML |
2 |
Author: Makarius |
|
3 |
||
36172 | 4 |
Type declarations (with object-logic arities) and type abbreviations. |
35626 | 5 |
*) |
6 |
||
7 |
signature TYPEDECL = |
|
8 |
sig |
|
35838 | 9 |
val read_constraint: Proof.context -> string option -> sort |
36153
1ac501e16a6a
replaced slightly odd Typedecl.predeclare_constraints by plain declaration of type arguments -- also avoid "recursive" declaration of type constructor, which can cause problems with sequential definitions B.foo = A.foo;
wenzelm
parents:
35838
diff
changeset
|
10 |
val basic_typedecl: binding * int * mixfix -> local_theory -> string * local_theory |
35834
0c71e0d72d7a
eliminated slightly odd typedecl_wrt in favour of explicit predeclare_constraints (which also works for recursive types);
wenzelm
parents:
35740
diff
changeset
|
11 |
val typedecl: binding * (string * sort) list * mixfix -> local_theory -> typ * local_theory |
0c71e0d72d7a
eliminated slightly odd typedecl_wrt in favour of explicit predeclare_constraints (which also works for recursive types);
wenzelm
parents:
35740
diff
changeset
|
12 |
val typedecl_global: binding * (string * sort) list * mixfix -> theory -> typ * theory |
36172 | 13 |
val abbrev: binding * string list * mixfix -> typ -> local_theory -> string * local_theory |
14 |
val abbrev_cmd: binding * string list * mixfix -> string -> local_theory -> string * local_theory |
|
15 |
val abbrev_global: binding * string list * mixfix -> typ -> theory -> string * theory |
|
35626 | 16 |
end; |
17 |
||
18 |
structure Typedecl: TYPEDECL = |
|
19 |
struct |
|
20 |
||
36153
1ac501e16a6a
replaced slightly odd Typedecl.predeclare_constraints by plain declaration of type arguments -- also avoid "recursive" declaration of type constructor, which can cause problems with sequential definitions B.foo = A.foo;
wenzelm
parents:
35838
diff
changeset
|
21 |
(* constraints *) |
1ac501e16a6a
replaced slightly odd Typedecl.predeclare_constraints by plain declaration of type arguments -- also avoid "recursive" declaration of type constructor, which can cause problems with sequential definitions B.foo = A.foo;
wenzelm
parents:
35838
diff
changeset
|
22 |
|
1ac501e16a6a
replaced slightly odd Typedecl.predeclare_constraints by plain declaration of type arguments -- also avoid "recursive" declaration of type constructor, which can cause problems with sequential definitions B.foo = A.foo;
wenzelm
parents:
35838
diff
changeset
|
23 |
fun read_constraint _ NONE = dummyS |
1ac501e16a6a
replaced slightly odd Typedecl.predeclare_constraints by plain declaration of type arguments -- also avoid "recursive" declaration of type constructor, which can cause problems with sequential definitions B.foo = A.foo;
wenzelm
parents:
35838
diff
changeset
|
24 |
| read_constraint ctxt (SOME s) = Syntax.read_sort ctxt s; |
1ac501e16a6a
replaced slightly odd Typedecl.predeclare_constraints by plain declaration of type arguments -- also avoid "recursive" declaration of type constructor, which can cause problems with sequential definitions B.foo = A.foo;
wenzelm
parents:
35838
diff
changeset
|
25 |
|
1ac501e16a6a
replaced slightly odd Typedecl.predeclare_constraints by plain declaration of type arguments -- also avoid "recursive" declaration of type constructor, which can cause problems with sequential definitions B.foo = A.foo;
wenzelm
parents:
35838
diff
changeset
|
26 |
|
35834
0c71e0d72d7a
eliminated slightly odd typedecl_wrt in favour of explicit predeclare_constraints (which also works for recursive types);
wenzelm
parents:
35740
diff
changeset
|
27 |
(* primitives *) |
0c71e0d72d7a
eliminated slightly odd typedecl_wrt in favour of explicit predeclare_constraints (which also works for recursive types);
wenzelm
parents:
35740
diff
changeset
|
28 |
|
36172 | 29 |
fun basic_decl decl (b, n, mx) lthy = |
35834
0c71e0d72d7a
eliminated slightly odd typedecl_wrt in favour of explicit predeclare_constraints (which also works for recursive types);
wenzelm
parents:
35740
diff
changeset
|
30 |
let val name = Local_Theory.full_name lthy b in |
0c71e0d72d7a
eliminated slightly odd typedecl_wrt in favour of explicit predeclare_constraints (which also works for recursive types);
wenzelm
parents:
35740
diff
changeset
|
31 |
lthy |
38757
2b3e054ae6fc
renamed Local_Theory.theory(_result) to Local_Theory.background_theory(_result) to emphasize that this belongs to the infrastructure and is rarely appropriate in user-space tools;
wenzelm
parents:
38388
diff
changeset
|
32 |
|> Local_Theory.background_theory (decl name) |
35834
0c71e0d72d7a
eliminated slightly odd typedecl_wrt in favour of explicit predeclare_constraints (which also works for recursive types);
wenzelm
parents:
35740
diff
changeset
|
33 |
|> Local_Theory.type_notation true Syntax.mode_default [(Type (name, replicate n dummyT), mx)] |
0c71e0d72d7a
eliminated slightly odd typedecl_wrt in favour of explicit predeclare_constraints (which also works for recursive types);
wenzelm
parents:
35740
diff
changeset
|
34 |
|> Local_Theory.type_alias b name |
0c71e0d72d7a
eliminated slightly odd typedecl_wrt in favour of explicit predeclare_constraints (which also works for recursive types);
wenzelm
parents:
35740
diff
changeset
|
35 |
|> pair name |
0c71e0d72d7a
eliminated slightly odd typedecl_wrt in favour of explicit predeclare_constraints (which also works for recursive types);
wenzelm
parents:
35740
diff
changeset
|
36 |
end; |
0c71e0d72d7a
eliminated slightly odd typedecl_wrt in favour of explicit predeclare_constraints (which also works for recursive types);
wenzelm
parents:
35740
diff
changeset
|
37 |
|
42375
774df7c59508
report Name_Space.declare/define, relatively to context;
wenzelm
parents:
42360
diff
changeset
|
38 |
fun basic_typedecl (b, n, mx) lthy = |
59970 | 39 |
basic_decl (fn name => |
40 |
Sign.add_type lthy (b, n, NoSyn) #> |
|
41 |
(case Object_Logic.get_base_sort lthy of |
|
42 |
SOME S => Axclass.arity_axiomatization (name, replicate n S, S) |
|
43 |
| NONE => I)) (b, n, mx) lthy; |
|
35834
0c71e0d72d7a
eliminated slightly odd typedecl_wrt in favour of explicit predeclare_constraints (which also works for recursive types);
wenzelm
parents:
35740
diff
changeset
|
44 |
|
0c71e0d72d7a
eliminated slightly odd typedecl_wrt in favour of explicit predeclare_constraints (which also works for recursive types);
wenzelm
parents:
35740
diff
changeset
|
45 |
|
36172 | 46 |
(* global type -- without dependencies on type parameters of the context *) |
47 |
||
48 |
fun global_type lthy (b, raw_args) = |
|
35626 | 49 |
let |
42381
309ec68442c6
added Binding.print convenience, which includes quote already;
wenzelm
parents:
42375
diff
changeset
|
50 |
fun err msg = error (msg ^ " in type declaration " ^ Binding.print b); |
35681 | 51 |
|
35834
0c71e0d72d7a
eliminated slightly odd typedecl_wrt in favour of explicit predeclare_constraints (which also works for recursive types);
wenzelm
parents:
35740
diff
changeset
|
52 |
val _ = has_duplicates (eq_fst op =) raw_args andalso err "Duplicate parameters"; |
42360 | 53 |
val args = map (TFree o Proof_Context.check_tfree lthy) raw_args; |
36156 | 54 |
val T = Type (Local_Theory.full_name lthy b, args); |
35681 | 55 |
|
56 |
val bad_args = |
|
57 |
#2 (Term.dest_Type (Logic.type_map (singleton (Variable.polymorphic lthy)) T)) |
|
58 |
|> filter_out Term.is_TVar; |
|
36172 | 59 |
val _ = null bad_args orelse |
35740
d3726291f252
added typedecl_wrt, which affects default sorts of type args;
wenzelm
parents:
35714
diff
changeset
|
60 |
err ("Locally fixed type arguments " ^ |
35834
0c71e0d72d7a
eliminated slightly odd typedecl_wrt in favour of explicit predeclare_constraints (which also works for recursive types);
wenzelm
parents:
35740
diff
changeset
|
61 |
commas_quote (map (Syntax.string_of_typ lthy) bad_args)); |
36172 | 62 |
in T end; |
63 |
||
64 |
||
65 |
(* type declarations *) |
|
66 |
||
67 |
fun typedecl (b, raw_args, mx) lthy = |
|
68 |
let val T = global_type lthy (b, raw_args) in |
|
35681 | 69 |
lthy |
36172 | 70 |
|> basic_typedecl (b, length raw_args, mx) |
35834
0c71e0d72d7a
eliminated slightly odd typedecl_wrt in favour of explicit predeclare_constraints (which also works for recursive types);
wenzelm
parents:
35740
diff
changeset
|
71 |
|> snd |
35681 | 72 |
|> Variable.declare_typ T |
35626 | 73 |
|> pair T |
74 |
end; |
|
75 |
||
35681 | 76 |
fun typedecl_global decl = |
38388 | 77 |
Named_Target.theory_init |
35681 | 78 |
#> typedecl decl |
79 |
#> Local_Theory.exit_result_global Morphism.typ; |
|
80 |
||
36172 | 81 |
|
82 |
(* type abbreviations *) |
|
83 |
||
36457
7355af2a7e8a
tuned user-level type abbrevs: explicit warning concerning ignored sort constraints -- sorts never affect formation of types and type abbrevs strip sorts internally;
wenzelm
parents:
36179
diff
changeset
|
84 |
local |
7355af2a7e8a
tuned user-level type abbrevs: explicit warning concerning ignored sort constraints -- sorts never affect formation of types and type abbrevs strip sorts internally;
wenzelm
parents:
36179
diff
changeset
|
85 |
|
36172 | 86 |
fun gen_abbrev prep_typ (b, vs, mx) raw_rhs lthy = |
87 |
let |
|
88 |
val Type (name, _) = global_type lthy (b, map (rpair dummyS) vs); |
|
36457
7355af2a7e8a
tuned user-level type abbrevs: explicit warning concerning ignored sort constraints -- sorts never affect formation of types and type abbrevs strip sorts internally;
wenzelm
parents:
36179
diff
changeset
|
89 |
val rhs = prep_typ b lthy raw_rhs |
42381
309ec68442c6
added Binding.print convenience, which includes quote already;
wenzelm
parents:
42375
diff
changeset
|
90 |
handle ERROR msg => cat_error msg ("in type abbreviation " ^ Binding.print b); |
36172 | 91 |
in |
92 |
lthy |
|
42375
774df7c59508
report Name_Space.declare/define, relatively to context;
wenzelm
parents:
42360
diff
changeset
|
93 |
|> basic_decl (fn _ => Sign.add_type_abbrev lthy (b, vs, rhs)) (b, length vs, mx) |
36172 | 94 |
|> snd |
95 |
|> pair name |
|
96 |
end; |
|
97 |
||
36457
7355af2a7e8a
tuned user-level type abbrevs: explicit warning concerning ignored sort constraints -- sorts never affect formation of types and type abbrevs strip sorts internally;
wenzelm
parents:
36179
diff
changeset
|
98 |
fun read_abbrev b ctxt raw_rhs = |
7355af2a7e8a
tuned user-level type abbrevs: explicit warning concerning ignored sort constraints -- sorts never affect formation of types and type abbrevs strip sorts internally;
wenzelm
parents:
36179
diff
changeset
|
99 |
let |
42360 | 100 |
val rhs = Proof_Context.read_typ_syntax (ctxt |> Proof_Context.set_defsort []) raw_rhs; |
36457
7355af2a7e8a
tuned user-level type abbrevs: explicit warning concerning ignored sort constraints -- sorts never affect formation of types and type abbrevs strip sorts internally;
wenzelm
parents:
36179
diff
changeset
|
101 |
val ignored = Term.fold_atyps_sorts (fn (_, []) => I | (T, _) => insert (op =) T) rhs []; |
7355af2a7e8a
tuned user-level type abbrevs: explicit warning concerning ignored sort constraints -- sorts never affect formation of types and type abbrevs strip sorts internally;
wenzelm
parents:
36179
diff
changeset
|
102 |
val _ = |
56294
85911b8a6868
prefer Context_Position where a context is available;
wenzelm
parents:
51685
diff
changeset
|
103 |
if not (null ignored) andalso Context_Position.is_visible ctxt then |
85911b8a6868
prefer Context_Position where a context is available;
wenzelm
parents:
51685
diff
changeset
|
104 |
warning |
85911b8a6868
prefer Context_Position where a context is available;
wenzelm
parents:
51685
diff
changeset
|
105 |
("Ignoring sort constraints in type variables(s): " ^ |
85911b8a6868
prefer Context_Position where a context is available;
wenzelm
parents:
51685
diff
changeset
|
106 |
commas_quote (map (Syntax.string_of_typ ctxt) (rev ignored)) ^ |
85911b8a6868
prefer Context_Position where a context is available;
wenzelm
parents:
51685
diff
changeset
|
107 |
"\nin type abbreviation " ^ Binding.print b) |
85911b8a6868
prefer Context_Position where a context is available;
wenzelm
parents:
51685
diff
changeset
|
108 |
else (); |
36457
7355af2a7e8a
tuned user-level type abbrevs: explicit warning concerning ignored sort constraints -- sorts never affect formation of types and type abbrevs strip sorts internally;
wenzelm
parents:
36179
diff
changeset
|
109 |
in rhs end; |
7355af2a7e8a
tuned user-level type abbrevs: explicit warning concerning ignored sort constraints -- sorts never affect formation of types and type abbrevs strip sorts internally;
wenzelm
parents:
36179
diff
changeset
|
110 |
|
7355af2a7e8a
tuned user-level type abbrevs: explicit warning concerning ignored sort constraints -- sorts never affect formation of types and type abbrevs strip sorts internally;
wenzelm
parents:
36179
diff
changeset
|
111 |
in |
7355af2a7e8a
tuned user-level type abbrevs: explicit warning concerning ignored sort constraints -- sorts never affect formation of types and type abbrevs strip sorts internally;
wenzelm
parents:
36179
diff
changeset
|
112 |
|
42360 | 113 |
val abbrev = gen_abbrev (K Proof_Context.cert_typ_syntax); |
36457
7355af2a7e8a
tuned user-level type abbrevs: explicit warning concerning ignored sort constraints -- sorts never affect formation of types and type abbrevs strip sorts internally;
wenzelm
parents:
36179
diff
changeset
|
114 |
val abbrev_cmd = gen_abbrev read_abbrev; |
7355af2a7e8a
tuned user-level type abbrevs: explicit warning concerning ignored sort constraints -- sorts never affect formation of types and type abbrevs strip sorts internally;
wenzelm
parents:
36179
diff
changeset
|
115 |
|
7355af2a7e8a
tuned user-level type abbrevs: explicit warning concerning ignored sort constraints -- sorts never affect formation of types and type abbrevs strip sorts internally;
wenzelm
parents:
36179
diff
changeset
|
116 |
end; |
36172 | 117 |
|
118 |
fun abbrev_global decl rhs = |
|
38388 | 119 |
Named_Target.theory_init |
36172 | 120 |
#> abbrev decl rhs |
121 |
#> Local_Theory.exit_result_global (K I); |
|
122 |
||
35626 | 123 |
end; |
124 |