| author | wenzelm | 
| Fri, 20 Sep 2024 19:51:08 +0200 | |
| changeset 80914 | d97fdabd9e2b | 
| parent 80636 | 4041e7c8059d | 
| child 81253 | bbed9f218158 | 
| permissions | -rw-r--r-- | 
| 53538 | 1 | (* Author: Alexander Krauss, TU Muenchen | 
| 2 | Author: Christian Sternagel, University of Innsbruck | |
| 37789 | 3 | |
| 52893 | 4 | Adhoc overloading of constants based on their types. | 
| 37789 | 5 | *) | 
| 6 | ||
| 7 | signature ADHOC_OVERLOADING = | |
| 8 | sig | |
| 52622 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 9 | val is_overloaded: Proof.context -> string -> bool | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 10 | val generic_add_overloaded: string -> Context.generic -> Context.generic | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 11 | val generic_remove_overloaded: string -> Context.generic -> Context.generic | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 12 | val generic_add_variant: string -> term -> Context.generic -> Context.generic | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 13 | (*If the list of variants is empty at the end of "generic_remove_variant", then | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 14 | "generic_remove_overloaded" is called implicitly.*) | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 15 | val generic_remove_variant: string -> term -> Context.generic -> Context.generic | 
| 45422 | 16 | val show_variants: bool Config.T | 
| 37789 | 17 | end | 
| 18 | ||
| 19 | structure Adhoc_Overloading: ADHOC_OVERLOADING = | |
| 20 | struct | |
| 21 | ||
| 69593 | 22 | val show_variants = Attrib.setup_config_bool \<^binding>\<open>show_variants\<close> (K false); | 
| 37789 | 23 | |
| 53538 | 24 | |
| 37789 | 25 | (* errors *) | 
| 26 | ||
| 53008 
128bec4e3fca
indicate error-functions more prominently (by name prefix instead of suffix);
 Christian Sternagel parents: 
53007diff
changeset | 27 | fun err_duplicate_variant oconst = | 
| 52622 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 28 |   error ("Duplicate variant of " ^ quote oconst);
 | 
| 37789 | 29 | |
| 53008 
128bec4e3fca
indicate error-functions more prominently (by name prefix instead of suffix);
 Christian Sternagel parents: 
53007diff
changeset | 30 | fun err_not_a_variant oconst = | 
| 52622 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 31 |   error ("Not a variant of " ^  quote oconst);
 | 
| 37789 | 32 | |
| 53008 
128bec4e3fca
indicate error-functions more prominently (by name prefix instead of suffix);
 Christian Sternagel parents: 
53007diff
changeset | 33 | fun err_not_overloaded oconst = | 
| 52622 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 34 |   error ("Constant " ^ quote oconst ^ " is not declared as overloaded");
 | 
| 37789 | 35 | |
| 53540 
7903fe2c271b
prefer explicit type constraint (again, see also Type.appl_error);
 wenzelm parents: 
53538diff
changeset | 36 | fun err_unresolved_overloading ctxt0 (c, T) t instances = | 
| 
7903fe2c271b
prefer explicit type constraint (again, see also Type.appl_error);
 wenzelm parents: 
53538diff
changeset | 37 | let | 
| 
7903fe2c271b
prefer explicit type constraint (again, see also Type.appl_error);
 wenzelm parents: 
53538diff
changeset | 38 | val ctxt = Config.put show_variants true ctxt0 | 
| 
7903fe2c271b
prefer explicit type constraint (again, see also Type.appl_error);
 wenzelm parents: 
53538diff
changeset | 39 | val const_space = Proof_Context.const_space ctxt | 
| 
7903fe2c271b
prefer explicit type constraint (again, see also Type.appl_error);
 wenzelm parents: 
53538diff
changeset | 40 | val prt_const = | 
| 
7903fe2c271b
prefer explicit type constraint (again, see also Type.appl_error);
 wenzelm parents: 
53538diff
changeset | 41 | Pretty.block [Name_Space.pretty ctxt const_space c, Pretty.str " ::", Pretty.brk 1, | 
| 
7903fe2c271b
prefer explicit type constraint (again, see also Type.appl_error);
 wenzelm parents: 
53538diff
changeset | 42 | Pretty.quote (Syntax.pretty_typ ctxt T)] | 
| 52688 
1e13b2515e2b
show variants in error messages; more precise error messages (give witnesses for multiple instances)
 Christian Sternagel parents: 
52687diff
changeset | 43 | in | 
| 53537 | 44 | error (Pretty.string_of (Pretty.chunks [ | 
| 45 | Pretty.block [ | |
| 46 | Pretty.str "Unresolved adhoc overloading of constant", Pretty.brk 1, | |
| 53540 
7903fe2c271b
prefer explicit type constraint (again, see also Type.appl_error);
 wenzelm parents: 
53538diff
changeset | 47 | prt_const, Pretty.brk 1, Pretty.str "in term", Pretty.brk 1, | 
| 
7903fe2c271b
prefer explicit type constraint (again, see also Type.appl_error);
 wenzelm parents: 
53538diff
changeset | 48 | Pretty.block [Pretty.quote (Syntax.pretty_term ctxt t)]], | 
| 53537 | 49 | Pretty.block ( | 
| 50 | (if null instances then [Pretty.str "no instances"] | |
| 51 | else Pretty.fbreaks ( | |
| 52 | Pretty.str "multiple instances:" :: | |
| 53540 
7903fe2c271b
prefer explicit type constraint (again, see also Type.appl_error);
 wenzelm parents: 
53538diff
changeset | 53 | map (Pretty.mark Markup.item o Syntax.pretty_term ctxt) instances)))])) | 
| 52688 
1e13b2515e2b
show variants in error messages; more precise error messages (give witnesses for multiple instances)
 Christian Sternagel parents: 
52687diff
changeset | 54 | end; | 
| 37789 | 55 | |
| 53538 | 56 | |
| 52622 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 57 | (* generic data *) | 
| 37789 | 58 | |
| 52622 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 59 | fun variants_eq ((v1, T1), (v2, T2)) = | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 60 | Term.aconv_untyped (v1, v2) andalso T1 = T2; | 
| 37789 | 61 | |
| 52622 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 62 | structure Overload_Data = Generic_Data | 
| 37789 | 63 | ( | 
| 64 | type T = | |
| 52622 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 65 |     {variants : (term * typ) list Symtab.table,
 | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 66 | oconsts : string Termtab.table}; | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 67 |   val empty = {variants = Symtab.empty, oconsts = Termtab.empty};
 | 
| 37789 | 68 | |
| 41472 
f6ab14e61604
misc tuning and comments based on review of Theory_Data, Proof_Data, Generic_Data usage;
 wenzelm parents: 
37818diff
changeset | 69 | fun merge | 
| 52622 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 70 |     ({variants = vtab1, oconsts = otab1},
 | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 71 |      {variants = vtab2, oconsts = otab2}) : T =
 | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 72 | let | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 73 | fun merge_oconsts _ (oconst1, oconst2) = | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 74 | if oconst1 = oconst2 then oconst1 | 
| 53008 
128bec4e3fca
indicate error-functions more prominently (by name prefix instead of suffix);
 Christian Sternagel parents: 
53007diff
changeset | 75 | else err_duplicate_variant oconst1; | 
| 52622 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 76 | in | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 77 |       {variants = Symtab.merge_list variants_eq (vtab1, vtab2),
 | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 78 | oconsts = Termtab.join merge_oconsts (otab1, otab2)} | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 79 | end; | 
| 37789 | 80 | ); | 
| 81 | ||
| 82 | fun map_tables f g = | |
| 52622 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 83 |   Overload_Data.map (fn {variants = vtab, oconsts = otab} =>
 | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 84 |     {variants = f vtab, oconsts = g otab});
 | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 85 | |
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 86 | val is_overloaded = Symtab.defined o #variants o Overload_Data.get o Context.Proof; | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 87 | val get_variants = Symtab.lookup o #variants o Overload_Data.get o Context.Proof; | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 88 | val get_overloaded = Termtab.lookup o #oconsts o Overload_Data.get o Context.Proof; | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 89 | |
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 90 | fun generic_add_overloaded oconst context = | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 91 | if is_overloaded (Context.proof_of context) oconst then context | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 92 | else map_tables (Symtab.update (oconst, [])) I context; | 
| 37789 | 93 | |
| 52622 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 94 | fun generic_remove_overloaded oconst context = | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 95 | let | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 96 | fun remove_oconst_and_variants context oconst = | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 97 | let | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 98 | val remove_variants = | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 99 | (case get_variants (Context.proof_of context) oconst of | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 100 | NONE => I | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 101 | | SOME vs => fold (Termtab.remove (op =) o rpair oconst o fst) vs); | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 102 | in map_tables (Symtab.delete_safe oconst) remove_variants context end; | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 103 | in | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 104 | if is_overloaded (Context.proof_of context) oconst then remove_oconst_and_variants context oconst | 
| 53008 
128bec4e3fca
indicate error-functions more prominently (by name prefix instead of suffix);
 Christian Sternagel parents: 
53007diff
changeset | 105 | else err_not_overloaded oconst | 
| 52622 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 106 | end; | 
| 37789 | 107 | |
| 52622 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 108 | local | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 109 | fun generic_variant add oconst t context = | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 110 | let | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 111 | val ctxt = Context.proof_of context; | 
| 53008 
128bec4e3fca
indicate error-functions more prominently (by name prefix instead of suffix);
 Christian Sternagel parents: 
53007diff
changeset | 112 | val _ = if is_overloaded ctxt oconst then () else err_not_overloaded oconst; | 
| 53005 
47db379a6cf9
move treatment of polymorphism to adhoc overloading command;
 Christian Sternagel parents: 
53004diff
changeset | 113 | val T = t |> fastype_of; | 
| 52622 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 114 | val t' = Term.map_types (K dummyT) t; | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 115 | in | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 116 | if add then | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 117 | let | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 118 | val _ = | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 119 | (case get_overloaded ctxt t' of | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 120 | NONE => () | 
| 53008 
128bec4e3fca
indicate error-functions more prominently (by name prefix instead of suffix);
 Christian Sternagel parents: 
53007diff
changeset | 121 | | SOME oconst' => err_duplicate_variant oconst'); | 
| 52622 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 122 | in | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 123 | map_tables (Symtab.cons_list (oconst, (t', T))) (Termtab.update (t', oconst)) context | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 124 | end | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 125 | else | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 126 | let | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 127 | val _ = | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 128 | if member variants_eq (the (get_variants ctxt oconst)) (t', T) then () | 
| 53008 
128bec4e3fca
indicate error-functions more prominently (by name prefix instead of suffix);
 Christian Sternagel parents: 
53007diff
changeset | 129 | else err_not_a_variant oconst; | 
| 52622 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 130 | in | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 131 | map_tables (Symtab.map_entry oconst (remove1 variants_eq (t', T))) | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 132 | (Termtab.delete_safe t') context | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 133 | |> (fn context => | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 134 | (case get_variants (Context.proof_of context) oconst of | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 135 | SOME [] => generic_remove_overloaded oconst context | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 136 | | _ => context)) | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 137 | end | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 138 | end; | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 139 | in | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 140 | val generic_add_variant = generic_variant true; | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 141 | val generic_remove_variant = generic_variant false; | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 142 | end; | 
| 37789 | 143 | |
| 53538 | 144 | |
| 37789 | 145 | (* check / uncheck *) | 
| 146 | ||
| 53004 | 147 | fun unifiable_with thy T1 T2 = | 
| 37789 | 148 | let | 
| 149 | val maxidx1 = Term.maxidx_of_typ T1; | |
| 150 | val T2' = Logic.incr_tvar (maxidx1 + 1) T2; | |
| 52622 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 151 | val maxidx2 = Term.maxidx_typ T2' maxidx1; | 
| 53004 | 152 | in can (Sign.typ_unify thy (T1, T2')) (Vartab.empty, maxidx2) end; | 
| 37789 | 153 | |
| 53006 
83d9984ee639
avoid misleading "instances" in function name;
 Christian Sternagel parents: 
53005diff
changeset | 154 | fun get_candidates ctxt (c, T) = | 
| 53007 | 155 | get_variants ctxt c | 
| 156 | |> Option.map (map_filter (fn (t, T') => | |
| 80127 
39f9084a9668
make adhoc_overloading respect type constraints
 Kevin Kappelmann <kevin.kappelmann@tum.de> parents: 
78095diff
changeset | 157 | if unifiable_with (Proof_Context.theory_of ctxt) T T' | 
| 
39f9084a9668
make adhoc_overloading respect type constraints
 Kevin Kappelmann <kevin.kappelmann@tum.de> parents: 
78095diff
changeset | 158 | (*keep the type constraint for the type-inference check phase*) | 
| 
39f9084a9668
make adhoc_overloading respect type constraints
 Kevin Kappelmann <kevin.kappelmann@tum.de> parents: 
78095diff
changeset | 159 | then SOME (Type.constraint T t) | 
| 53007 | 160 | else NONE)); | 
| 52687 | 161 | |
| 53007 | 162 | fun insert_variants ctxt t (oconst as Const (c, T)) = | 
| 53006 
83d9984ee639
avoid misleading "instances" in function name;
 Christian Sternagel parents: 
53005diff
changeset | 163 | (case get_candidates ctxt (c, T) of | 
| 53008 
128bec4e3fca
indicate error-functions more prominently (by name prefix instead of suffix);
 Christian Sternagel parents: 
53007diff
changeset | 164 | SOME [] => err_unresolved_overloading ctxt (c, T) t [] | 
| 53007 | 165 | | SOME [variant] => variant | 
| 166 | | _ => oconst) | |
| 167 | | insert_variants _ _ oconst = oconst; | |
| 37789 | 168 | |
| 54004 | 169 | fun insert_overloaded ctxt = | 
| 170 | let | |
| 171 | fun proc t = | |
| 172 | Term.map_types (K dummyT) t | |
| 173 | |> get_overloaded ctxt | |
| 174 | |> Option.map (Const o rpair (Term.type_of t)); | |
| 175 | in | |
| 55237 
1e341728bae9
prefer top-down rewriting for output (i.e. uncheck), in accordance to term abbreviations (see 5d2fe4e09354) and AST translations;
 wenzelm parents: 
54468diff
changeset | 176 | Pattern.rewrite_term_top (Proof_Context.theory_of ctxt) [] [proc] | 
| 54004 | 177 | end; | 
| 53007 | 178 | |
| 179 | fun check ctxt = | |
| 180 | map (fn t => Term.map_aterms (insert_variants ctxt t) t); | |
| 181 | ||
| 54468 
f6ffe53387ef
reintroduced e2d08b9c9047, lost in 54e290da6da8 + e13b0c88c798
 traytel parents: 
54004diff
changeset | 182 | fun uncheck ctxt ts = | 
| 
f6ffe53387ef
reintroduced e2d08b9c9047, lost in 54e290da6da8 + e13b0c88c798
 traytel parents: 
54004diff
changeset | 183 | if Config.get ctxt show_variants orelse exists (is_none o try Term.type_of) ts then ts | 
| 
f6ffe53387ef
reintroduced e2d08b9c9047, lost in 54e290da6da8 + e13b0c88c798
 traytel parents: 
54004diff
changeset | 184 | else map (insert_overloaded ctxt) ts; | 
| 53007 | 185 | |
| 186 | fun reject_unresolved ctxt = | |
| 52622 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 187 | let | 
| 53007 | 188 | val the_candidates = the o get_candidates ctxt; | 
| 37789 | 189 | fun check_unresolved t = | 
| 52622 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 190 | (case filter (is_overloaded ctxt o fst) (Term.add_consts t []) of | 
| 53007 | 191 | [] => t | 
| 53008 
128bec4e3fca
indicate error-functions more prominently (by name prefix instead of suffix);
 Christian Sternagel parents: 
53007diff
changeset | 192 | | (cT :: _) => err_unresolved_overloading ctxt cT t (the_candidates cT)); | 
| 53007 | 193 | in map check_unresolved end; | 
| 37789 | 194 | |
| 53538 | 195 | |
| 37789 | 196 | (* setup *) | 
| 197 | ||
| 52622 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 198 | val _ = Context.>> | 
| 53007 | 199 | (Syntax_Phases.term_check 0 "adhoc_overloading" check | 
| 200 | #> Syntax_Phases.term_check 1 "adhoc_overloading_unresolved_check" reject_unresolved | |
| 201 | #> Syntax_Phases.term_uncheck 0 "adhoc_overloading" uncheck); | |
| 37789 | 202 | |
| 53538 | 203 | |
| 52622 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 204 | (* commands *) | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 205 | |
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 206 | fun generic_adhoc_overloading_cmd add = | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 207 | if add then | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 208 | fold (fn (oconst, ts) => | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 209 | generic_add_overloaded oconst | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 210 | #> fold (generic_add_variant oconst) ts) | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 211 | else | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 212 | fold (fn (oconst, ts) => | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 213 | fold (generic_remove_variant oconst) ts); | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 214 | |
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 215 | fun adhoc_overloading_cmd' add args phi = | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 216 | let val args' = args | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 217 | |> map (apsnd (map_filter (fn t => | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 218 | let val t' = Morphism.term phi t; | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 219 | in if Term.aconv_untyped (t, t') then SOME t' else NONE end))); | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 220 | in generic_adhoc_overloading_cmd add args' end; | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 221 | |
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 222 | fun adhoc_overloading_cmd add raw_args lthy = | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 223 | let | 
| 55954 | 224 | fun const_name ctxt = | 
| 80636 
4041e7c8059d
tuned: more explicit dest_Const_name and dest_Const_type;
 wenzelm parents: 
80127diff
changeset | 225 |       dest_Const_name o Proof_Context.read_const {proper = false, strict = false} ctxt;  (* FIXME {proper = true, strict = true} (!?) *)
 | 
| 53005 
47db379a6cf9
move treatment of polymorphism to adhoc overloading command;
 Christian Sternagel parents: 
53004diff
changeset | 226 | fun read_term ctxt = singleton (Variable.polymorphic ctxt) o Syntax.read_term ctxt; | 
| 52622 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 227 | val args = | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 228 | raw_args | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 229 | |> map (apfst (const_name lthy)) | 
| 53005 
47db379a6cf9
move treatment of polymorphism to adhoc overloading command;
 Christian Sternagel parents: 
53004diff
changeset | 230 | |> map (apsnd (map (read_term lthy))); | 
| 52622 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 231 | in | 
| 78095 | 232 |     Local_Theory.declaration {syntax = true, pervasive = false, pos = Position.thread_data ()}
 | 
| 52622 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 233 | (adhoc_overloading_cmd' add args) lthy | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 234 | end; | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 235 | |
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 236 | val _ = | 
| 69593 | 237 | Outer_Syntax.local_theory \<^command_keyword>\<open>adhoc_overloading\<close> | 
| 52893 | 238 | "add adhoc overloading for constants / fixed variables" | 
| 52622 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 239 | (Parse.and_list1 (Parse.const -- Scan.repeat Parse.term) >> adhoc_overloading_cmd true); | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 240 | |
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 241 | val _ = | 
| 69593 | 242 | Outer_Syntax.local_theory \<^command_keyword>\<open>no_adhoc_overloading\<close> | 
| 59414 | 243 | "delete adhoc overloading for constants / fixed variables" | 
| 52622 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 244 | (Parse.and_list1 (Parse.const -- Scan.repeat Parse.term) >> adhoc_overloading_cmd false); | 
| 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 245 | |
| 45422 | 246 | end; | 
| 52622 
e0ff1625e96d
localized and modernized adhoc-overloading (patch by Christian Sternagel);
 wenzelm parents: 
50768diff
changeset | 247 |