author | boehmes |
Wed, 12 May 2010 23:53:59 +0200 | |
changeset 36895 | a96f9793d9c5 |
parent 36610 | bafd82950e24 |
child 37146 | f652333bbf8e |
permissions | -rw-r--r-- |
20894 | 1 |
(* Title: Pure/Isar/theory_target.ML |
2 |
Author: Makarius |
|
30437 | 3 |
Author: Florian Haftmann, TU Muenchen |
20894 | 4 |
|
25542 | 5 |
Common theory/locale/class/instantiation/overloading targets. |
20894 | 6 |
*) |
7 |
||
8 |
signature THEORY_TARGET = |
|
9 |
sig |
|
35205 | 10 |
val peek: local_theory -> |
11 |
{target: string, |
|
12 |
is_locale: bool, |
|
13 |
is_class: bool, |
|
14 |
instantiation: string list * (string * sort) list * sort, |
|
25864 | 15 |
overloading: (string * (string * typ) * bool) list} |
25269 | 16 |
val init: string option -> theory -> local_theory |
35205 | 17 |
val context_cmd: xstring -> theory -> local_theory |
25864 | 18 |
val instantiation: string list * (string * sort) list * sort -> theory -> local_theory |
29971 | 19 |
val instantiation_cmd: xstring list * xstring list * xstring -> theory -> local_theory |
25864 | 20 |
val overloading: (string * (string * typ) * bool) list -> theory -> local_theory |
26049
8186c03194ed
overloading: reduced code redundancy, no xstrings here;
wenzelm
parents:
25984
diff
changeset
|
21 |
val overloading_cmd: (string * string * bool) list -> theory -> local_theory |
20894 | 22 |
end; |
23 |
||
33553 | 24 |
structure Theory_Target: THEORY_TARGET = |
20894 | 25 |
struct |
26 |
||
21006 | 27 |
(* context data *) |
28 |
||
29576 | 29 |
datatype target = Target of {target: string, is_locale: bool, |
25864 | 30 |
is_class: bool, instantiation: string list * (string * sort) list * sort, |
31 |
overloading: (string * (string * typ) * bool) list}; |
|
25012
448af76a1ba3
pass explicit target record -- more informative peek operation;
wenzelm
parents:
25002
diff
changeset
|
32 |
|
29576 | 33 |
fun make_target target is_locale is_class instantiation overloading = |
34 |
Target {target = target, is_locale = is_locale, |
|
25519 | 35 |
is_class = is_class, instantiation = instantiation, overloading = overloading}; |
25291 | 36 |
|
29576 | 37 |
val global_target = make_target "" false false ([], [], []) []; |
25012
448af76a1ba3
pass explicit target record -- more informative peek operation;
wenzelm
parents:
25002
diff
changeset
|
38 |
|
33519 | 39 |
structure Data = Proof_Data |
21006 | 40 |
( |
25012
448af76a1ba3
pass explicit target record -- more informative peek operation;
wenzelm
parents:
25002
diff
changeset
|
41 |
type T = target; |
25291 | 42 |
fun init _ = global_target; |
21006 | 43 |
); |
44 |
||
25012
448af76a1ba3
pass explicit target record -- more informative peek operation;
wenzelm
parents:
25002
diff
changeset
|
45 |
val peek = (fn Target args => args) o Data.get; |
21006 | 46 |
|
47 |
||
20894 | 48 |
(* pretty *) |
49 |
||
32785 | 50 |
fun pretty_thy ctxt target is_class = |
20894 | 51 |
let |
52 |
val thy = ProofContext.theory_of ctxt; |
|
29576 | 53 |
val target_name = (if is_class then "class " else "locale ") ^ Locale.extern thy target; |
30437 | 54 |
val fixes = |
55 |
map (fn (x, T) => (Binding.name x, SOME T, NoSyn)) (#1 (ProofContext.inferred_fixes ctxt)); |
|
56 |
val assumes = |
|
30473
e0b66c11e7e4
Assumption.all_prems_of, Assumption.all_assms_of;
wenzelm
parents:
30438
diff
changeset
|
57 |
map (fn A => (Attrib.empty_binding, [(Thm.term_of A, [])])) (Assumption.all_assms_of ctxt); |
20894 | 58 |
val elems = |
59 |
(if null fixes then [] else [Element.Fixes fixes]) @ |
|
60 |
(if null assumes then [] else [Element.Assumes assumes]); |
|
26049
8186c03194ed
overloading: reduced code redundancy, no xstrings here;
wenzelm
parents:
25984
diff
changeset
|
61 |
in |
8186c03194ed
overloading: reduced code redundancy, no xstrings here;
wenzelm
parents:
25984
diff
changeset
|
62 |
if target = "" then [] |
25607 | 63 |
else if null elems then [Pretty.str target_name] |
64 |
else [Pretty.big_list (target_name ^ " =") |
|
65 |
(map (Pretty.chunks o Element.pretty_ctxt ctxt) elems)] |
|
20894 | 66 |
end; |
67 |
||
32785 | 68 |
fun pretty (Target {target, is_class, instantiation, overloading, ...}) ctxt = |
25607 | 69 |
Pretty.block [Pretty.str "theory", Pretty.brk 1, |
70 |
Pretty.str (Context.theory_name (ProofContext.theory_of ctxt))] :: |
|
71 |
(if not (null overloading) then [Overloading.pretty ctxt] |
|
29358 | 72 |
else if not (null (#1 instantiation)) then [Class_Target.pretty_instantiation ctxt] |
32785 | 73 |
else pretty_thy ctxt target is_class); |
25607 | 74 |
|
20894 | 75 |
|
33456
fbd47f9b9b12
allow "pervasive" local theory declarations, which are applied the background theory;
wenzelm
parents:
33282
diff
changeset
|
76 |
(* generic declarations *) |
fbd47f9b9b12
allow "pervasive" local theory declarations, which are applied the background theory;
wenzelm
parents:
33282
diff
changeset
|
77 |
|
fbd47f9b9b12
allow "pervasive" local theory declarations, which are applied the background theory;
wenzelm
parents:
33282
diff
changeset
|
78 |
local |
24838 | 79 |
|
33456
fbd47f9b9b12
allow "pervasive" local theory declarations, which are applied the background theory;
wenzelm
parents:
33282
diff
changeset
|
80 |
fun direct_decl decl = |
fbd47f9b9b12
allow "pervasive" local theory declarations, which are applied the background theory;
wenzelm
parents:
33282
diff
changeset
|
81 |
let val decl0 = Morphism.form decl in |
33671 | 82 |
Local_Theory.theory (Context.theory_map decl0) #> |
83 |
Local_Theory.target (Context.proof_map decl0) |
|
33456
fbd47f9b9b12
allow "pervasive" local theory declarations, which are applied the background theory;
wenzelm
parents:
33282
diff
changeset
|
84 |
end; |
fbd47f9b9b12
allow "pervasive" local theory declarations, which are applied the background theory;
wenzelm
parents:
33282
diff
changeset
|
85 |
|
fbd47f9b9b12
allow "pervasive" local theory declarations, which are applied the background theory;
wenzelm
parents:
33282
diff
changeset
|
86 |
fun target_decl add (Target {target, ...}) pervasive decl lthy = |
24838 | 87 |
let |
33671 | 88 |
val global_decl = Morphism.transform (Local_Theory.global_morphism lthy) decl; |
89 |
val target_decl = Morphism.transform (Local_Theory.target_morphism lthy) decl; |
|
24838 | 90 |
in |
25012
448af76a1ba3
pass explicit target record -- more informative peek operation;
wenzelm
parents:
25002
diff
changeset
|
91 |
if target = "" then |
24838 | 92 |
lthy |
35127
5b29c1660047
apply global morphism for theory, instantiation and overloading target; n.b. target morphism and global morphism coincide for theory target
haftmann
parents:
33764
diff
changeset
|
93 |
|> direct_decl global_decl |
24838 | 94 |
else |
95 |
lthy |
|
33456
fbd47f9b9b12
allow "pervasive" local theory declarations, which are applied the background theory;
wenzelm
parents:
33282
diff
changeset
|
96 |
|> pervasive ? direct_decl global_decl |
33671 | 97 |
|> Local_Theory.target (add target target_decl) |
24838 | 98 |
end; |
99 |
||
33456
fbd47f9b9b12
allow "pervasive" local theory declarations, which are applied the background theory;
wenzelm
parents:
33282
diff
changeset
|
100 |
in |
fbd47f9b9b12
allow "pervasive" local theory declarations, which are applied the background theory;
wenzelm
parents:
33282
diff
changeset
|
101 |
|
29576 | 102 |
val declaration = target_decl Locale.add_declaration; |
35798
fd1bb29f8170
replaced type_syntax/term_syntax by uniform syntax_declaration;
wenzelm
parents:
35765
diff
changeset
|
103 |
val syntax_declaration = target_decl Locale.add_syntax_declaration; |
24838 | 104 |
|
33456
fbd47f9b9b12
allow "pervasive" local theory declarations, which are applied the background theory;
wenzelm
parents:
33282
diff
changeset
|
105 |
end; |
fbd47f9b9b12
allow "pervasive" local theory declarations, which are applied the background theory;
wenzelm
parents:
33282
diff
changeset
|
106 |
|
25105
c9f67836c4d8
internal tuning: class_target, fork_mixfix, declare_const (singleton), abbrev;
wenzelm
parents:
25096
diff
changeset
|
107 |
fun class_target (Target {target, ...}) f = |
33671 | 108 |
Local_Theory.raw_theory f #> |
109 |
Local_Theory.target (Class_Target.refresh_syntax target); |
|
24838 | 110 |
|
21611
fc95ff1fe738
notes: proper import/export of proofs (still inactive);
wenzelm
parents:
21594
diff
changeset
|
111 |
|
20894 | 112 |
(* notes *) |
113 |
||
21611
fc95ff1fe738
notes: proper import/export of proofs (still inactive);
wenzelm
parents:
21594
diff
changeset
|
114 |
fun import_export_proof ctxt (name, raw_th) = |
21594
2859c94d67d4
reworked notes: towards proper import/export of proof terms;
wenzelm
parents:
21585
diff
changeset
|
115 |
let |
21611
fc95ff1fe738
notes: proper import/export of proofs (still inactive);
wenzelm
parents:
21594
diff
changeset
|
116 |
val thy = ProofContext.theory_of ctxt; |
36610
bafd82950e24
renamed ProofContext.init to ProofContext.init_global to emphasize that this is not the real thing;
wenzelm
parents:
36106
diff
changeset
|
117 |
val thy_ctxt = ProofContext.init_global thy; |
21611
fc95ff1fe738
notes: proper import/export of proofs (still inactive);
wenzelm
parents:
21594
diff
changeset
|
118 |
val certT = Thm.ctyp_of thy; |
fc95ff1fe738
notes: proper import/export of proofs (still inactive);
wenzelm
parents:
21594
diff
changeset
|
119 |
val cert = Thm.cterm_of thy; |
21594
2859c94d67d4
reworked notes: towards proper import/export of proof terms;
wenzelm
parents:
21585
diff
changeset
|
120 |
|
21611
fc95ff1fe738
notes: proper import/export of proofs (still inactive);
wenzelm
parents:
21594
diff
changeset
|
121 |
(*export assumes/defines*) |
fc95ff1fe738
notes: proper import/export of proofs (still inactive);
wenzelm
parents:
21594
diff
changeset
|
122 |
val th = Goal.norm_result raw_th; |
35624 | 123 |
val (defs, th') = Local_Defs.export ctxt thy_ctxt th; |
30473
e0b66c11e7e4
Assumption.all_prems_of, Assumption.all_assms_of;
wenzelm
parents:
30438
diff
changeset
|
124 |
val assms = map (MetaSimplifier.rewrite_rule defs o Thm.assume) (Assumption.all_assms_of ctxt); |
21611
fc95ff1fe738
notes: proper import/export of proofs (still inactive);
wenzelm
parents:
21594
diff
changeset
|
125 |
val nprems = Thm.nprems_of th' - Thm.nprems_of th; |
fc95ff1fe738
notes: proper import/export of proofs (still inactive);
wenzelm
parents:
21594
diff
changeset
|
126 |
|
fc95ff1fe738
notes: proper import/export of proofs (still inactive);
wenzelm
parents:
21594
diff
changeset
|
127 |
(*export fixes*) |
22692 | 128 |
val tfrees = map TFree (Thm.fold_terms Term.add_tfrees th' []); |
129 |
val frees = map Free (Thm.fold_terms Term.add_frees th' []); |
|
21611
fc95ff1fe738
notes: proper import/export of proofs (still inactive);
wenzelm
parents:
21594
diff
changeset
|
130 |
val (th'' :: vs) = (th' :: map (Drule.mk_term o cert) (map Logic.mk_type tfrees @ frees)) |
fc95ff1fe738
notes: proper import/export of proofs (still inactive);
wenzelm
parents:
21594
diff
changeset
|
131 |
|> Variable.export ctxt thy_ctxt |
fc95ff1fe738
notes: proper import/export of proofs (still inactive);
wenzelm
parents:
21594
diff
changeset
|
132 |
|> Drule.zero_var_indexes_list; |
fc95ff1fe738
notes: proper import/export of proofs (still inactive);
wenzelm
parents:
21594
diff
changeset
|
133 |
|
fc95ff1fe738
notes: proper import/export of proofs (still inactive);
wenzelm
parents:
21594
diff
changeset
|
134 |
(*thm definition*) |
33700 | 135 |
val result = PureThy.name_thm true true name th''; |
21611
fc95ff1fe738
notes: proper import/export of proofs (still inactive);
wenzelm
parents:
21594
diff
changeset
|
136 |
|
fc95ff1fe738
notes: proper import/export of proofs (still inactive);
wenzelm
parents:
21594
diff
changeset
|
137 |
(*import fixes*) |
fc95ff1fe738
notes: proper import/export of proofs (still inactive);
wenzelm
parents:
21594
diff
changeset
|
138 |
val (tvars, vars) = |
fc95ff1fe738
notes: proper import/export of proofs (still inactive);
wenzelm
parents:
21594
diff
changeset
|
139 |
chop (length tfrees) (map (Thm.term_of o Drule.dest_term) vs) |
fc95ff1fe738
notes: proper import/export of proofs (still inactive);
wenzelm
parents:
21594
diff
changeset
|
140 |
|>> map Logic.dest_type; |
fc95ff1fe738
notes: proper import/export of proofs (still inactive);
wenzelm
parents:
21594
diff
changeset
|
141 |
|
fc95ff1fe738
notes: proper import/export of proofs (still inactive);
wenzelm
parents:
21594
diff
changeset
|
142 |
val instT = map_filter (fn (TVar v, T) => SOME (v, T) | _ => NONE) (tvars ~~ tfrees); |
fc95ff1fe738
notes: proper import/export of proofs (still inactive);
wenzelm
parents:
21594
diff
changeset
|
143 |
val inst = filter (is_Var o fst) (vars ~~ frees); |
fc95ff1fe738
notes: proper import/export of proofs (still inactive);
wenzelm
parents:
21594
diff
changeset
|
144 |
val cinstT = map (pairself certT o apfst TVar) instT; |
31977 | 145 |
val cinst = map (pairself (cert o Term.map_types (Term_Subst.instantiateT instT))) inst; |
21611
fc95ff1fe738
notes: proper import/export of proofs (still inactive);
wenzelm
parents:
21594
diff
changeset
|
146 |
val result' = Thm.instantiate (cinstT, cinst) result; |
fc95ff1fe738
notes: proper import/export of proofs (still inactive);
wenzelm
parents:
21594
diff
changeset
|
147 |
|
fc95ff1fe738
notes: proper import/export of proofs (still inactive);
wenzelm
parents:
21594
diff
changeset
|
148 |
(*import assumes/defines*) |
21594
2859c94d67d4
reworked notes: towards proper import/export of proof terms;
wenzelm
parents:
21585
diff
changeset
|
149 |
val assm_tac = FIRST' (map (fn assm => Tactic.compose_tac (false, assm, 0)) assms); |
21611
fc95ff1fe738
notes: proper import/export of proofs (still inactive);
wenzelm
parents:
21594
diff
changeset
|
150 |
val result'' = |
fc95ff1fe738
notes: proper import/export of proofs (still inactive);
wenzelm
parents:
21594
diff
changeset
|
151 |
(case SINGLE (Seq.INTERVAL assm_tac 1 nprems) result' of |
fc95ff1fe738
notes: proper import/export of proofs (still inactive);
wenzelm
parents:
21594
diff
changeset
|
152 |
NONE => raise THM ("Failed to re-import result", 0, [result']) |
35739 | 153 |
| SOME res => Local_Defs.contract ctxt defs (Thm.cprop_of th) res) |
21644 | 154 |
|> Goal.norm_result |
33700 | 155 |
|> PureThy.name_thm false false name; |
21611
fc95ff1fe738
notes: proper import/export of proofs (still inactive);
wenzelm
parents:
21594
diff
changeset
|
156 |
|
fc95ff1fe738
notes: proper import/export of proofs (still inactive);
wenzelm
parents:
21594
diff
changeset
|
157 |
in (result'', result) end; |
fc95ff1fe738
notes: proper import/export of proofs (still inactive);
wenzelm
parents:
21594
diff
changeset
|
158 |
|
29576 | 159 |
fun notes (Target {target, is_locale, ...}) kind facts lthy = |
21585 | 160 |
let |
21594
2859c94d67d4
reworked notes: towards proper import/export of proof terms;
wenzelm
parents:
21585
diff
changeset
|
161 |
val thy = ProofContext.theory_of lthy; |
2859c94d67d4
reworked notes: towards proper import/export of proof terms;
wenzelm
parents:
21585
diff
changeset
|
162 |
val facts' = facts |
28991 | 163 |
|> map (fn (a, bs) => (a, PureThy.burrow_fact (PureThy.name_multi |
33671 | 164 |
(Local_Theory.full_name lthy (fst a))) bs)) |
21615
1bd558879c44
notes: proper naming of thm proof, activated import_export_proof;
wenzelm
parents:
21613
diff
changeset
|
165 |
|> PureThy.map_facts (import_export_proof lthy); |
21611
fc95ff1fe738
notes: proper import/export of proofs (still inactive);
wenzelm
parents:
21594
diff
changeset
|
166 |
val local_facts = PureThy.map_facts #1 facts' |
fc95ff1fe738
notes: proper import/export of proofs (still inactive);
wenzelm
parents:
21594
diff
changeset
|
167 |
|> Attrib.map_facts (Attrib.attribute_i thy); |
fc95ff1fe738
notes: proper import/export of proofs (still inactive);
wenzelm
parents:
21594
diff
changeset
|
168 |
val target_facts = PureThy.map_facts #1 facts' |
33671 | 169 |
|> is_locale ? Element.facts_map (Element.morph_ctxt (Local_Theory.target_morphism lthy)); |
21611
fc95ff1fe738
notes: proper import/export of proofs (still inactive);
wenzelm
parents:
21594
diff
changeset
|
170 |
val global_facts = PureThy.map_facts #2 facts' |
25012
448af76a1ba3
pass explicit target record -- more informative peek operation;
wenzelm
parents:
25002
diff
changeset
|
171 |
|> Attrib.map_facts (if is_locale then K I else Attrib.attribute_i thy); |
21594
2859c94d67d4
reworked notes: towards proper import/export of proof terms;
wenzelm
parents:
21585
diff
changeset
|
172 |
in |
33167 | 173 |
lthy |
33671 | 174 |
|> Local_Theory.theory (PureThy.note_thmss kind global_facts #> snd) |
175 |
|> not is_locale ? Local_Theory.target (ProofContext.note_thmss kind global_facts #> snd) |
|
176 |
|> is_locale ? Local_Theory.target (Locale.add_thmss target kind target_facts) |
|
30761
ac7570d80c3d
renamed ProofContext.note_thmss_i to ProofContext.note_thmss, eliminated obsolete external version;
wenzelm
parents:
30519
diff
changeset
|
177 |
|> ProofContext.note_thmss kind local_facts |
20894 | 178 |
end; |
179 |
||
180 |
||
35764 | 181 |
(* consts *) |
24939 | 182 |
|
25105
c9f67836c4d8
internal tuning: class_target, fork_mixfix, declare_const (singleton), abbrev;
wenzelm
parents:
25096
diff
changeset
|
183 |
fun fork_mixfix (Target {is_locale, is_class, ...}) mx = |
c9f67836c4d8
internal tuning: class_target, fork_mixfix, declare_const (singleton), abbrev;
wenzelm
parents:
25096
diff
changeset
|
184 |
if not is_locale then (NoSyn, NoSyn, mx) |
c9f67836c4d8
internal tuning: class_target, fork_mixfix, declare_const (singleton), abbrev;
wenzelm
parents:
25096
diff
changeset
|
185 |
else if not is_class then (NoSyn, mx, NoSyn) |
c9f67836c4d8
internal tuning: class_target, fork_mixfix, declare_const (singleton), abbrev;
wenzelm
parents:
25096
diff
changeset
|
186 |
else (mx, NoSyn, NoSyn); |
25068 | 187 |
|
33167 | 188 |
fun locale_const (Target {target, is_class, ...}) (prmode as (mode, _)) ((b, mx), rhs) phi = |
24939 | 189 |
let |
28965 | 190 |
val b' = Morphism.binding phi b; |
24939 | 191 |
val rhs' = Morphism.term phi rhs; |
28861 | 192 |
val arg = (b', Term.close_schematic_term rhs'); |
33537
06c87d2c5b5a
locale_const/target_notation: uniform use of Term.aconv_untyped;
wenzelm
parents:
33519
diff
changeset
|
193 |
val same_shape = Term.aconv_untyped (rhs, rhs'); |
25212
9dd61cb753ae
locale_const: in_class workaround prevents additional locale version of class consts;
wenzelm
parents:
25150
diff
changeset
|
194 |
(* FIXME workaround based on educated guess *) |
30278 | 195 |
val prefix' = Binding.prefix_of b'; |
33282 | 196 |
val class_global = |
197 |
Binding.eq_name (b, b') andalso |
|
198 |
not (null prefix') andalso |
|
199 |
fst (snd (split_last prefix')) = Class_Target.class_prefix target; |
|
24939 | 200 |
in |
33537
06c87d2c5b5a
locale_const/target_notation: uniform use of Term.aconv_untyped;
wenzelm
parents:
33519
diff
changeset
|
201 |
not (is_class andalso (same_shape orelse class_global)) ? |
25212
9dd61cb753ae
locale_const: in_class workaround prevents additional locale version of class consts;
wenzelm
parents:
25150
diff
changeset
|
202 |
(Context.mapping_result |
33173
b8ca12f6681a
eliminated obsolete tags for types/consts -- now handled via name space, in strongly typed fashion;
wenzelm
parents:
33167
diff
changeset
|
203 |
(Sign.add_abbrev PrintMode.internal arg) |
b8ca12f6681a
eliminated obsolete tags for types/consts -- now handled via name space, in strongly typed fashion;
wenzelm
parents:
33167
diff
changeset
|
204 |
(ProofContext.add_abbrev PrintMode.internal arg) |
25212
9dd61cb753ae
locale_const: in_class workaround prevents additional locale version of class consts;
wenzelm
parents:
25150
diff
changeset
|
205 |
#-> (fn (lhs' as Const (d, _), _) => |
33537
06c87d2c5b5a
locale_const/target_notation: uniform use of Term.aconv_untyped;
wenzelm
parents:
33519
diff
changeset
|
206 |
same_shape ? |
25212
9dd61cb753ae
locale_const: in_class workaround prevents additional locale version of class consts;
wenzelm
parents:
25150
diff
changeset
|
207 |
(Context.mapping (Sign.revert_abbrev mode d) (ProofContext.revert_abbrev mode d) #> |
9dd61cb753ae
locale_const: in_class workaround prevents additional locale version of class consts;
wenzelm
parents:
25150
diff
changeset
|
208 |
Morphism.form (ProofContext.target_notation true prmode [(lhs', mx)])))) |
24939 | 209 |
end; |
210 |
||
211 |
||
212 |
(* abbrev *) |
|
213 |
||
28083
103d9282a946
explicit type Name.binding for higher-specification elements;
wenzelm
parents:
27690
diff
changeset
|
214 |
fun abbrev (ta as Target {target, is_locale, is_class, ...}) prmode ((b, mx), t) lthy = |
24939 | 215 |
let |
36610
bafd82950e24
renamed ProofContext.init to ProofContext.init_global to emphasize that this is not the real thing;
wenzelm
parents:
36106
diff
changeset
|
216 |
val thy_ctxt = ProofContext.init_global (ProofContext.theory_of lthy); |
33671 | 217 |
val target_ctxt = Local_Theory.target_of lthy; |
25105
c9f67836c4d8
internal tuning: class_target, fork_mixfix, declare_const (singleton), abbrev;
wenzelm
parents:
25096
diff
changeset
|
218 |
|
c9f67836c4d8
internal tuning: class_target, fork_mixfix, declare_const (singleton), abbrev;
wenzelm
parents:
25096
diff
changeset
|
219 |
val (mx1, mx2, mx3) = fork_mixfix ta mx; |
c9f67836c4d8
internal tuning: class_target, fork_mixfix, declare_const (singleton), abbrev;
wenzelm
parents:
25096
diff
changeset
|
220 |
val t' = Assumption.export_term lthy target_ctxt t; |
c9f67836c4d8
internal tuning: class_target, fork_mixfix, declare_const (singleton), abbrev;
wenzelm
parents:
25096
diff
changeset
|
221 |
val xs = map Free (rev (Variable.add_fixed target_ctxt t' [])); |
c9f67836c4d8
internal tuning: class_target, fork_mixfix, declare_const (singleton), abbrev;
wenzelm
parents:
25096
diff
changeset
|
222 |
val u = fold_rev lambda xs t'; |
c9f67836c4d8
internal tuning: class_target, fork_mixfix, declare_const (singleton), abbrev;
wenzelm
parents:
25096
diff
changeset
|
223 |
val global_rhs = |
c9f67836c4d8
internal tuning: class_target, fork_mixfix, declare_const (singleton), abbrev;
wenzelm
parents:
25096
diff
changeset
|
224 |
singleton (Variable.export_terms (Variable.declare_term u target_ctxt) thy_ctxt) u; |
25121 | 225 |
in |
226 |
lthy |> |
|
227 |
(if is_locale then |
|
33671 | 228 |
Local_Theory.theory_result (Sign.add_abbrev PrintMode.internal (b, global_rhs)) |
25121 | 229 |
#-> (fn (lhs, _) => |
35845
e5980f0ad025
renamed varify/unvarify operations to varify_global/unvarify_global to emphasize that these only work in a global situation;
wenzelm
parents:
35798
diff
changeset
|
230 |
let val lhs' = Term.list_comb (Logic.unvarify_global lhs, xs) in |
35798
fd1bb29f8170
replaced type_syntax/term_syntax by uniform syntax_declaration;
wenzelm
parents:
35765
diff
changeset
|
231 |
syntax_declaration ta false (locale_const ta prmode ((b, mx2), lhs')) #> |
33173
b8ca12f6681a
eliminated obsolete tags for types/consts -- now handled via name space, in strongly typed fashion;
wenzelm
parents:
33167
diff
changeset
|
232 |
is_class ? class_target ta (Class_Target.abbrev target prmode ((b, mx1), t')) |
25105
c9f67836c4d8
internal tuning: class_target, fork_mixfix, declare_const (singleton), abbrev;
wenzelm
parents:
25096
diff
changeset
|
233 |
end) |
c9f67836c4d8
internal tuning: class_target, fork_mixfix, declare_const (singleton), abbrev;
wenzelm
parents:
25096
diff
changeset
|
234 |
else |
33671 | 235 |
Local_Theory.theory |
33173
b8ca12f6681a
eliminated obsolete tags for types/consts -- now handled via name space, in strongly typed fashion;
wenzelm
parents:
33167
diff
changeset
|
236 |
(Sign.add_abbrev (#1 prmode) (b, global_rhs) #-> (fn (lhs, _) => |
25121 | 237 |
Sign.notation true prmode [(lhs, mx3)]))) |
33173
b8ca12f6681a
eliminated obsolete tags for types/consts -- now handled via name space, in strongly typed fashion;
wenzelm
parents:
33167
diff
changeset
|
238 |
|> ProofContext.add_abbrev PrintMode.internal (b, t) |> snd |
35624 | 239 |
|> Local_Defs.fixed_abbrev ((b, NoSyn), t) |
24939 | 240 |
end; |
241 |
||
242 |
||
25022 | 243 |
(* define *) |
24939 | 244 |
|
35764 | 245 |
local |
246 |
||
247 |
fun syntax_error c = error ("Illegal mixfix syntax for overloaded constant " ^ quote c); |
|
248 |
||
35765
09e238561460
local theory specifications handle hidden polymorphism implicitly;
wenzelm
parents:
35764
diff
changeset
|
249 |
fun declare_const (ta as Target {target, is_locale, is_class, ...}) |
09e238561460
local theory specifications handle hidden polymorphism implicitly;
wenzelm
parents:
35764
diff
changeset
|
250 |
extra_tfrees xs ((b, T), mx) lthy = |
35764 | 251 |
let |
35765
09e238561460
local theory specifications handle hidden polymorphism implicitly;
wenzelm
parents:
35764
diff
changeset
|
252 |
val type_params = map (Logic.mk_type o TFree) extra_tfrees; |
09e238561460
local theory specifications handle hidden polymorphism implicitly;
wenzelm
parents:
35764
diff
changeset
|
253 |
val term_params = |
35764 | 254 |
rev (Variable.fixes_of (Local_Theory.target_of lthy)) |
255 |
|> map_filter (fn (_, x) => |
|
256 |
(case AList.lookup (op =) xs x of |
|
35765
09e238561460
local theory specifications handle hidden polymorphism implicitly;
wenzelm
parents:
35764
diff
changeset
|
257 |
SOME T => SOME (Free (x, T)) |
35764 | 258 |
| NONE => NONE)); |
35765
09e238561460
local theory specifications handle hidden polymorphism implicitly;
wenzelm
parents:
35764
diff
changeset
|
259 |
val params = type_params @ term_params; |
09e238561460
local theory specifications handle hidden polymorphism implicitly;
wenzelm
parents:
35764
diff
changeset
|
260 |
|
09e238561460
local theory specifications handle hidden polymorphism implicitly;
wenzelm
parents:
35764
diff
changeset
|
261 |
val U = map Term.fastype_of params ---> T; |
35764 | 262 |
val (mx1, mx2, mx3) = fork_mixfix ta mx; |
263 |
val (const, lthy') = lthy |> |
|
264 |
(case Class_Target.instantiation_param lthy b of |
|
265 |
SOME c' => |
|
266 |
if mx3 <> NoSyn then syntax_error c' |
|
267 |
else Local_Theory.theory_result (AxClass.declare_overloaded (c', U)) |
|
268 |
##> Class_Target.confirm_declaration b |
|
269 |
| NONE => |
|
270 |
(case Overloading.operation lthy b of |
|
271 |
SOME (c', _) => |
|
272 |
if mx3 <> NoSyn then syntax_error c' |
|
273 |
else Local_Theory.theory_result (Overloading.declare (c', U)) |
|
274 |
##> Overloading.confirm b |
|
275 |
| NONE => Local_Theory.theory_result (Sign.declare_const ((b, U), mx3)))); |
|
35765
09e238561460
local theory specifications handle hidden polymorphism implicitly;
wenzelm
parents:
35764
diff
changeset
|
276 |
val t = Term.list_comb (const, params); |
35764 | 277 |
in |
278 |
lthy' |
|
35798
fd1bb29f8170
replaced type_syntax/term_syntax by uniform syntax_declaration;
wenzelm
parents:
35765
diff
changeset
|
279 |
|> is_locale ? syntax_declaration ta false (locale_const ta Syntax.mode_default ((b, mx2), t)) |
35858
0d394a82337e
handle hidden polymorphism in class target (without class target syntax, though)
haftmann
parents:
35845
diff
changeset
|
280 |
|> is_class ? class_target ta (Class_Target.declare target ((b, mx1), (type_params, t))) |
35764 | 281 |
|> Local_Defs.add_def ((b, NoSyn), t) |
282 |
end; |
|
283 |
||
284 |
in |
|
285 |
||
33764
7bcefaab8d41
Local_Theory.define: eliminated slightly odd kind argument -- such low-level definitions should be hardly ever exposed to end-users anyway;
wenzelm
parents:
33724
diff
changeset
|
286 |
fun define ta ((b, mx), ((name, atts), rhs)) lthy = |
24939 | 287 |
let |
24987 | 288 |
val thy = ProofContext.theory_of lthy; |
36610
bafd82950e24
renamed ProofContext.init to ProofContext.init_global to emphasize that this is not the real thing;
wenzelm
parents:
36106
diff
changeset
|
289 |
val thy_ctxt = ProofContext.init_global thy; |
24939 | 290 |
|
30437 | 291 |
val name' = Thm.def_binding_optional b name; |
35717 | 292 |
|
293 |
val crhs = Thm.cterm_of thy rhs; |
|
294 |
val (defs, rhs') = Local_Defs.export_cterm lthy thy_ctxt crhs ||> Thm.term_of; |
|
295 |
val rhs_conv = MetaSimplifier.rewrite true defs crhs; |
|
296 |
||
33671 | 297 |
val xs = Variable.add_fixed (Local_Theory.target_of lthy) rhs' []; |
24939 | 298 |
val T = Term.fastype_of rhs; |
35765
09e238561460
local theory specifications handle hidden polymorphism implicitly;
wenzelm
parents:
35764
diff
changeset
|
299 |
val tfreesT = Term.add_tfreesT T (fold (Term.add_tfreesT o #2) xs []); |
09e238561460
local theory specifications handle hidden polymorphism implicitly;
wenzelm
parents:
35764
diff
changeset
|
300 |
val extra_tfrees = |
09e238561460
local theory specifications handle hidden polymorphism implicitly;
wenzelm
parents:
35764
diff
changeset
|
301 |
fold_types (fold_atyps |
09e238561460
local theory specifications handle hidden polymorphism implicitly;
wenzelm
parents:
35764
diff
changeset
|
302 |
(fn TFree v => if member (op =) tfreesT v then I else insert (op =) v | _ => I)) rhs [] |
09e238561460
local theory specifications handle hidden polymorphism implicitly;
wenzelm
parents:
35764
diff
changeset
|
303 |
|> sort_wrt #1; |
24939 | 304 |
|
25105
c9f67836c4d8
internal tuning: class_target, fork_mixfix, declare_const (singleton), abbrev;
wenzelm
parents:
25096
diff
changeset
|
305 |
(*const*) |
35765
09e238561460
local theory specifications handle hidden polymorphism implicitly;
wenzelm
parents:
35764
diff
changeset
|
306 |
val ((lhs, local_def), lthy2) = lthy |> declare_const ta extra_tfrees xs ((b, T), mx); |
25022 | 307 |
val (_, lhs') = Logic.dest_equals (Thm.prop_of local_def); |
35765
09e238561460
local theory specifications handle hidden polymorphism implicitly;
wenzelm
parents:
35764
diff
changeset
|
308 |
val Const (head, _) = Term.head_of lhs'; |
24939 | 309 |
|
310 |
(*def*) |
|
25022 | 311 |
val (global_def, lthy3) = lthy2 |
33671 | 312 |
|> Local_Theory.theory_result |
33282 | 313 |
(case Overloading.operation lthy b of |
35765
09e238561460
local theory specifications handle hidden polymorphism implicitly;
wenzelm
parents:
35764
diff
changeset
|
314 |
SOME (_, checked) => Overloading.define checked name' (head, rhs') |
30519
c05c0199826f
coherent binding policy with primitive target operations
haftmann
parents:
30473
diff
changeset
|
315 |
| NONE => |
35764 | 316 |
if is_some (Class_Target.instantiation_param lthy b) |
35765
09e238561460
local theory specifications handle hidden polymorphism implicitly;
wenzelm
parents:
35764
diff
changeset
|
317 |
then AxClass.define_overloaded name' (head, rhs') |
36106
19deea200358
Thm.add_axiom/add_def: return internal name of foundational axiom;
wenzelm
parents:
35858
diff
changeset
|
318 |
else Thm.add_def false false (name', Logic.mk_equals (lhs', rhs')) #>> snd); |
35624 | 319 |
val def = Local_Defs.trans_terms lthy3 |
25022 | 320 |
[(*c == global.c xs*) local_def, |
321 |
(*global.c xs == rhs'*) global_def, |
|
25485 | 322 |
(*rhs' == rhs*) Thm.symmetric rhs_conv]; |
24939 | 323 |
|
25105
c9f67836c4d8
internal tuning: class_target, fork_mixfix, declare_const (singleton), abbrev;
wenzelm
parents:
25096
diff
changeset
|
324 |
(*note*) |
24939 | 325 |
val ([(res_name, [res])], lthy4) = lthy3 |
33764
7bcefaab8d41
Local_Theory.define: eliminated slightly odd kind argument -- such low-level definitions should be hardly ever exposed to end-users anyway;
wenzelm
parents:
33724
diff
changeset
|
326 |
|> notes ta "" [((name', atts), [([def], [])])]; |
24939 | 327 |
in ((lhs, (res_name, res)), lthy4) end; |
328 |
||
35764 | 329 |
end; |
330 |
||
24939 | 331 |
|
35205 | 332 |
(* init various targets *) |
25291 | 333 |
|
334 |
local |
|
20894 | 335 |
|
25291 | 336 |
fun init_target _ NONE = global_target |
33670
02b7738aef6a
eliminated slightly odd kind argument of LocalTheory.note(s);
wenzelm
parents:
33553
diff
changeset
|
337 |
| init_target thy (SOME target) = |
35205 | 338 |
if Locale.defined thy target |
29710 | 339 |
then make_target target true (Class_Target.is_class thy target) ([], [], []) [] |
340 |
else error ("No such locale: " ^ quote target); |
|
25291 | 341 |
|
29576 | 342 |
fun init_ctxt (Target {target, is_locale, is_class, instantiation, overloading}) = |
29358 | 343 |
if not (null (#1 instantiation)) then Class_Target.init_instantiation instantiation |
25519 | 344 |
else if not (null overloading) then Overloading.init overloading |
36610
bafd82950e24
renamed ProofContext.init to ProofContext.init_global to emphasize that this is not the real thing;
wenzelm
parents:
36106
diff
changeset
|
345 |
else if not is_locale then ProofContext.init_global |
29576 | 346 |
else if not is_class then Locale.init target |
29358 | 347 |
else Class_Target.init target; |
25269 | 348 |
|
25542 | 349 |
fun init_lthy (ta as Target {target, instantiation, overloading, ...}) = |
25291 | 350 |
Data.put ta #> |
33724 | 351 |
Local_Theory.init NONE (Long_Name.base_name target) |
25291 | 352 |
{pretty = pretty ta, |
353 |
abbrev = abbrev ta, |
|
354 |
define = define ta, |
|
355 |
notes = notes ta, |
|
356 |
declaration = declaration ta, |
|
35798
fd1bb29f8170
replaced type_syntax/term_syntax by uniform syntax_declaration;
wenzelm
parents:
35765
diff
changeset
|
357 |
syntax_declaration = syntax_declaration ta, |
25291 | 358 |
reinit = fn lthy => init_lthy_ctxt ta (ProofContext.theory_of lthy), |
33671 | 359 |
exit = Local_Theory.target_of o |
29358 | 360 |
(if not (null (#1 instantiation)) then Class_Target.conclude_instantiation |
26049
8186c03194ed
overloading: reduced code redundancy, no xstrings here;
wenzelm
parents:
25984
diff
changeset
|
361 |
else if not (null overloading) then Overloading.conclude |
8186c03194ed
overloading: reduced code redundancy, no xstrings here;
wenzelm
parents:
25984
diff
changeset
|
362 |
else I)} |
25291 | 363 |
and init_lthy_ctxt ta = init_lthy ta o init_ctxt ta; |
20894 | 364 |
|
26049
8186c03194ed
overloading: reduced code redundancy, no xstrings here;
wenzelm
parents:
25984
diff
changeset
|
365 |
fun gen_overloading prep_const raw_ops thy = |
8186c03194ed
overloading: reduced code redundancy, no xstrings here;
wenzelm
parents:
25984
diff
changeset
|
366 |
let |
36610
bafd82950e24
renamed ProofContext.init to ProofContext.init_global to emphasize that this is not the real thing;
wenzelm
parents:
36106
diff
changeset
|
367 |
val ctxt = ProofContext.init_global thy; |
26049
8186c03194ed
overloading: reduced code redundancy, no xstrings here;
wenzelm
parents:
25984
diff
changeset
|
368 |
val ops = raw_ops |> map (fn (name, const, checked) => |
8186c03194ed
overloading: reduced code redundancy, no xstrings here;
wenzelm
parents:
25984
diff
changeset
|
369 |
(name, Term.dest_Const (prep_const ctxt const), checked)); |
29576 | 370 |
in thy |> init_lthy_ctxt (make_target "" false false ([], [], []) ops) end; |
26049
8186c03194ed
overloading: reduced code redundancy, no xstrings here;
wenzelm
parents:
25984
diff
changeset
|
371 |
|
25291 | 372 |
in |
20894 | 373 |
|
25291 | 374 |
fun init target thy = init_lthy_ctxt (init_target thy target) thy; |
25269 | 375 |
|
35205 | 376 |
fun context_cmd "-" thy = init NONE thy |
377 |
| context_cmd target thy = init (SOME (Locale.intern thy target)) thy; |
|
33282 | 378 |
|
29576 | 379 |
fun instantiation arities = init_lthy_ctxt (make_target "" false false arities []); |
35205 | 380 |
fun instantiation_cmd arities thy = instantiation (Class_Target.read_multi_arity thy arities) thy; |
25519 | 381 |
|
26049
8186c03194ed
overloading: reduced code redundancy, no xstrings here;
wenzelm
parents:
25984
diff
changeset
|
382 |
val overloading = gen_overloading (fn ctxt => Syntax.check_term ctxt o Const); |
8186c03194ed
overloading: reduced code redundancy, no xstrings here;
wenzelm
parents:
25984
diff
changeset
|
383 |
val overloading_cmd = gen_overloading Syntax.read_term; |
25462 | 384 |
|
20894 | 385 |
end; |
25291 | 386 |
|
387 |
end; |
|
388 |