| author | wenzelm | 
| Sat, 16 Jul 2016 00:11:03 +0200 | |
| changeset 63512 | 1c7b1e294fb5 | 
| parent 63402 | f199837304d7 | 
| child 66334 | b210ae666a42 | 
| permissions | -rw-r--r-- | 
| 38379 
67d71449e85b
more convenient split of class modules: class and class_declaration
 haftmann parents: 
38376diff
changeset | 1 | (* Title: Pure/Isar/class_declaration.ML | 
| 24218 | 2 | Author: Florian Haftmann, TU Muenchen | 
| 3 | ||
| 38379 
67d71449e85b
more convenient split of class modules: class and class_declaration
 haftmann parents: 
38376diff
changeset | 4 | Declaring classes and subclass relations. | 
| 24218 | 5 | *) | 
| 6 | ||
| 38379 
67d71449e85b
more convenient split of class modules: class and class_declaration
 haftmann parents: 
38376diff
changeset | 7 | signature CLASS_DECLARATION = | 
| 24218 | 8 | sig | 
| 57181 
2d13bf9ea77b
dropped obscure and unused ad-hoc before_exit hook for named targets
 haftmann parents: 
56921diff
changeset | 9 | val class: binding -> class list -> | 
| 41585 
45d7da4e4ccf
added before_exit continuation for named targets (locale, class etc.), e.g. for final check/cleanup as in VC management;
 wenzelm parents: 
40188diff
changeset | 10 | Element.context_i list -> theory -> string * local_theory | 
| 57181 
2d13bf9ea77b
dropped obscure and unused ad-hoc before_exit hook for named targets
 haftmann parents: 
56921diff
changeset | 11 | val class_cmd: binding -> xstring list -> | 
| 41585 
45d7da4e4ccf
added before_exit continuation for named targets (locale, class etc.), e.g. for final check/cleanup as in VC management;
 wenzelm parents: 
40188diff
changeset | 12 | Element.context list -> theory -> string * local_theory | 
| 57181 
2d13bf9ea77b
dropped obscure and unused ad-hoc before_exit hook for named targets
 haftmann parents: 
56921diff
changeset | 13 | val prove_subclass: tactic -> class -> | 
| 41585 
45d7da4e4ccf
added before_exit continuation for named targets (locale, class etc.), e.g. for final check/cleanup as in VC management;
 wenzelm parents: 
40188diff
changeset | 14 | local_theory -> local_theory | 
| 57181 
2d13bf9ea77b
dropped obscure and unused ad-hoc before_exit hook for named targets
 haftmann parents: 
56921diff
changeset | 15 | val subclass: class -> local_theory -> Proof.state | 
| 
2d13bf9ea77b
dropped obscure and unused ad-hoc before_exit hook for named targets
 haftmann parents: 
56921diff
changeset | 16 | val subclass_cmd: xstring -> local_theory -> Proof.state | 
| 24218 | 17 | end; | 
| 18 | ||
| 38379 
67d71449e85b
more convenient split of class modules: class and class_declaration
 haftmann parents: 
38376diff
changeset | 19 | structure Class_Declaration: CLASS_DECLARATION = | 
| 24218 | 20 | struct | 
| 21 | ||
| 29665 
2b956243d123
explicit check for exactly one type variable in class specification elements
 haftmann parents: 
29632diff
changeset | 22 | (** class definitions **) | 
| 24218 | 23 | |
| 24 | local | |
| 25 | ||
| 29665 
2b956243d123
explicit check for exactly one type variable in class specification elements
 haftmann parents: 
29632diff
changeset | 26 | (* calculating class-related rules including canonical interpretation *) | 
| 
2b956243d123
explicit check for exactly one type variable in class specification elements
 haftmann parents: 
29632diff
changeset | 27 | |
| 29547 | 28 | fun calculate thy class sups base_sort param_map assm_axiom = | 
| 29 | let | |
| 42360 | 30 | val empty_ctxt = Proof_Context.init_global thy; | 
| 29547 | 31 | |
| 32 | (* instantiation of canonical interpretation *) | |
| 29575 
41d604e59e93
improved and corrected reading of class specs -- still draft version
 haftmann parents: 
29558diff
changeset | 33 | val aT = TFree (Name.aT, base_sort); | 
| 29627 | 34 | val param_map_const = (map o apsnd) Const param_map; | 
| 35 | val param_map_inst = (map o apsnd) | |
| 36 | (Const o apsnd (map_atyps (K aT))) param_map; | |
| 37 | val const_morph = Element.inst_morphism thy | |
| 38 | (Symtab.empty, Symtab.make param_map_inst); | |
| 29797 | 39 | val typ_morph = Element.inst_morphism thy | 
| 40 | (Symtab.empty |> Symtab.update (Name.aT, TFree (Name.aT, [class])), Symtab.empty); | |
| 41 | val (([raw_props], [(_, raw_inst_morph)], export_morph), _) = empty_ctxt | |
| 29547 | 42 |       |> Expression.cert_goal_expression ([(class, (("", false),
 | 
| 29627 | 43 | Expression.Named param_map_const))], []); | 
| 45431 | 44 | val (props, inst_morph) = | 
| 45 | if null param_map | |
| 29797 | 46 | then (raw_props |> map (Morphism.term typ_morph), | 
| 47 | raw_inst_morph $> typ_morph) | |
| 48 | else (raw_props, raw_inst_morph); (*FIXME proper handling in | |
| 49 | locale.ML / expression.ML would be desirable*) | |
| 29547 | 50 | |
| 51 | (* witness for canonical interpretation *) | |
| 52636 | 52 | val some_prop = try the_single props; | 
| 53 | val some_witn = Option.map (fn prop => | |
| 45431 | 54 | let | 
| 38379 
67d71449e85b
more convenient split of class modules: class and class_declaration
 haftmann parents: 
38376diff
changeset | 55 | val sup_axioms = map_filter (fst o Class.rules thy) sups; | 
| 45431 | 56 | val loc_intro_tac = | 
| 57 | (case Locale.intros_of thy class of | |
| 58 | (_, NONE) => all_tac | |
| 59498 
50b60f501b05
proper context for resolve_tac, eresolve_tac, dresolve_tac, forward_tac etc.;
 wenzelm parents: 
58963diff
changeset | 59 | | (_, SOME intro) => ALLGOALS (resolve_tac empty_ctxt [intro])); | 
| 29547 | 60 | val tac = loc_intro_tac | 
| 54742 
7a86358a3c0b
proper context for basic Simplifier operations: rewrite_rule, rewrite_goals_rule, rewrite_goals_tac etc.;
 wenzelm parents: 
54740diff
changeset | 61 | THEN ALLGOALS (Proof_Context.fact_tac empty_ctxt (sup_axioms @ the_list assm_axiom)); | 
| 52636 | 62 | in Element.prove_witness empty_ctxt prop tac end) some_prop; | 
| 54883 
dd04a8b654fc
proper context for norm_hhf and derived operations;
 wenzelm parents: 
54882diff
changeset | 63 | val some_axiom = Option.map (Element.conclude_witness empty_ctxt) some_witn; | 
| 29547 | 64 | |
| 65 | (* canonical interpretation *) | |
| 66 | val base_morph = inst_morph | |
| 54740 | 67 | $> Morphism.binding_morphism "class_binding" (Binding.prefix false (Class.class_prefix class)) | 
| 52636 | 68 | $> Element.satisfy_morphism (the_list some_witn); | 
| 38379 
67d71449e85b
more convenient split of class modules: class and class_declaration
 haftmann parents: 
38376diff
changeset | 69 | val eq_morph = Element.eq_morphism thy (Class.these_defs thy sups); | 
| 29547 | 70 | |
| 71 | (* assm_intro *) | |
| 30344 
10a67c5ddddb
more uniform handling of binding in targets and derived elements;
 wenzelm parents: 
30335diff
changeset | 72 | fun prove_assm_intro thm = | 
| 29547 | 73 | let | 
| 31794 
71af1fd6a5e4
renamed Variable.import_thms to Variable.import (back again cf. ed7aa5a350ef -- Alice is no longer supported);
 wenzelm parents: 
31696diff
changeset | 74 | val ((_, [thm']), _) = Variable.import true [thm] empty_ctxt; | 
| 45431 | 75 | val const_eq_morph = | 
| 76 | (case eq_morph of | |
| 46856 | 77 | SOME eq_morph => const_morph $> eq_morph | 
| 45431 | 78 | | NONE => const_morph); | 
| 36674 
d95f39448121
eq_morphism is always optional: avoid trivial morphism for empty list of equations
 haftmann parents: 
36672diff
changeset | 79 | val thm'' = Morphism.thm const_eq_morph thm'; | 
| 54742 
7a86358a3c0b
proper context for basic Simplifier operations: rewrite_rule, rewrite_goals_rule, rewrite_goals_tac etc.;
 wenzelm parents: 
54740diff
changeset | 80 | in | 
| 
7a86358a3c0b
proper context for basic Simplifier operations: rewrite_rule, rewrite_goals_rule, rewrite_goals_tac etc.;
 wenzelm parents: 
54740diff
changeset | 81 | Goal.prove_sorry_global thy [] [] (Thm.prop_of thm'') | 
| 
7a86358a3c0b
proper context for basic Simplifier operations: rewrite_rule, rewrite_goals_rule, rewrite_goals_tac etc.;
 wenzelm parents: 
54740diff
changeset | 82 |           (fn {context = ctxt, ...} => ALLGOALS (Proof_Context.fact_tac ctxt [thm'']))
 | 
| 
7a86358a3c0b
proper context for basic Simplifier operations: rewrite_rule, rewrite_goals_rule, rewrite_goals_tac etc.;
 wenzelm parents: 
54740diff
changeset | 83 | end; | 
| 52636 | 84 | val some_assm_intro = Option.map prove_assm_intro (fst (Locale.intros_of thy class)); | 
| 29547 | 85 | |
| 86 | (* of_class *) | |
| 31943 
5e960a0780a2
renamed inclass/Inclass to of_class/OfClass, in accordance to of_sort;
 wenzelm parents: 
31904diff
changeset | 87 | val of_class_prop_concl = Logic.mk_of_class (aT, class); | 
| 45431 | 88 | val of_class_prop = | 
| 52636 | 89 | (case some_prop of | 
| 45431 | 90 | NONE => of_class_prop_concl | 
| 29627 | 91 | | SOME prop => Logic.mk_implies (Morphism.term const_morph | 
| 45431 | 92 | ((map_types o map_atyps) (K aT) prop), of_class_prop_concl)); | 
| 38379 
67d71449e85b
more convenient split of class modules: class and class_declaration
 haftmann parents: 
38376diff
changeset | 93 | val sup_of_classes = map (snd o Class.rules thy) sups; | 
| 35021 
c839a4c670c6
renamed old-style Drule.standard to Drule.export_without_context, to emphasize that this is in no way a standard operation;
 wenzelm parents: 
33671diff
changeset | 94 | val loc_axiom_intros = map Drule.export_without_context_open (Locale.axioms_of thy class); | 
| 51685 
385ef6706252
more standard module name Axclass (according to file name);
 wenzelm parents: 
51551diff
changeset | 95 | val axclass_intro = #intro (Axclass.get_info thy class); | 
| 59621 
291934bac95e
Thm.cterm_of and Thm.ctyp_of operate on local context;
 wenzelm parents: 
59498diff
changeset | 96 | val base_sort_trivs = Thm.of_sort (Thm.global_ctyp_of thy aT, base_sort); | 
| 58957 | 97 | fun tac ctxt = | 
| 45431 | 98 | REPEAT (SOMEGOAL | 
| 58957 | 99 | (match_tac ctxt (axclass_intro :: sup_of_classes @ loc_axiom_intros @ base_sort_trivs) | 
| 58963 
26bf09b95dda
proper context for assume_tac (atac remains as fall-back without context);
 wenzelm parents: 
58957diff
changeset | 100 | ORELSE' assume_tac ctxt)); | 
| 58957 | 101 | val of_class = Goal.prove_sorry_global thy [] [] of_class_prop (tac o #context); | 
| 29547 | 102 | |
| 52636 | 103 | in (base_morph, eq_morph, export_morph, some_axiom, some_assm_intro, of_class) end; | 
| 29547 | 104 | |
| 29632 
c3d576157244
fixed reading of class specs: declare class operations in context
 haftmann parents: 
29627diff
changeset | 105 | |
| 29665 
2b956243d123
explicit check for exactly one type variable in class specification elements
 haftmann parents: 
29632diff
changeset | 106 | (* reading and processing class specifications *) | 
| 
2b956243d123
explicit check for exactly one type variable in class specification elements
 haftmann parents: 
29632diff
changeset | 107 | |
| 36460 | 108 | fun prep_class_elems prep_decl thy sups raw_elems = | 
| 29632 
c3d576157244
fixed reading of class specs: declare class operations in context
 haftmann parents: 
29627diff
changeset | 109 | let | 
| 29665 
2b956243d123
explicit check for exactly one type variable in class specification elements
 haftmann parents: 
29632diff
changeset | 110 | (* user space type system: only permits 'a type variable, improves towards 'a *) | 
| 36460 | 111 | val algebra = Sign.classes_of thy; | 
| 112 | val inter_sort = curry (Sorts.inter_sort algebra); | |
| 45421 | 113 | val proto_base_sort = | 
| 114 | if null sups then Sign.defaultS thy | |
| 38379 
67d71449e85b
more convenient split of class modules: class and class_declaration
 haftmann parents: 
38376diff
changeset | 115 | else fold inter_sort (map (Class.base_sort thy) sups) []; | 
| 58294 
7f990b3d5189
explicit check phase to guide type inference of class expression towards one single type variable
 haftmann parents: 
58293diff
changeset | 116 | val is_param = member (op =) (map fst (Class.these_params thy sups)); | 
| 29665 
2b956243d123
explicit check for exactly one type variable in class specification elements
 haftmann parents: 
29632diff
changeset | 117 | val base_constraints = (map o apsnd) | 
| 60346 | 118 | (map_type_tfree (K (TVar ((Name.aT, 0), proto_base_sort))) o fst o fst o snd) | 
| 38379 
67d71449e85b
more convenient split of class modules: class and class_declaration
 haftmann parents: 
38376diff
changeset | 119 | (Class.these_operations thy sups); | 
| 62952 | 120 | val singleton_fixate = burrow_types (fn Ts => | 
| 29665 
2b956243d123
explicit check for exactly one type variable in class specification elements
 haftmann parents: 
29632diff
changeset | 121 | let | 
| 58293 | 122 | val tfrees = fold Term.add_tfreesT Ts []; | 
| 45433 
4283f3a57cf5
avoid separate typ_check phases, integrate into main term_check 0 instead (cf. its Syntax.check_typs in Type_Infer_Context.prepare);
 wenzelm parents: 
45432diff
changeset | 123 | val inferred_sort = | 
| 58293 | 124 | (fold o fold_atyps) (fn TVar (_, S) => inter_sort S | _ => I) Ts []; | 
| 45421 | 125 | val fixate_sort = | 
| 45432 
12cc89f1eb0c
clarified singleton_fixate: intersection with supersort is identity, only replace actual type inference parameters;
 wenzelm parents: 
45431diff
changeset | 126 | (case tfrees of | 
| 
12cc89f1eb0c
clarified singleton_fixate: intersection with supersort is identity, only replace actual type inference parameters;
 wenzelm parents: 
45431diff
changeset | 127 | [] => inferred_sort | 
| 45433 
4283f3a57cf5
avoid separate typ_check phases, integrate into main term_check 0 instead (cf. its Syntax.check_typs in Type_Infer_Context.prepare);
 wenzelm parents: 
45432diff
changeset | 128 | | [(a, S)] => | 
| 
4283f3a57cf5
avoid separate typ_check phases, integrate into main term_check 0 instead (cf. its Syntax.check_typs in Type_Infer_Context.prepare);
 wenzelm parents: 
45432diff
changeset | 129 | if a <> Name.aT then | 
| 
4283f3a57cf5
avoid separate typ_check phases, integrate into main term_check 0 instead (cf. its Syntax.check_typs in Type_Infer_Context.prepare);
 wenzelm parents: 
45432diff
changeset | 130 |                 error ("No type variable other than " ^ Name.aT ^ " allowed in class specification")
 | 
| 
4283f3a57cf5
avoid separate typ_check phases, integrate into main term_check 0 instead (cf. its Syntax.check_typs in Type_Infer_Context.prepare);
 wenzelm parents: 
45432diff
changeset | 131 | else if Sorts.sort_le algebra (S, inferred_sort) then S | 
| 45432 
12cc89f1eb0c
clarified singleton_fixate: intersection with supersort is identity, only replace actual type inference parameters;
 wenzelm parents: 
45431diff
changeset | 132 | else | 
| 
12cc89f1eb0c
clarified singleton_fixate: intersection with supersort is identity, only replace actual type inference parameters;
 wenzelm parents: 
45431diff
changeset | 133 |                 error ("Type inference imposes additional sort constraint " ^
 | 
| 
12cc89f1eb0c
clarified singleton_fixate: intersection with supersort is identity, only replace actual type inference parameters;
 wenzelm parents: 
45431diff
changeset | 134 | Syntax.string_of_sort_global thy inferred_sort ^ | 
| 
12cc89f1eb0c
clarified singleton_fixate: intersection with supersort is identity, only replace actual type inference parameters;
 wenzelm parents: 
45431diff
changeset | 135 | " of type parameter " ^ Name.aT ^ " of sort " ^ | 
| 
12cc89f1eb0c
clarified singleton_fixate: intersection with supersort is identity, only replace actual type inference parameters;
 wenzelm parents: 
45431diff
changeset | 136 | Syntax.string_of_sort_global thy S) | 
| 
12cc89f1eb0c
clarified singleton_fixate: intersection with supersort is identity, only replace actual type inference parameters;
 wenzelm parents: 
45431diff
changeset | 137 | | _ => error "Multiple type variables in class specification"); | 
| 
12cc89f1eb0c
clarified singleton_fixate: intersection with supersort is identity, only replace actual type inference parameters;
 wenzelm parents: 
45431diff
changeset | 138 | val fixateT = TFree (Name.aT, fixate_sort); | 
| 
12cc89f1eb0c
clarified singleton_fixate: intersection with supersort is identity, only replace actual type inference parameters;
 wenzelm parents: 
45431diff
changeset | 139 | in | 
| 58293 | 140 | (map o map_atyps) | 
| 141 | (fn T as TVar (xi, _) => if Type_Infer.is_param xi then fixateT else T | T => T) Ts | |
| 62952 | 142 | end); | 
| 143 | fun unify_params ts = | |
| 40188 
eddda8e38360
consider base sorts of superclasses simultaneously during processing of class specification -- avoids clash of different base sorts
 haftmann parents: 
38875diff
changeset | 144 | let | 
| 58294 
7f990b3d5189
explicit check phase to guide type inference of class expression towards one single type variable
 haftmann parents: 
58293diff
changeset | 145 | val param_Ts = (fold o fold_aterms) | 
| 
7f990b3d5189
explicit check phase to guide type inference of class expression towards one single type variable
 haftmann parents: 
58293diff
changeset | 146 | (fn Free (v, T) => if is_param v then fold_atyps (insert (op =)) T else I | _ => I) ts []; | 
| 58319 | 147 | val param_namesT = map_filter (try (fst o dest_TVar)) param_Ts; | 
| 148 | val param_T = if null param_namesT then NONE | |
| 58294 
7f990b3d5189
explicit check phase to guide type inference of class expression towards one single type variable
 haftmann parents: 
58293diff
changeset | 149 | else SOME (case get_first (try dest_TFree) param_Ts of | 
| 
7f990b3d5189
explicit check phase to guide type inference of class expression towards one single type variable
 haftmann parents: 
58293diff
changeset | 150 | SOME v_sort => TFree v_sort | | 
| 58319 | 151 | NONE => TVar (hd param_namesT, proto_base_sort)); | 
| 58294 
7f990b3d5189
explicit check phase to guide type inference of class expression towards one single type variable
 haftmann parents: 
58293diff
changeset | 152 | in case param_T of | 
| 
7f990b3d5189
explicit check phase to guide type inference of class expression towards one single type variable
 haftmann parents: 
58293diff
changeset | 153 | NONE => ts | | 
| 58319 | 154 | SOME T => map (subst_TVars (map (rpair T) param_namesT)) ts | 
| 40188 
eddda8e38360
consider base sorts of superclasses simultaneously during processing of class specification -- avoids clash of different base sorts
 haftmann parents: 
38875diff
changeset | 155 | end; | 
| 29632 
c3d576157244
fixed reading of class specs: declare class operations in context
 haftmann parents: 
29627diff
changeset | 156 | |
| 35120 | 157 | (* preprocessing elements, retrieving base sort from type-checked elements *) | 
| 42402 
c7139609b67d
simplified check/uncheck interfaces: result comparison is hardwired by default;
 wenzelm parents: 
42375diff
changeset | 158 | val raw_supexpr = | 
| 
c7139609b67d
simplified check/uncheck interfaces: result comparison is hardwired by default;
 wenzelm parents: 
42375diff
changeset | 159 |       (map (fn sup => (sup, (("", false), Expression.Positional []))) sups, []);
 | 
| 
c7139609b67d
simplified check/uncheck interfaces: result comparison is hardwired by default;
 wenzelm parents: 
42375diff
changeset | 160 | val init_class_body = | 
| 
c7139609b67d
simplified check/uncheck interfaces: result comparison is hardwired by default;
 wenzelm parents: 
42375diff
changeset | 161 | fold (Proof_Context.add_const_constraint o apsnd SOME) base_constraints | 
| 38379 
67d71449e85b
more convenient split of class modules: class and class_declaration
 haftmann parents: 
38376diff
changeset | 162 | #> Class.redeclare_operations thy sups | 
| 62952 | 163 | #> Context.proof_map (Syntax_Phases.term_check 0 "singleton_fixate" (K singleton_fixate)); | 
| 47311 
1addbe2a7458
close context elements via Expression.cert/read_declaration;
 wenzelm parents: 
46922diff
changeset | 164 | val ((raw_supparams, _, raw_inferred_elems, _), _) = | 
| 42402 
c7139609b67d
simplified check/uncheck interfaces: result comparison is hardwired by default;
 wenzelm parents: 
42375diff
changeset | 165 | Proof_Context.init_global thy | 
| 62952 | 166 | |> Context.proof_map (Syntax_Phases.term_check 0 "unify_params" (K unify_params)) | 
| 32206 | 167 | |> prep_decl raw_supexpr init_class_body raw_elems; | 
| 38435 | 168 | fun filter_element (Element.Fixes []) = NONE | 
| 169 | | filter_element (e as Element.Fixes _) = SOME e | |
| 170 | | filter_element (Element.Constrains []) = NONE | |
| 171 | | filter_element (e as Element.Constrains _) = SOME e | |
| 172 | | filter_element (Element.Assumes []) = NONE | |
| 173 | | filter_element (e as Element.Assumes _) = SOME e | |
| 45421 | 174 | | filter_element (Element.Defines _) = | 
| 175 |           error ("\"defines\" element not allowed in class specification.")
 | |
| 176 | | filter_element (Element.Notes _) = | |
| 177 |           error ("\"notes\" element not allowed in class specification.");
 | |
| 38435 | 178 | val inferred_elems = map_filter filter_element raw_inferred_elems; | 
| 29665 
2b956243d123
explicit check for exactly one type variable in class specification elements
 haftmann parents: 
29632diff
changeset | 179 | fun fold_element_types f (Element.Fixes fxs) = fold (fn (_, SOME T, _) => f T) fxs | 
| 
2b956243d123
explicit check for exactly one type variable in class specification elements
 haftmann parents: 
29632diff
changeset | 180 | | fold_element_types f (Element.Constrains cnstrs) = fold (f o snd) cnstrs | 
| 
2b956243d123
explicit check for exactly one type variable in class specification elements
 haftmann parents: 
29632diff
changeset | 181 | | fold_element_types f (Element.Assumes assms) = fold (fold (fn (t, ts) => | 
| 42402 
c7139609b67d
simplified check/uncheck interfaces: result comparison is hardwired by default;
 wenzelm parents: 
42375diff
changeset | 182 | fold_types f t #> (fold o fold_types) f ts) o snd) assms; | 
| 45421 | 183 | val base_sort = | 
| 184 | if null inferred_elems then proto_base_sort | |
| 185 | else | |
| 186 | (case (fold o fold_element_types) Term.add_tfreesT inferred_elems [] of | |
| 187 | [] => error "No type variable in class specification" | |
| 29665 
2b956243d123
explicit check for exactly one type variable in class specification elements
 haftmann parents: 
29632diff
changeset | 188 | | [(_, sort)] => sort | 
| 45421 | 189 | | _ => error "Multiple type variables in class specification"); | 
| 32206 | 190 | val supparams = map (fn ((c, T), _) => | 
| 191 | (c, map_atyps (K (TFree (Name.aT, base_sort))) T)) raw_supparams; | |
| 192 | val supparam_names = map fst supparams; | |
| 193 | fun mk_param ((c, _), _) = Free (c, (the o AList.lookup (op =) supparams) c); | |
| 194 |     val supexpr = (map (fn sup => (sup, (("", false),
 | |
| 195 | Expression.Positional (map (SOME o mk_param) (Locale.params_of thy sup))))) sups, | |
| 196 | map (fn (c, T) => (Binding.name c, SOME T, NoSyn)) supparams); | |
| 29575 
41d604e59e93
improved and corrected reading of class specs -- still draft version
 haftmann parents: 
29558diff
changeset | 197 | |
| 32206 | 198 | in (base_sort, supparam_names, supexpr, inferred_elems) end; | 
| 29575 
41d604e59e93
improved and corrected reading of class specs -- still draft version
 haftmann parents: 
29558diff
changeset | 199 | |
| 29665 
2b956243d123
explicit check for exactly one type variable in class specification elements
 haftmann parents: 
29632diff
changeset | 200 | val cert_class_elems = prep_class_elems Expression.cert_declaration; | 
| 
2b956243d123
explicit check for exactly one type variable in class specification elements
 haftmann parents: 
29632diff
changeset | 201 | val read_class_elems = prep_class_elems Expression.cert_read_declaration; | 
| 29575 
41d604e59e93
improved and corrected reading of class specs -- still draft version
 haftmann parents: 
29558diff
changeset | 202 | |
| 29665 
2b956243d123
explicit check for exactly one type variable in class specification elements
 haftmann parents: 
29632diff
changeset | 203 | fun prep_class_spec prep_class prep_class_elems thy raw_supclasses raw_elems = | 
| 29575 
41d604e59e93
improved and corrected reading of class specs -- still draft version
 haftmann parents: 
29558diff
changeset | 204 | let | 
| 46922 
3717f3878714
source positions for locale and class expressions;
 wenzelm parents: 
46856diff
changeset | 205 | val thy_ctxt = Proof_Context.init_global thy; | 
| 29665 
2b956243d123
explicit check for exactly one type variable in class specification elements
 haftmann parents: 
29632diff
changeset | 206 | |
| 29575 
41d604e59e93
improved and corrected reading of class specs -- still draft version
 haftmann parents: 
29558diff
changeset | 207 | (* prepare import *) | 
| 
41d604e59e93
improved and corrected reading of class specs -- still draft version
 haftmann parents: 
29558diff
changeset | 208 | val inter_sort = curry (Sorts.inter_sort (Sign.classes_of thy)); | 
| 46922 
3717f3878714
source positions for locale and class expressions;
 wenzelm parents: 
46856diff
changeset | 209 | val sups = Sign.minimize_sort thy (map (prep_class thy_ctxt) raw_supclasses); | 
| 45431 | 210 | val _ = | 
| 211 | (case filter_out (Class.is_class thy) sups of | |
| 212 | [] => () | |
| 213 |       | no_classes => error ("No (proper) classes: " ^ commas_quote no_classes));
 | |
| 38379 
67d71449e85b
more convenient split of class modules: class and class_declaration
 haftmann parents: 
38376diff
changeset | 214 | val raw_supparams = (map o apsnd) (snd o snd) (Class.these_params thy sups); | 
| 32206 | 215 | val raw_supparam_names = map fst raw_supparams; | 
| 45431 | 216 | val _ = | 
| 217 | if has_duplicates (op =) raw_supparam_names then | |
| 218 |         error ("Duplicate parameter(s) in superclasses: " ^
 | |
| 219 | (commas_quote (duplicates (op =) raw_supparam_names))) | |
| 29575 
41d604e59e93
improved and corrected reading of class specs -- still draft version
 haftmann parents: 
29558diff
changeset | 220 | else (); | 
| 
41d604e59e93
improved and corrected reading of class specs -- still draft version
 haftmann parents: 
29558diff
changeset | 221 | |
| 
41d604e59e93
improved and corrected reading of class specs -- still draft version
 haftmann parents: 
29558diff
changeset | 222 | (* infer types and base sort *) | 
| 45431 | 223 | val (base_sort, supparam_names, supexpr, inferred_elems) = prep_class_elems thy sups raw_elems; | 
| 32206 | 224 | val sup_sort = inter_sort base_sort sups; | 
| 29575 
41d604e59e93
improved and corrected reading of class specs -- still draft version
 haftmann parents: 
29558diff
changeset | 225 | |
| 
41d604e59e93
improved and corrected reading of class specs -- still draft version
 haftmann parents: 
29558diff
changeset | 226 | (* process elements as class specification *) | 
| 46922 
3717f3878714
source positions for locale and class expressions;
 wenzelm parents: 
46856diff
changeset | 227 | val class_ctxt = Class.begin sups base_sort thy_ctxt; | 
| 47311 
1addbe2a7458
close context elements via Expression.cert/read_declaration;
 wenzelm parents: 
46922diff
changeset | 228 | val ((_, _, syntax_elems, _), _) = class_ctxt | 
| 29702 | 229 | |> Expression.cert_declaration supexpr I inferred_elems; | 
| 45431 | 230 | fun check_vars e vs = | 
| 231 | if null vs then | |
| 232 |         error ("No type variable in part of specification element " ^
 | |
| 233 | Pretty.string_of (Pretty.chunks (Element.pretty_ctxt class_ctxt e))) | |
| 29665 
2b956243d123
explicit check for exactly one type variable in class specification elements
 haftmann parents: 
29632diff
changeset | 234 | else (); | 
| 
2b956243d123
explicit check for exactly one type variable in class specification elements
 haftmann parents: 
29632diff
changeset | 235 | fun check_element (e as Element.Fixes fxs) = | 
| 45431 | 236 | List.app (fn (_, SOME T, _) => check_vars e (Term.add_tfreesT T [])) fxs | 
| 29665 
2b956243d123
explicit check for exactly one type variable in class specification elements
 haftmann parents: 
29632diff
changeset | 237 | | check_element (e as Element.Assumes assms) = | 
| 45431 | 238 | List.app (fn (_, ts_pss) => | 
| 239 | List.app (fn (t, _) => check_vars e (Term.add_tfrees t [])) ts_pss) assms | |
| 240 | | check_element _ = (); | |
| 241 | val _ = List.app check_element syntax_elems; | |
| 29665 
2b956243d123
explicit check for exactly one type variable in class specification elements
 haftmann parents: 
29632diff
changeset | 242 | fun fork_syn (Element.Fixes xs) = | 
| 30344 
10a67c5ddddb
more uniform handling of binding in targets and derived elements;
 wenzelm parents: 
30335diff
changeset | 243 | fold_map (fn (c, ty, syn) => cons (c, syn) #> pair (c, ty, NoSyn)) xs | 
| 29665 
2b956243d123
explicit check for exactly one type variable in class specification elements
 haftmann parents: 
29632diff
changeset | 244 | #>> Element.Fixes | 
| 
2b956243d123
explicit check for exactly one type variable in class specification elements
 haftmann parents: 
29632diff
changeset | 245 | | fork_syn x = pair x; | 
| 29575 
41d604e59e93
improved and corrected reading of class specs -- still draft version
 haftmann parents: 
29558diff
changeset | 246 | val (elems, global_syntax) = fold_map fork_syn syntax_elems []; | 
| 29665 
2b956243d123
explicit check for exactly one type variable in class specification elements
 haftmann parents: 
29632diff
changeset | 247 | |
| 32713 | 248 | in (((sups, supparam_names), (sup_sort, base_sort, supexpr)), (elems, global_syntax)) end; | 
| 29575 
41d604e59e93
improved and corrected reading of class specs -- still draft version
 haftmann parents: 
29558diff
changeset | 249 | |
| 29665 
2b956243d123
explicit check for exactly one type variable in class specification elements
 haftmann parents: 
29632diff
changeset | 250 | val cert_class_spec = prep_class_spec (K I) cert_class_elems; | 
| 46922 
3717f3878714
source positions for locale and class expressions;
 wenzelm parents: 
46856diff
changeset | 251 | val read_class_spec = prep_class_spec Proof_Context.read_class read_class_elems; | 
| 29665 
2b956243d123
explicit check for exactly one type variable in class specification elements
 haftmann parents: 
29632diff
changeset | 252 | |
| 
2b956243d123
explicit check for exactly one type variable in class specification elements
 haftmann parents: 
29632diff
changeset | 253 | |
| 
2b956243d123
explicit check for exactly one type variable in class specification elements
 haftmann parents: 
29632diff
changeset | 254 | (* class establishment *) | 
| 29575 
41d604e59e93
improved and corrected reading of class specs -- still draft version
 haftmann parents: 
29558diff
changeset | 255 | |
| 32206 | 256 | fun add_consts class base_sort sups supparam_names global_syntax thy = | 
| 24968 
f9bafc868847
replaced Sign.add_consts_authentic by Sign.declare_const;
 wenzelm parents: 
24949diff
changeset | 257 | let | 
| 29816 | 258 | (*FIXME simplify*) | 
| 32206 | 259 | val supconsts = supparam_names | 
| 38379 
67d71449e85b
more convenient split of class modules: class and class_declaration
 haftmann parents: 
38376diff
changeset | 260 | |> AList.make (snd o the o AList.lookup (op =) (Class.these_params thy sups)) | 
| 25683 | 261 | |> (map o apsnd o apsnd o map_atyps o K o TFree) (Name.aT, [class]); | 
| 29509 
1ff0f3f08a7b
migrated class package to new locale implementation
 haftmann parents: 
29439diff
changeset | 262 | val all_params = Locale.params_of thy class; | 
| 32206 | 263 | val raw_params = (snd o chop (length supparam_names)) all_params; | 
| 30755 
7ef503d216c2
simplified internal locale parameters: maintain proper name and type, instead of binding and constraint;
 wenzelm parents: 
30585diff
changeset | 264 | fun add_const ((raw_c, raw_ty), _) thy = | 
| 25683 | 265 | let | 
| 30755 
7ef503d216c2
simplified internal locale parameters: maintain proper name and type, instead of binding and constraint;
 wenzelm parents: 
30585diff
changeset | 266 | val b = Binding.name raw_c; | 
| 30344 
10a67c5ddddb
more uniform handling of binding in targets and derived elements;
 wenzelm parents: 
30335diff
changeset | 267 | val c = Sign.full_name thy b; | 
| 25683 | 268 | val ty = map_atyps (K (TFree (Name.aT, base_sort))) raw_ty; | 
| 269 | val ty0 = Type.strip_sorts ty; | |
| 270 | val ty' = map_atyps (K (TFree (Name.aT, [class]))) ty0; | |
| 30344 
10a67c5ddddb
more uniform handling of binding in targets and derived elements;
 wenzelm parents: 
30335diff
changeset | 271 | val syn = (the_default NoSyn o AList.lookup Binding.eq_name global_syntax) b; | 
| 25683 | 272 | in | 
| 273 | thy | |
| 42375 
774df7c59508
report Name_Space.declare/define, relatively to context;
 wenzelm parents: 
42360diff
changeset | 274 | |> Sign.declare_const_global ((b, ty0), syn) | 
| 25683 | 275 | |> snd | 
| 42494 | 276 | |> pair ((Variable.check_name b, ty), (c, ty')) | 
| 25683 | 277 | end; | 
| 28715 
238f9966c80e
class morphism stemming from locale interpretation
 haftmann parents: 
28674diff
changeset | 278 | in | 
| 
238f9966c80e
class morphism stemming from locale interpretation
 haftmann parents: 
28674diff
changeset | 279 | thy | 
| 38379 
67d71449e85b
more convenient split of class modules: class and class_declaration
 haftmann parents: 
38376diff
changeset | 280 | |> Sign.add_path (Class.class_prefix class) | 
| 28715 
238f9966c80e
class morphism stemming from locale interpretation
 haftmann parents: 
28674diff
changeset | 281 | |> fold_map add_const raw_params | 
| 
238f9966c80e
class morphism stemming from locale interpretation
 haftmann parents: 
28674diff
changeset | 282 | ||> Sign.restore_naming thy | 
| 
238f9966c80e
class morphism stemming from locale interpretation
 haftmann parents: 
28674diff
changeset | 283 | |-> (fn params => pair (supconsts @ (map o apfst) fst params, params)) | 
| 
238f9966c80e
class morphism stemming from locale interpretation
 haftmann parents: 
28674diff
changeset | 284 | end; | 
| 
238f9966c80e
class morphism stemming from locale interpretation
 haftmann parents: 
28674diff
changeset | 285 | |
| 32206 | 286 | fun adjungate_axclass bname class base_sort sups supsort supparam_names global_syntax thy = | 
| 28715 
238f9966c80e
class morphism stemming from locale interpretation
 haftmann parents: 
28674diff
changeset | 287 | let | 
| 29816 | 288 | (*FIXME simplify*) | 
| 25683 | 289 | fun globalize param_map = map_aterms | 
| 290 | (fn Free (v, ty) => Const ((fst o the o AList.lookup (op =) param_map) v, ty) | |
| 291 | | t => t); | |
| 29509 
1ff0f3f08a7b
migrated class package to new locale implementation
 haftmann parents: 
29439diff
changeset | 292 | val raw_pred = Locale.intros_of thy class | 
| 25683 | 293 | |> fst | 
| 35845 
e5980f0ad025
renamed varify/unvarify operations to varify_global/unvarify_global to emphasize that these only work in a global situation;
 wenzelm parents: 
35669diff
changeset | 294 | |> Option.map (Logic.unvarify_global o Logic.strip_imp_concl o Thm.prop_of); | 
| 45431 | 295 | fun get_axiom thy = | 
| 51685 
385ef6706252
more standard module name Axclass (according to file name);
 wenzelm parents: 
51551diff
changeset | 296 | (case #axioms (Axclass.get_info thy class) of | 
| 45431 | 297 | [] => NONE | 
| 298 | | [thm] => SOME thm); | |
| 24968 
f9bafc868847
replaced Sign.add_consts_authentic by Sign.declare_const;
 wenzelm parents: 
24949diff
changeset | 299 | in | 
| 
f9bafc868847
replaced Sign.add_consts_authentic by Sign.declare_const;
 wenzelm parents: 
24949diff
changeset | 300 | thy | 
| 63352 | 301 | |> add_consts class base_sort sups supparam_names global_syntax |-> (fn (param_map, params) => | 
| 302 | Axclass.define_class (bname, supsort) | |
| 303 | (map (fst o snd) params) | |
| 304 | [(Binding.empty_atts, Option.map (globalize param_map) raw_pred |> the_list)] | |
| 305 | #> snd | |
| 306 | #> `get_axiom | |
| 307 | #-> (fn assm_axiom => fold (Sign.add_const_constraint o apsnd SOME o snd) params | |
| 308 | #> pair (param_map, params, assm_axiom))) | |
| 24968 
f9bafc868847
replaced Sign.add_consts_authentic by Sign.declare_const;
 wenzelm parents: 
24949diff
changeset | 309 | end; | 
| 
f9bafc868847
replaced Sign.add_consts_authentic by Sign.declare_const;
 wenzelm parents: 
24949diff
changeset | 310 | |
| 57181 
2d13bf9ea77b
dropped obscure and unused ad-hoc before_exit hook for named targets
 haftmann parents: 
56921diff
changeset | 311 | fun gen_class prep_class_spec b raw_supclasses raw_elems thy = | 
| 24748 | 312 | let | 
| 36635 
080b755377c0
locale predicates of classes carry a mandatory "class" prefix
 haftmann parents: 
36464diff
changeset | 313 | val class = Sign.full_name thy b; | 
| 56921 
5bf71b4da706
note of_class rule for type classes in theory: useful to promote class instance proofs to locale interpretation proofs
 haftmann parents: 
54883diff
changeset | 314 | val prefix = Binding.qualify true "class"; | 
| 32206 | 315 | val (((sups, supparam_names), (supsort, base_sort, supexpr)), (elems, global_syntax)) = | 
| 316 | prep_class_spec thy raw_supclasses raw_elems; | |
| 24218 | 317 | in | 
| 318 | thy | |
| 57181 
2d13bf9ea77b
dropped obscure and unused ad-hoc before_exit hook for named targets
 haftmann parents: 
56921diff
changeset | 319 | |> Expression.add_locale b (prefix b) supexpr elems | 
| 33671 | 320 | |> snd |> Local_Theory.exit_global | 
| 36635 
080b755377c0
locale predicates of classes carry a mandatory "class" prefix
 haftmann parents: 
36464diff
changeset | 321 | |> adjungate_axclass b class base_sort sups supsort supparam_names global_syntax | 
| 29526 | 322 | |-> (fn (param_map, params, assm_axiom) => | 
| 29547 | 323 | `(fn thy => calculate thy class sups base_sort param_map assm_axiom) | 
| 52636 | 324 | #-> (fn (base_morph, eq_morph, export_morph, some_axiom, some_assm_intro, of_class) => | 
| 38107 | 325 | Context.theory_map (Locale.add_registration (class, base_morph) | 
| 326 | (Option.map (rpair true) eq_morph) export_morph) | |
| 56921 
5bf71b4da706
note of_class rule for type classes in theory: useful to promote class instance proofs to locale interpretation proofs
 haftmann parents: 
54883diff
changeset | 327 | #> Class.register class sups params base_sort base_morph export_morph some_axiom some_assm_intro of_class | 
| 
5bf71b4da706
note of_class rule for type classes in theory: useful to promote class instance proofs to locale interpretation proofs
 haftmann parents: 
54883diff
changeset | 328 | #> Global_Theory.store_thm (prefix (Binding.qualified_name (class ^ ".of_class.intro")), of_class))) | 
| 
5bf71b4da706
note of_class rule for type classes in theory: useful to promote class instance proofs to locale interpretation proofs
 haftmann parents: 
54883diff
changeset | 329 | |> snd | 
| 63402 | 330 | |> Named_Target.init NONE class | 
| 25038 | 331 | |> pair class | 
| 24218 | 332 | end; | 
| 333 | ||
| 334 | in | |
| 335 | ||
| 29509 
1ff0f3f08a7b
migrated class package to new locale implementation
 haftmann parents: 
29439diff
changeset | 336 | val class = gen_class cert_class_spec; | 
| 26518 | 337 | val class_cmd = gen_class read_class_spec; | 
| 24218 | 338 | |
| 339 | end; (*local*) | |
| 340 | ||
| 341 | ||
| 45421 | 342 | |
| 29358 | 343 | (** subclass relations **) | 
| 25462 | 344 | |
| 29358 | 345 | local | 
| 25462 | 346 | |
| 57181 
2d13bf9ea77b
dropped obscure and unused ad-hoc before_exit hook for named targets
 haftmann parents: 
56921diff
changeset | 347 | fun gen_subclass prep_class do_proof raw_sup lthy = | 
| 25462 | 348 | let | 
| 42360 | 349 | val thy = Proof_Context.theory_of lthy; | 
| 29558 | 350 | val proto_sup = prep_class thy raw_sup; | 
| 63268 | 351 | val proto_sub = | 
| 352 | (case Named_Target.class_of lthy of | |
| 57182 | 353 | SOME class => class | 
| 63268 | 354 | | NONE => error "Not in a class target"); | 
| 51685 
385ef6706252
more standard module name Axclass (according to file name);
 wenzelm parents: 
51551diff
changeset | 355 | val (sub, sup) = Axclass.cert_classrel thy (proto_sub, proto_sup); | 
| 29509 
1ff0f3f08a7b
migrated class package to new locale implementation
 haftmann parents: 
29439diff
changeset | 356 | |
| 
1ff0f3f08a7b
migrated class package to new locale implementation
 haftmann parents: 
29439diff
changeset | 357 |     val expr = ([(sup, (("", false), Expression.Positional []))], []);
 | 
| 29558 | 358 | val (([props], deps, export), goal_ctxt) = | 
| 29509 
1ff0f3f08a7b
migrated class package to new locale implementation
 haftmann parents: 
29439diff
changeset | 359 | Expression.cert_goal_expression expr lthy; | 
| 29526 | 360 | val some_prop = try the_single props; | 
| 29558 | 361 | val some_dep_morph = try the_single (map snd deps); | 
| 362 | fun after_qed some_wit = | |
| 54866 
7b9a67cbd48f
self-contained formulation of subclass command, avoiding hard-wired Named_Target.init
 haftmann parents: 
54742diff
changeset | 363 | Class.register_subclass (sub, sup) some_dep_morph some_wit export; | 
| 29558 | 364 | in do_proof after_qed some_prop goal_ctxt end; | 
| 25485 | 365 | |
| 29575 
41d604e59e93
improved and corrected reading of class specs -- still draft version
 haftmann parents: 
29558diff
changeset | 366 | fun user_proof after_qed some_prop = | 
| 
41d604e59e93
improved and corrected reading of class specs -- still draft version
 haftmann parents: 
29558diff
changeset | 367 | Element.witness_proof (after_qed o try the_single o the_single) | 
| 
41d604e59e93
improved and corrected reading of class specs -- still draft version
 haftmann parents: 
29558diff
changeset | 368 | [the_list some_prop]; | 
| 25485 | 369 | |
| 29575 
41d604e59e93
improved and corrected reading of class specs -- still draft version
 haftmann parents: 
29558diff
changeset | 370 | fun tactic_proof tac after_qed some_prop ctxt = | 
| 
41d604e59e93
improved and corrected reading of class specs -- still draft version
 haftmann parents: 
29558diff
changeset | 371 | after_qed (Option.map | 
| 
41d604e59e93
improved and corrected reading of class specs -- still draft version
 haftmann parents: 
29558diff
changeset | 372 | (fn prop => Element.prove_witness ctxt prop tac) some_prop) ctxt; | 
| 28666 | 373 | |
| 29358 | 374 | in | 
| 28666 | 375 | |
| 57181 
2d13bf9ea77b
dropped obscure and unused ad-hoc before_exit hook for named targets
 haftmann parents: 
56921diff
changeset | 376 | fun prove_subclass tac = gen_subclass (K I) (tactic_proof tac); | 
| 54882 | 377 | |
| 378 | fun subclass x = gen_subclass (K I) user_proof x; | |
| 379 | fun subclass_cmd x = | |
| 380 | gen_subclass (Proof_Context.read_class o Proof_Context.init_global) user_proof x; | |
| 25462 | 381 | |
| 29358 | 382 | end; (*local*) | 
| 383 | ||
| 24218 | 384 | end; |