author | haftmann |
Wed, 23 Dec 2009 08:31:15 +0100 | |
changeset 34173 | 458ced35abb8 |
parent 33977 | 406d8e34a3cf |
child 34184 | 248e1fd702e9 |
permissions | -rw-r--r-- |
24219 | 1 |
(* Title: Pure/Isar/code.ML |
2 |
Author: Florian Haftmann, TU Muenchen |
|
3 |
||
34173
458ced35abb8
reduced code generator cache to the baremost minimum
haftmann
parents:
33977
diff
changeset
|
4 |
Abstract executable ingredients of theory. Management of data |
458ced35abb8
reduced code generator cache to the baremost minimum
haftmann
parents:
33977
diff
changeset
|
5 |
dependent on executable ingredients as synchronized cache; purged |
458ced35abb8
reduced code generator cache to the baremost minimum
haftmann
parents:
33977
diff
changeset
|
6 |
on any change of underlying executable ingredients. |
24219 | 7 |
*) |
8 |
||
9 |
signature CODE = |
|
10 |
sig |
|
31957 | 11 |
(*constants*) |
12 |
val check_const: theory -> term -> string |
|
13 |
val read_bare_const: theory -> string -> string * typ |
|
14 |
val read_const: theory -> string -> string |
|
31962 | 15 |
val string_of_const: theory -> string -> string |
33940
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
16 |
val cert_signature: theory -> typ -> typ |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
17 |
val read_signature: theory -> string -> typ |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
18 |
val const_typ: theory -> string -> typ |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
19 |
val subst_signatures: theory -> term -> term |
31962 | 20 |
val args_number: theory -> string -> int |
31957 | 21 |
|
31156 | 22 |
(*constructor sets*) |
23 |
val constrset_of_consts: theory -> (string * typ) list |
|
24 |
-> string * ((string * sort) list * (string * typ list) list) |
|
25 |
||
26 |
(*code equations*) |
|
31962 | 27 |
val mk_eqn: theory -> thm * bool -> thm * bool |
28 |
val mk_eqn_warning: theory -> thm -> (thm * bool) option |
|
29 |
val mk_eqn_liberal: theory -> thm -> (thm * bool) option |
|
31156 | 30 |
val assert_eqn: theory -> thm * bool -> thm * bool |
31 |
val assert_eqns_const: theory -> string |
|
32 |
-> (thm * bool) list -> (thm * bool) list |
|
31957 | 33 |
val const_typ_eqn: theory -> thm -> string * typ |
31156 | 34 |
val typscheme_eqn: theory -> thm -> (string * sort) list * typ |
32873 | 35 |
val typscheme_eqns: theory -> string -> thm list -> (string * sort) list * typ |
32929 | 36 |
val standard_typscheme: theory -> thm list -> thm list |
31156 | 37 |
|
31962 | 38 |
(*executable code*) |
33940
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
39 |
val add_type: string -> theory -> theory |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
40 |
val add_type_cmd: string -> theory -> theory |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
41 |
val add_signature: string * typ -> theory -> theory |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
42 |
val add_signature_cmd: string * string -> theory -> theory |
31156 | 43 |
val add_datatype: (string * typ) list -> theory -> theory |
44 |
val add_datatype_cmd: string list -> theory -> theory |
|
45 |
val type_interpretation: |
|
46 |
(string * ((string * sort) list * (string * typ list) list) |
|
47 |
-> theory -> theory) -> theory -> theory |
|
28368 | 48 |
val add_eqn: thm -> theory -> theory |
31088 | 49 |
val add_nbe_eqn: thm -> theory -> theory |
28368 | 50 |
val add_default_eqn: thm -> theory -> theory |
28703 | 51 |
val add_default_eqn_attribute: attribute |
52 |
val add_default_eqn_attrib: Attrib.src |
|
28368 | 53 |
val del_eqn: thm -> theory -> theory |
54 |
val del_eqns: string -> theory -> theory |
|
24844
98c006a30218
certificates for code generator case expressions
haftmann
parents:
24837
diff
changeset
|
55 |
val add_case: thm -> theory -> theory |
98c006a30218
certificates for code generator case expressions
haftmann
parents:
24837
diff
changeset
|
56 |
val add_undefined: string -> theory -> theory |
24219 | 57 |
val get_datatype: theory -> string -> ((string * sort) list * (string * typ list) list) |
24423
ae9cd0e92423
overloaded definitions accompanied by explicit constants
haftmann
parents:
24283
diff
changeset
|
58 |
val get_datatype_of_constr: theory -> string -> string option |
31156 | 59 |
val these_eqns: theory -> string -> (thm * bool) list |
31642 | 60 |
val all_eqns: theory -> (thm * bool) list |
30023
55954f726043
permissive check for pattern discipline in case schemes
haftmann
parents:
29970
diff
changeset
|
61 |
val get_case_scheme: theory -> string -> (int * (int * string list)) option |
31890
e943b039f0ac
an intermediate step towards a refined translation of cases
haftmann
parents:
31642
diff
changeset
|
62 |
val undefineds: theory -> string list |
24219 | 63 |
val print_codesetup: theory -> unit |
31957 | 64 |
|
65 |
(*infrastructure*) |
|
31998
2c7a24f74db9
code attributes use common underscore convention
haftmann
parents:
31971
diff
changeset
|
66 |
val set_code_target_attr: (string -> thm -> theory -> theory) -> theory -> theory |
31957 | 67 |
val purge_data: theory -> theory |
24219 | 68 |
end; |
69 |
||
70 |
signature CODE_DATA_ARGS = |
|
71 |
sig |
|
72 |
type T |
|
73 |
val empty: T |
|
74 |
end; |
|
75 |
||
76 |
signature CODE_DATA = |
|
77 |
sig |
|
78 |
type T |
|
79 |
val change: theory -> (T -> T) -> T |
|
80 |
val change_yield: theory -> (T -> 'a * T) -> 'a * T |
|
81 |
end; |
|
82 |
||
83 |
signature PRIVATE_CODE = |
|
84 |
sig |
|
85 |
include CODE |
|
34173
458ced35abb8
reduced code generator cache to the baremost minimum
haftmann
parents:
33977
diff
changeset
|
86 |
val declare_data: Object.T -> serial |
24219 | 87 |
val change_data: serial * ('a -> Object.T) * (Object.T -> 'a) |
88 |
-> theory -> ('a -> 'a) -> 'a |
|
89 |
val change_yield_data: serial * ('a -> Object.T) * (Object.T -> 'a) |
|
90 |
-> theory -> ('a -> 'b * 'a) -> 'b * 'a |
|
91 |
end; |
|
92 |
||
93 |
structure Code : PRIVATE_CODE = |
|
94 |
struct |
|
95 |
||
31962 | 96 |
(** auxiliary **) |
97 |
||
98 |
(* printing *) |
|
31156 | 99 |
|
32966
5b21661fe618
indicate CRITICAL nature of various setmp combinators;
wenzelm
parents:
32929
diff
changeset
|
100 |
fun string_of_typ thy = setmp_CRITICAL show_sorts true (Syntax.string_of_typ_global thy); |
31962 | 101 |
|
31156 | 102 |
fun string_of_const thy c = case AxClass.inst_of_param thy c |
103 |
of SOME (c, tyco) => Sign.extern_const thy c ^ " " ^ enclose "[" "]" (Sign.extern_type thy tyco) |
|
104 |
| NONE => Sign.extern_const thy c; |
|
105 |
||
31962 | 106 |
|
107 |
(* constants *) |
|
31156 | 108 |
|
33940
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
109 |
fun typ_equiv tys = Type.raw_instance tys andalso Type.raw_instance (swap tys); |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
110 |
|
31962 | 111 |
fun check_bare_const thy t = case try dest_Const t |
112 |
of SOME c_ty => c_ty |
|
113 |
| NONE => error ("Not a constant: " ^ Syntax.string_of_term_global thy t); |
|
31156 | 114 |
|
31962 | 115 |
fun check_const thy = AxClass.unoverload_const thy o check_bare_const thy; |
116 |
||
117 |
fun read_bare_const thy = check_bare_const thy o Syntax.read_term_global thy; |
|
118 |
||
119 |
fun read_const thy = AxClass.unoverload_const thy o read_bare_const thy; |
|
31156 | 120 |
|
32872
019201eb7e07
variables in type schemes must be renamed simultaneously with variables in equations
haftmann
parents:
32738
diff
changeset
|
121 |
|
31962 | 122 |
|
123 |
(** data store **) |
|
124 |
||
125 |
(* code equations *) |
|
126 |
||
33006 | 127 |
type eqns = bool * (thm * bool) list; |
128 |
(*default flag, theorems with proper flag *) |
|
31962 | 129 |
|
130 |
fun add_drop_redundant thy (thm, proper) thms = |
|
131 |
let |
|
132 |
val args_of = snd o strip_comb o map_types Type.strip_sorts |
|
133 |
o fst o Logic.dest_equals o Thm.plain_prop_of; |
|
134 |
val args = args_of thm; |
|
135 |
val incr_idx = Logic.incr_indexes ([], Thm.maxidx_of thm + 1); |
|
136 |
fun matches_args args' = length args <= length args' andalso |
|
33957 | 137 |
Pattern.matchess thy (args, (map incr_idx o take (length args)) args'); |
31962 | 138 |
fun drop (thm', proper') = if (proper orelse not proper') |
139 |
andalso matches_args (args_of thm') then |
|
32091
30e2ffbba718
proper context for Display.pretty_thm etc. or old-style versions Display.pretty_thm_global, Display.pretty_thm_without_context etc.;
wenzelm
parents:
32070
diff
changeset
|
140 |
(warning ("Code generator: dropping redundant code equation\n" ^ |
30e2ffbba718
proper context for Display.pretty_thm etc. or old-style versions Display.pretty_thm_global, Display.pretty_thm_without_context etc.;
wenzelm
parents:
32070
diff
changeset
|
141 |
Display.string_of_thm_global thy thm'); true) |
31962 | 142 |
else false; |
143 |
in (thm, proper) :: filter_out drop thms end; |
|
144 |
||
33006 | 145 |
fun add_thm thy _ thm (false, thms) = (false, add_drop_redundant thy thm thms) |
146 |
| add_thm thy true thm (true, thms) = (true, thms @ [thm]) |
|
147 |
| add_thm thy false thm (true, thms) = (false, [thm]); |
|
31962 | 148 |
|
33006 | 149 |
fun del_thm thm = apsnd (remove (eq_fst Thm.eq_thm_prop) (thm, true)); |
31962 | 150 |
|
151 |
||
152 |
(* executable code data *) |
|
153 |
||
154 |
datatype spec = Spec of { |
|
155 |
history_concluded: bool, |
|
33940
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
156 |
signatures: int Symtab.table * typ Symtab.table, |
31962 | 157 |
eqns: ((bool * eqns) * (serial * eqns) list) Symtab.table |
158 |
(*with explicit history*), |
|
159 |
dtyps: ((serial * ((string * sort) list * (string * typ list) list)) list) Symtab.table |
|
160 |
(*with explicit history*), |
|
161 |
cases: (int * (int * string list)) Symtab.table * unit Symtab.table |
|
162 |
}; |
|
163 |
||
33940
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
164 |
fun make_spec (history_concluded, ((signatures, eqns), (dtyps, cases))) = |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
165 |
Spec { history_concluded = history_concluded, |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
166 |
signatures = signatures, eqns = eqns, dtyps = dtyps, cases = cases }; |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
167 |
fun map_spec f (Spec { history_concluded = history_concluded, signatures = signatures, |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
168 |
eqns = eqns, dtyps = dtyps, cases = cases }) = |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
169 |
make_spec (f (history_concluded, ((signatures, eqns), (dtyps, cases)))); |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
170 |
fun merge_spec (Spec { history_concluded = _, signatures = (tycos1, sigs1), eqns = eqns1, |
31962 | 171 |
dtyps = dtyps1, cases = (cases1, undefs1) }, |
33940
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
172 |
Spec { history_concluded = _, signatures = (tycos2, sigs2), eqns = eqns2, |
31962 | 173 |
dtyps = dtyps2, cases = (cases2, undefs2) }) = |
31156 | 174 |
let |
33940
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
175 |
val signatures = (Symtab.merge (op =) (tycos1, tycos2), |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
176 |
Symtab.merge typ_equiv (sigs1, sigs2)); |
31962 | 177 |
fun merge_eqns ((_, history1), (_, history2)) = |
178 |
let |
|
179 |
val raw_history = AList.merge (op = : serial * serial -> bool) |
|
180 |
(K true) (history1, history2) |
|
181 |
val filtered_history = filter_out (fst o snd) raw_history |
|
182 |
val history = if null filtered_history |
|
183 |
then raw_history else filtered_history; |
|
184 |
in ((false, (snd o hd) history), history) end; |
|
185 |
val eqns = Symtab.join (K merge_eqns) (eqns1, eqns2); |
|
186 |
val dtyps = Symtab.join (K (AList.merge (op =) (K true))) (dtyps1, dtyps2); |
|
187 |
val cases = (Symtab.merge (K true) (cases1, cases2), |
|
188 |
Symtab.merge (K true) (undefs1, undefs2)); |
|
33940
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
189 |
in make_spec (false, ((signatures, eqns), (dtyps, cases))) end; |
31962 | 190 |
|
191 |
fun history_concluded (Spec { history_concluded, ... }) = history_concluded; |
|
33940
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
192 |
fun the_signatures (Spec { signatures, ... }) = signatures; |
31962 | 193 |
fun the_eqns (Spec { eqns, ... }) = eqns; |
194 |
fun the_dtyps (Spec { dtyps, ... }) = dtyps; |
|
195 |
fun the_cases (Spec { cases, ... }) = cases; |
|
32544 | 196 |
val map_history_concluded = map_spec o apfst; |
33940
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
197 |
val map_signatures = map_spec o apsnd o apfst o apfst; |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
198 |
val map_eqns = map_spec o apsnd o apfst o apsnd; |
31962 | 199 |
val map_dtyps = map_spec o apsnd o apsnd o apfst; |
200 |
val map_cases = map_spec o apsnd o apsnd o apsnd; |
|
201 |
||
202 |
||
203 |
(* data slots dependent on executable code *) |
|
204 |
||
205 |
(*private copy avoids potential conflict of table exceptions*) |
|
31971
8c1b845ed105
renamed functor TableFun to Table, and GraphFun to Graph;
wenzelm
parents:
31962
diff
changeset
|
206 |
structure Datatab = Table(type key = int val ord = int_ord); |
31962 | 207 |
|
208 |
local |
|
209 |
||
34173
458ced35abb8
reduced code generator cache to the baremost minimum
haftmann
parents:
33977
diff
changeset
|
210 |
type kind = { empty: Object.T }; |
31962 | 211 |
|
32738 | 212 |
val kinds = Unsynchronized.ref (Datatab.empty: kind Datatab.table); |
31962 | 213 |
|
214 |
fun invoke f k = case Datatab.lookup (! kinds) k |
|
215 |
of SOME kind => f kind |
|
216 |
| NONE => sys_error "Invalid code data identifier"; |
|
217 |
||
218 |
in |
|
219 |
||
34173
458ced35abb8
reduced code generator cache to the baremost minimum
haftmann
parents:
33977
diff
changeset
|
220 |
fun declare_data empty = |
31962 | 221 |
let |
222 |
val k = serial (); |
|
34173
458ced35abb8
reduced code generator cache to the baremost minimum
haftmann
parents:
33977
diff
changeset
|
223 |
val kind = { empty = empty }; |
458ced35abb8
reduced code generator cache to the baremost minimum
haftmann
parents:
33977
diff
changeset
|
224 |
val _ = CRITICAL (fn () => Unsynchronized.change kinds (Datatab.update (k, kind))); |
31962 | 225 |
in k end; |
226 |
||
227 |
fun invoke_init k = invoke (fn kind => #empty kind) k; |
|
228 |
||
229 |
end; (*local*) |
|
230 |
||
231 |
||
232 |
(* theory store *) |
|
233 |
||
234 |
local |
|
235 |
||
236 |
type data = Object.T Datatab.table; |
|
34173
458ced35abb8
reduced code generator cache to the baremost minimum
haftmann
parents:
33977
diff
changeset
|
237 |
fun create_data data = Synchronized.var "code data" data; |
458ced35abb8
reduced code generator cache to the baremost minimum
haftmann
parents:
33977
diff
changeset
|
238 |
fun empty_data () = create_data Datatab.empty; |
31962 | 239 |
|
240 |
structure Code_Data = TheoryDataFun |
|
241 |
( |
|
34173
458ced35abb8
reduced code generator cache to the baremost minimum
haftmann
parents:
33977
diff
changeset
|
242 |
type T = spec * data Synchronized.var; |
33940
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
243 |
val empty = (make_spec (false, (((Symtab.empty, Symtab.empty), Symtab.empty), |
34173
458ced35abb8
reduced code generator cache to the baremost minimum
haftmann
parents:
33977
diff
changeset
|
244 |
(Symtab.empty, (Symtab.empty, Symtab.empty)))), empty_data ()); |
458ced35abb8
reduced code generator cache to the baremost minimum
haftmann
parents:
33977
diff
changeset
|
245 |
fun copy (spec, data) = (spec, create_data (Synchronized.value data)); |
31962 | 246 |
val extend = copy; |
33969 | 247 |
fun merge _ ((spec1, _), (spec2, _)) = |
34173
458ced35abb8
reduced code generator cache to the baremost minimum
haftmann
parents:
33977
diff
changeset
|
248 |
(merge_spec (spec1, spec2), empty_data ()); |
31962 | 249 |
); |
250 |
||
251 |
fun thy_data f thy = f ((snd o Code_Data.get) thy); |
|
252 |
||
34173
458ced35abb8
reduced code generator cache to the baremost minimum
haftmann
parents:
33977
diff
changeset
|
253 |
fun get_ensure_init kind data = |
458ced35abb8
reduced code generator cache to the baremost minimum
haftmann
parents:
33977
diff
changeset
|
254 |
case Datatab.lookup (Synchronized.value data) kind |
31962 | 255 |
of SOME x => x |
256 |
| NONE => let val y = invoke_init kind |
|
34173
458ced35abb8
reduced code generator cache to the baremost minimum
haftmann
parents:
33977
diff
changeset
|
257 |
in (Synchronized.change data (Datatab.update (kind, y)); y) end; |
31962 | 258 |
|
259 |
in |
|
260 |
||
261 |
(* access to executable code *) |
|
262 |
||
263 |
val the_exec = fst o Code_Data.get; |
|
264 |
||
34173
458ced35abb8
reduced code generator cache to the baremost minimum
haftmann
parents:
33977
diff
changeset
|
265 |
fun map_exec_purge f = |
458ced35abb8
reduced code generator cache to the baremost minimum
haftmann
parents:
33977
diff
changeset
|
266 |
Code_Data.map (fn (exec, data) => (f exec, empty_data ())); |
31962 | 267 |
|
34173
458ced35abb8
reduced code generator cache to the baremost minimum
haftmann
parents:
33977
diff
changeset
|
268 |
val purge_data = (Code_Data.map o apsnd) (fn _ => empty_data ()); |
31962 | 269 |
|
34173
458ced35abb8
reduced code generator cache to the baremost minimum
haftmann
parents:
33977
diff
changeset
|
270 |
fun change_eqns delete c f = (map_exec_purge o map_eqns |
33006 | 271 |
o (if delete then Symtab.map_entry c else Symtab.map_default (c, ((false, (true, [])), []))) |
31962 | 272 |
o apfst) (fn (_, eqns) => (true, f eqns)); |
273 |
||
33006 | 274 |
fun del_eqns c = change_eqns true c (K (false, [])); |
31962 | 275 |
|
276 |
||
277 |
(* tackling equation history *) |
|
278 |
||
279 |
fun get_eqns thy c = |
|
280 |
Symtab.lookup ((the_eqns o the_exec) thy) c |
|
33006 | 281 |
|> Option.map (snd o snd o fst) |
31962 | 282 |
|> these; |
283 |
||
284 |
fun continue_history thy = if (history_concluded o the_exec) thy |
|
285 |
then thy |
|
286 |
|> (Code_Data.map o apfst o map_history_concluded) (K false) |
|
287 |
|> SOME |
|
288 |
else NONE; |
|
289 |
||
290 |
fun conclude_history thy = if (history_concluded o the_exec) thy |
|
291 |
then NONE |
|
292 |
else thy |
|
293 |
|> (Code_Data.map o apfst) |
|
294 |
((map_eqns o Symtab.map) (fn ((changed, current), history) => |
|
295 |
((false, current), |
|
296 |
if changed then (serial (), current) :: history else history)) |
|
297 |
#> map_history_concluded (K true)) |
|
298 |
|> SOME; |
|
299 |
||
300 |
val _ = Context.>> (Context.map_theory (Code_Data.init |
|
301 |
#> Theory.at_begin continue_history |
|
302 |
#> Theory.at_end conclude_history)); |
|
303 |
||
304 |
||
305 |
(* access to data dependent on abstract executable code *) |
|
306 |
||
307 |
fun change_data (kind, mk, dest) = |
|
308 |
let |
|
309 |
fun chnge data_ref f = |
|
310 |
let |
|
311 |
val data = get_ensure_init kind data_ref; |
|
312 |
val data' = f (dest data); |
|
34173
458ced35abb8
reduced code generator cache to the baremost minimum
haftmann
parents:
33977
diff
changeset
|
313 |
in (Synchronized.change data_ref (Datatab.update (kind, mk data')); data') end; |
31962 | 314 |
in thy_data chnge end; |
315 |
||
316 |
fun change_yield_data (kind, mk, dest) = |
|
317 |
let |
|
318 |
fun chnge data_ref f = |
|
319 |
let |
|
320 |
val data = get_ensure_init kind data_ref; |
|
321 |
val (x, data') = f (dest data); |
|
34173
458ced35abb8
reduced code generator cache to the baremost minimum
haftmann
parents:
33977
diff
changeset
|
322 |
in (x, (Synchronized.change data_ref (Datatab.update (kind, mk data')); data')) end; |
31962 | 323 |
in thy_data chnge end; |
324 |
||
325 |
end; (*local*) |
|
326 |
||
327 |
||
328 |
(** foundation **) |
|
329 |
||
330 |
(* constants *) |
|
331 |
||
33940
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
332 |
fun arity_number thy tyco = case Symtab.lookup ((fst o the_signatures o the_exec) thy) tyco |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
333 |
of SOME n => n |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
334 |
| NONE => Sign.arity_number thy tyco; |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
335 |
|
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
336 |
fun build_tsig thy = |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
337 |
let |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
338 |
val (tycos, _) = (the_signatures o the_exec) thy; |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
339 |
val decls = (#types o Type.rep_tsig o Sign.tsig_of) thy |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
340 |
|> apsnd (Symtab.fold (fn (tyco, n) => |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
341 |
Symtab.update (tyco, Type.LogicalType n)) tycos); |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
342 |
in Type.build_tsig ((Name_Space.empty "", Sorts.empty_algebra), [], decls) end; |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
343 |
|
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
344 |
fun cert_signature thy = Logic.varifyT o Type.cert_typ (build_tsig thy) o Type.no_tvars; |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
345 |
|
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
346 |
fun read_signature thy = cert_signature thy o Type.strip_sorts |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
347 |
o Syntax.parse_typ (ProofContext.init thy); |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
348 |
|
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
349 |
fun expand_signature thy = Type.cert_typ_mode Type.mode_syntax (Sign.tsig_of thy); |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
350 |
|
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
351 |
fun lookup_typ thy = Symtab.lookup ((snd o the_signatures o the_exec) thy); |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
352 |
|
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
353 |
fun const_typ thy c = case lookup_typ thy c |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
354 |
of SOME ty => ty |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
355 |
| NONE => (Type.strip_sorts o Sign.the_const_type thy) c; |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
356 |
|
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
357 |
fun subst_signature thy c ty = |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
358 |
let |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
359 |
fun mk_subst (Type (tyco, tys1)) (ty2 as Type (tyco2, tys2)) = |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
360 |
fold2 mk_subst tys1 tys2 |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
361 |
| mk_subst ty (TVar (v, sort)) = Vartab.update (v, ([], ty)) |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
362 |
in case lookup_typ thy c |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
363 |
of SOME ty' => Envir.subst_type (mk_subst ty (expand_signature thy ty') Vartab.empty) ty' |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
364 |
| NONE => ty |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
365 |
end; |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
366 |
|
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
367 |
fun subst_signatures thy = map_aterms (fn Const (c, ty) => Const (c, subst_signature thy c ty) | t => t); |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
368 |
|
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
369 |
fun args_number thy = length o fst o strip_type o const_typ thy; |
31962 | 370 |
|
371 |
||
372 |
(* datatypes *) |
|
31156 | 373 |
|
374 |
fun constrset_of_consts thy cs = |
|
375 |
let |
|
376 |
val _ = map (fn (c, _) => if (is_some o AxClass.class_of_param thy) c |
|
377 |
then error ("Is a class parameter: " ^ string_of_const thy c) else ()) cs; |
|
33531 | 378 |
fun no_constr s (c, ty) = error ("Not a datatype constructor:\n" ^ string_of_const thy c |
379 |
^ " :: " ^ string_of_typ thy ty ^ "\n" ^ enclose "(" ")" s); |
|
31156 | 380 |
fun last_typ c_ty ty = |
381 |
let |
|
33531 | 382 |
val tfrees = Term.add_tfreesT ty []; |
31156 | 383 |
val (tyco, vs) = ((apsnd o map) (dest_TFree) o dest_Type o snd o strip_type) ty |
33531 | 384 |
handle TYPE _ => no_constr "bad type" c_ty |
385 |
val _ = if has_duplicates (eq_fst (op =)) vs |
|
386 |
then no_constr "duplicate type variables in datatype" c_ty else (); |
|
387 |
val _ = if length tfrees <> length vs |
|
388 |
then no_constr "type variables missing in datatype" c_ty else (); |
|
31156 | 389 |
in (tyco, vs) end; |
33940
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
390 |
fun ty_sorts (c, raw_ty) = |
31156 | 391 |
let |
33940
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
392 |
val ty = subst_signature thy c raw_ty; |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
393 |
val ty_decl = (Logic.unvarifyT o const_typ thy) c; |
31156 | 394 |
val (tyco, _) = last_typ (c, ty) ty_decl; |
395 |
val (_, vs) = last_typ (c, ty) ty; |
|
396 |
in ((tyco, map snd vs), (c, (map fst vs, ty))) end; |
|
397 |
fun add ((tyco', sorts'), c) ((tyco, sorts), cs) = |
|
398 |
let |
|
31998
2c7a24f74db9
code attributes use common underscore convention
haftmann
parents:
31971
diff
changeset
|
399 |
val _ = if (tyco' : string) <> tyco |
31156 | 400 |
then error "Different type constructors in constructor set" |
401 |
else (); |
|
402 |
val sorts'' = map2 (curry (Sorts.inter_sort (Sign.classes_of thy))) sorts' sorts |
|
403 |
in ((tyco, sorts), c :: cs) end; |
|
404 |
fun inst vs' (c, (vs, ty)) = |
|
405 |
let |
|
406 |
val the_v = the o AList.lookup (op =) (vs ~~ vs'); |
|
407 |
val ty' = map_atyps (fn TFree (v, _) => TFree (the_v v)) ty; |
|
408 |
in (c, (fst o strip_type) ty') end; |
|
409 |
val c' :: cs' = map ty_sorts cs; |
|
410 |
val ((tyco, sorts), cs'') = fold add cs' (apsnd single c'); |
|
411 |
val vs = Name.names Name.context Name.aT sorts; |
|
412 |
val cs''' = map (inst vs) cs''; |
|
413 |
in (tyco, (vs, rev cs''')) end; |
|
414 |
||
31962 | 415 |
fun get_datatype thy tyco = |
416 |
case these (Symtab.lookup ((the_dtyps o the_exec) thy) tyco) |
|
417 |
of (_, spec) :: _ => spec |
|
33940
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
418 |
| [] => arity_number thy tyco |
31962 | 419 |
|> Name.invents Name.context Name.aT |
420 |
|> map (rpair []) |
|
421 |
|> rpair []; |
|
422 |
||
423 |
fun get_datatype_of_constr thy c = |
|
33940
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
424 |
case (snd o strip_type o const_typ thy) c |
31962 | 425 |
of Type (tyco, _) => if member (op =) ((map fst o snd o get_datatype thy) tyco) c |
426 |
then SOME tyco else NONE |
|
427 |
| _ => NONE; |
|
428 |
||
429 |
fun is_constr thy = is_some o get_datatype_of_constr thy; |
|
430 |
||
31156 | 431 |
|
432 |
(* code equations *) |
|
433 |
||
434 |
exception BAD_THM of string; |
|
435 |
fun bad_thm msg = raise BAD_THM msg; |
|
436 |
fun error_thm f thm = f thm handle BAD_THM msg => error msg; |
|
31642 | 437 |
fun warning_thm f thm = SOME (f thm) handle BAD_THM msg => (warning msg; NONE) |
31156 | 438 |
fun try_thm f thm = SOME (f thm) handle BAD_THM _ => NONE; |
439 |
||
440 |
fun is_linear thm = |
|
441 |
let val (_, args) = (strip_comb o fst o Logic.dest_equals o Thm.plain_prop_of) thm |
|
442 |
in not (has_duplicates (op =) ((fold o fold_aterms) |
|
443 |
(fn Var (v, _) => cons v | _ => I) args [])) end; |
|
444 |
||
31962 | 445 |
fun gen_assert_eqn thy is_constr_pat (thm, proper) = |
31156 | 446 |
let |
447 |
val (lhs, rhs) = (Logic.dest_equals o Thm.plain_prop_of) thm |
|
32091
30e2ffbba718
proper context for Display.pretty_thm etc. or old-style versions Display.pretty_thm_global, Display.pretty_thm_without_context etc.;
wenzelm
parents:
32070
diff
changeset
|
448 |
handle TERM _ => bad_thm ("Not an equation: " ^ Display.string_of_thm_global thy thm) |
30e2ffbba718
proper context for Display.pretty_thm etc. or old-style versions Display.pretty_thm_global, Display.pretty_thm_without_context etc.;
wenzelm
parents:
32070
diff
changeset
|
449 |
| THM _ => bad_thm ("Not an equation: " ^ Display.string_of_thm_global thy thm); |
31156 | 450 |
fun vars_of t = fold_aterms (fn Var (v, _) => insert (op =) v |
451 |
| Free _ => bad_thm ("Illegal free variable in equation\n" |
|
32091
30e2ffbba718
proper context for Display.pretty_thm etc. or old-style versions Display.pretty_thm_global, Display.pretty_thm_without_context etc.;
wenzelm
parents:
32070
diff
changeset
|
452 |
^ Display.string_of_thm_global thy thm) |
31156 | 453 |
| _ => I) t []; |
454 |
fun tvars_of t = fold_term_types (fn _ => |
|
455 |
fold_atyps (fn TVar (v, _) => insert (op =) v |
|
456 |
| TFree _ => bad_thm |
|
32091
30e2ffbba718
proper context for Display.pretty_thm etc. or old-style versions Display.pretty_thm_global, Display.pretty_thm_without_context etc.;
wenzelm
parents:
32070
diff
changeset
|
457 |
("Illegal free type variable in equation\n" ^ Display.string_of_thm_global thy thm))) t []; |
31156 | 458 |
val lhs_vs = vars_of lhs; |
459 |
val rhs_vs = vars_of rhs; |
|
460 |
val lhs_tvs = tvars_of lhs; |
|
461 |
val rhs_tvs = tvars_of rhs; |
|
462 |
val _ = if null (subtract (op =) lhs_vs rhs_vs) |
|
463 |
then () |
|
464 |
else bad_thm ("Free variables on right hand side of equation\n" |
|
32091
30e2ffbba718
proper context for Display.pretty_thm etc. or old-style versions Display.pretty_thm_global, Display.pretty_thm_without_context etc.;
wenzelm
parents:
32070
diff
changeset
|
465 |
^ Display.string_of_thm_global thy thm); |
31156 | 466 |
val _ = if null (subtract (op =) lhs_tvs rhs_tvs) |
467 |
then () |
|
468 |
else bad_thm ("Free type variables on right hand side of equation\n" |
|
32091
30e2ffbba718
proper context for Display.pretty_thm etc. or old-style versions Display.pretty_thm_global, Display.pretty_thm_without_context etc.;
wenzelm
parents:
32070
diff
changeset
|
469 |
^ Display.string_of_thm_global thy thm) |
30e2ffbba718
proper context for Display.pretty_thm etc. or old-style versions Display.pretty_thm_global, Display.pretty_thm_without_context etc.;
wenzelm
parents:
32070
diff
changeset
|
470 |
val (head, args) = (strip_comb o fst o Logic.dest_equals o Thm.plain_prop_of) thm; |
31156 | 471 |
val (c, ty) = case head |
472 |
of Const (c_ty as (_, ty)) => (AxClass.unoverload_const thy c_ty, ty) |
|
32091
30e2ffbba718
proper context for Display.pretty_thm etc. or old-style versions Display.pretty_thm_global, Display.pretty_thm_without_context etc.;
wenzelm
parents:
32070
diff
changeset
|
473 |
| _ => bad_thm ("Equation not headed by constant\n" ^ Display.string_of_thm_global thy thm); |
31156 | 474 |
fun check _ (Abs _) = bad_thm |
475 |
("Abstraction on left hand side of equation\n" |
|
32091
30e2ffbba718
proper context for Display.pretty_thm etc. or old-style versions Display.pretty_thm_global, Display.pretty_thm_without_context etc.;
wenzelm
parents:
32070
diff
changeset
|
476 |
^ Display.string_of_thm_global thy thm) |
31156 | 477 |
| check 0 (Var _) = () |
478 |
| check _ (Var _) = bad_thm |
|
479 |
("Variable with application on left hand side of equation\n" |
|
32091
30e2ffbba718
proper context for Display.pretty_thm etc. or old-style versions Display.pretty_thm_global, Display.pretty_thm_without_context etc.;
wenzelm
parents:
32070
diff
changeset
|
480 |
^ Display.string_of_thm_global thy thm) |
31156 | 481 |
| check n (t1 $ t2) = (check (n+1) t1; check 0 t2) |
33940
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
482 |
| check n (Const (c_ty as (_, ty))) = |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
483 |
let |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
484 |
val c' = AxClass.unoverload_const thy c_ty |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
485 |
in if n = (length o fst o strip_type o subst_signature thy c') ty |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
486 |
then if not proper orelse is_constr_pat c' |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
487 |
then () |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
488 |
else bad_thm (quote c ^ " is not a constructor, on left hand side of equation\n" |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
489 |
^ Display.string_of_thm_global thy thm) |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
490 |
else bad_thm |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
491 |
("Partially applied constant " ^ quote c ^ " on left hand side of equation\n" |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
492 |
^ Display.string_of_thm_global thy thm) |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
493 |
end; |
31156 | 494 |
val _ = map (check 0) args; |
495 |
val _ = if not proper orelse is_linear thm then () |
|
496 |
else bad_thm ("Duplicate variables on left hand side of equation\n" |
|
32091
30e2ffbba718
proper context for Display.pretty_thm etc. or old-style versions Display.pretty_thm_global, Display.pretty_thm_without_context etc.;
wenzelm
parents:
32070
diff
changeset
|
497 |
^ Display.string_of_thm_global thy thm); |
31156 | 498 |
val _ = if (is_none o AxClass.class_of_param thy) c |
499 |
then () |
|
33940
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
500 |
else bad_thm ("Overloaded constant as head in equation\n" |
32091
30e2ffbba718
proper context for Display.pretty_thm etc. or old-style versions Display.pretty_thm_global, Display.pretty_thm_without_context etc.;
wenzelm
parents:
32070
diff
changeset
|
501 |
^ Display.string_of_thm_global thy thm) |
31962 | 502 |
val _ = if not (is_constr thy c) |
31156 | 503 |
then () |
504 |
else bad_thm ("Constructor as head in equation\n" |
|
32091
30e2ffbba718
proper context for Display.pretty_thm etc. or old-style versions Display.pretty_thm_global, Display.pretty_thm_without_context etc.;
wenzelm
parents:
32070
diff
changeset
|
505 |
^ Display.string_of_thm_global thy thm) |
31156 | 506 |
val ty_decl = Sign.the_const_type thy c; |
507 |
val _ = if Sign.typ_equiv thy (Type.strip_sorts ty_decl, Type.strip_sorts ty) |
|
508 |
then () else bad_thm ("Type\n" ^ string_of_typ thy ty |
|
509 |
^ "\nof equation\n" |
|
32091
30e2ffbba718
proper context for Display.pretty_thm etc. or old-style versions Display.pretty_thm_global, Display.pretty_thm_without_context etc.;
wenzelm
parents:
32070
diff
changeset
|
510 |
^ Display.string_of_thm_global thy thm |
31156 | 511 |
^ "\nis incompatible with declared function type\n" |
512 |
^ string_of_typ thy ty_decl) |
|
513 |
in (thm, proper) end; |
|
514 |
||
31962 | 515 |
fun assert_eqn thy = error_thm (gen_assert_eqn thy (is_constr thy)); |
516 |
||
517 |
fun meta_rewrite thy = LocalDefs.meta_rewrite_rule (ProofContext.init thy); |
|
31156 | 518 |
|
31962 | 519 |
fun mk_eqn thy = error_thm (gen_assert_eqn thy (K true)) o |
520 |
apfst (meta_rewrite thy); |
|
521 |
||
522 |
fun mk_eqn_warning thy = Option.map (fn (thm, _) => (thm, is_linear thm)) |
|
523 |
o warning_thm (gen_assert_eqn thy (K true)) o rpair false o meta_rewrite thy; |
|
524 |
||
525 |
fun mk_eqn_liberal thy = Option.map (fn (thm, _) => (thm, is_linear thm)) |
|
526 |
o try_thm (gen_assert_eqn thy (K true)) o rpair false o meta_rewrite thy; |
|
31156 | 527 |
|
33940
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
528 |
val head_eqn = dest_Const o fst o strip_comb o fst o Logic.dest_equals o Thm.plain_prop_of; |
31156 | 529 |
|
31957 | 530 |
fun const_typ_eqn thy thm = |
31156 | 531 |
let |
32640
ba6531df2c64
corrected order of type variables in code equations; more precise certificate for cases
haftmann
parents:
32544
diff
changeset
|
532 |
val (c, ty) = head_eqn thm; |
31156 | 533 |
val c' = AxClass.unoverload_const thy (c, ty); |
33940
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
534 |
(*permissive wrt. to overloaded constants!*) |
31156 | 535 |
in (c', ty) end; |
33940
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
536 |
|
31957 | 537 |
fun const_eqn thy = fst o const_typ_eqn thy; |
31156 | 538 |
|
33940
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
539 |
fun raw_typscheme thy (c, ty) = |
32873 | 540 |
(map dest_TFree (Sign.const_typargs thy (c, ty)), Type.strip_sorts ty); |
33940
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
541 |
|
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
542 |
fun typscheme thy (c, ty) = raw_typscheme thy (c, subst_signature thy c ty); |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
543 |
|
32873 | 544 |
fun typscheme_eqn thy = typscheme thy o apsnd Logic.unvarifyT o const_typ_eqn thy; |
33940
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
545 |
|
32873 | 546 |
fun typscheme_eqns thy c [] = |
547 |
let |
|
33940
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
548 |
val raw_ty = const_typ thy c; |
32873 | 549 |
val tvars = Term.add_tvar_namesT raw_ty []; |
550 |
val tvars' = case AxClass.class_of_param thy c |
|
551 |
of SOME class => [TFree (Name.aT, [class])] |
|
552 |
| NONE => Name.invent_list [] Name.aT (length tvars) |
|
553 |
|> map (fn v => TFree (v, [])); |
|
554 |
val ty = typ_subst_TVars (tvars ~~ tvars') raw_ty; |
|
33940
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
555 |
in raw_typscheme thy (c, ty) end |
33969 | 556 |
| typscheme_eqns thy c (thm :: _) = typscheme_eqn thy thm; |
32872
019201eb7e07
variables in type schemes must be renamed simultaneously with variables in equations
haftmann
parents:
32738
diff
changeset
|
557 |
|
31962 | 558 |
fun assert_eqns_const thy c eqns = |
559 |
let |
|
560 |
fun cert (eqn as (thm, _)) = if c = const_eqn thy thm |
|
561 |
then eqn else error ("Wrong head of code equation,\nexpected constant " |
|
32091
30e2ffbba718
proper context for Display.pretty_thm etc. or old-style versions Display.pretty_thm_global, Display.pretty_thm_without_context etc.;
wenzelm
parents:
32070
diff
changeset
|
562 |
^ string_of_const thy c ^ "\n" ^ Display.string_of_thm_global thy thm) |
31962 | 563 |
in map (cert o assert_eqn thy) eqns end; |
31156 | 564 |
|
32929 | 565 |
fun standard_typscheme thy thms = |
32354 | 566 |
let |
32640
ba6531df2c64
corrected order of type variables in code equations; more precise certificate for cases
haftmann
parents:
32544
diff
changeset
|
567 |
fun tvars_of T = rev (Term.add_tvarsT T []); |
ba6531df2c64
corrected order of type variables in code equations; more precise certificate for cases
haftmann
parents:
32544
diff
changeset
|
568 |
val vss = map (tvars_of o snd o head_eqn) thms; |
32354 | 569 |
fun inter_sorts vs = |
570 |
fold (curry (Sorts.inter_sort (Sign.classes_of thy)) o snd) vs []; |
|
571 |
val sorts = map_transpose inter_sorts vss; |
|
32873 | 572 |
val vts = Name.names Name.context Name.aT sorts |
32354 | 573 |
|> map (fn (v, sort) => TVar ((v, 0), sort)); |
574 |
in map2 (fn vs => Thm.certify_instantiate (vs ~~ vts, [])) vss thms end; |
|
31962 | 575 |
|
576 |
fun these_eqns thy c = |
|
577 |
get_eqns thy c |
|
578 |
|> (map o apfst) (Thm.transfer thy) |
|
32929 | 579 |
|> burrow_fst (standard_typscheme thy); |
31962 | 580 |
|
581 |
fun all_eqns thy = |
|
582 |
Symtab.dest ((the_eqns o the_exec) thy) |
|
33006 | 583 |
|> maps (snd o snd o fst o snd); |
31962 | 584 |
|
585 |
||
586 |
(* cases *) |
|
31156 | 587 |
|
588 |
fun case_certificate thm = |
|
589 |
let |
|
590 |
val ((head, raw_case_expr), cases) = (apfst Logic.dest_equals |
|
32640
ba6531df2c64
corrected order of type variables in code equations; more precise certificate for cases
haftmann
parents:
32544
diff
changeset
|
591 |
o apsnd Logic.dest_conjunctions o Logic.dest_implies o Thm.plain_prop_of) thm; |
31156 | 592 |
val _ = case head of Free _ => true |
593 |
| Var _ => true |
|
594 |
| _ => raise TERM ("case_cert", []); |
|
595 |
val ([(case_var, _)], case_expr) = Term.strip_abs_eta 1 raw_case_expr; |
|
596 |
val (Const (case_const, _), raw_params) = strip_comb case_expr; |
|
597 |
val n = find_index (fn Free (v, _) => v = case_var | _ => false) raw_params; |
|
598 |
val _ = if n = ~1 then raise TERM ("case_cert", []) else (); |
|
599 |
val params = map (fst o dest_Var) (nth_drop n raw_params); |
|
600 |
fun dest_case t = |
|
601 |
let |
|
602 |
val (head' $ t_co, rhs) = Logic.dest_equals t; |
|
603 |
val _ = if head' = head then () else raise TERM ("case_cert", []); |
|
604 |
val (Const (co, _), args) = strip_comb t_co; |
|
605 |
val (Var (param, _), args') = strip_comb rhs; |
|
606 |
val _ = if args' = args then () else raise TERM ("case_cert", []); |
|
607 |
in (param, co) end; |
|
608 |
fun analyze_cases cases = |
|
609 |
let |
|
610 |
val co_list = fold (AList.update (op =) o dest_case) cases []; |
|
611 |
in map (the o AList.lookup (op =) co_list) params end; |
|
612 |
fun analyze_let t = |
|
613 |
let |
|
614 |
val (head' $ arg, Var (param', _) $ arg') = Logic.dest_equals t; |
|
615 |
val _ = if head' = head then () else raise TERM ("case_cert", []); |
|
616 |
val _ = if arg' = arg then () else raise TERM ("case_cert", []); |
|
617 |
val _ = if [param'] = params then () else raise TERM ("case_cert", []); |
|
618 |
in [] end; |
|
619 |
fun analyze (cases as [let_case]) = |
|
620 |
(analyze_cases cases handle Bind => analyze_let let_case) |
|
621 |
| analyze cases = analyze_cases cases; |
|
622 |
in (case_const, (n, analyze cases)) end; |
|
623 |
||
624 |
fun case_cert thm = case_certificate thm |
|
625 |
handle Bind => error "bad case certificate" |
|
626 |
| TERM _ => error "bad case certificate"; |
|
627 |
||
31962 | 628 |
fun get_case_scheme thy = Symtab.lookup ((fst o the_cases o the_exec) thy); |
24219 | 629 |
|
31962 | 630 |
val undefineds = Symtab.keys o snd o the_cases o the_exec; |
24219 | 631 |
|
632 |
||
31962 | 633 |
(* diagnostic *) |
24219 | 634 |
|
635 |
fun print_codesetup thy = |
|
636 |
let |
|
637 |
val ctxt = ProofContext.init thy; |
|
24844
98c006a30218
certificates for code generator case expressions
haftmann
parents:
24837
diff
changeset
|
638 |
val exec = the_exec thy; |
33006 | 639 |
fun pretty_eqns (s, (_, eqns)) = |
24219 | 640 |
(Pretty.block o Pretty.fbreaks) ( |
33006 | 641 |
Pretty.str s :: map (Display.pretty_thm ctxt o fst) eqns |
24219 | 642 |
); |
643 |
fun pretty_dtyp (s, []) = |
|
644 |
Pretty.str s |
|
645 |
| pretty_dtyp (s, cos) = |
|
646 |
(Pretty.block o Pretty.breaks) ( |
|
647 |
Pretty.str s |
|
648 |
:: Pretty.str "=" |
|
31156 | 649 |
:: separate (Pretty.str "|") (map (fn (c, []) => Pretty.str (string_of_const thy c) |
24219 | 650 |
| (c, tys) => |
651 |
(Pretty.block o Pretty.breaks) |
|
31156 | 652 |
(Pretty.str (string_of_const thy c) |
26947
133905a0c493
moved global pretty/string_of functions from Sign to Syntax;
wenzelm
parents:
26928
diff
changeset
|
653 |
:: Pretty.str "of" |
133905a0c493
moved global pretty/string_of functions from Sign to Syntax;
wenzelm
parents:
26928
diff
changeset
|
654 |
:: map (Pretty.quote o Syntax.pretty_typ_global thy) tys)) cos) |
24219 | 655 |
); |
28368 | 656 |
val eqns = the_eqns exec |
24423
ae9cd0e92423
overloaded definitions accompanied by explicit constants
haftmann
parents:
24283
diff
changeset
|
657 |
|> Symtab.dest |
31156 | 658 |
|> (map o apfst) (string_of_const thy) |
28695 | 659 |
|> (map o apsnd) (snd o fst) |
24219 | 660 |
|> sort (string_ord o pairself fst); |
661 |
val dtyps = the_dtyps exec |
|
662 |
|> Symtab.dest |
|
28695 | 663 |
|> map (fn (dtco, (_, (vs, cos)) :: _) => |
31957 | 664 |
(string_of_typ thy (Type (dtco, map TFree vs)), cos)) |
24219 | 665 |
|> sort (string_ord o pairself fst) |
666 |
in |
|
667 |
(Pretty.writeln o Pretty.chunks) [ |
|
668 |
Pretty.block ( |
|
30023
55954f726043
permissive check for pattern discipline in case schemes
haftmann
parents:
29970
diff
changeset
|
669 |
Pretty.str "code equations:" |
24219 | 670 |
:: Pretty.fbrk |
33006 | 671 |
:: (Pretty.fbreaks o map pretty_eqns) eqns |
24219 | 672 |
), |
25968 | 673 |
Pretty.block ( |
24219 | 674 |
Pretty.str "datatypes:" |
675 |
:: Pretty.fbrk |
|
676 |
:: (Pretty.fbreaks o map pretty_dtyp) dtyps |
|
677 |
) |
|
678 |
] |
|
679 |
end; |
|
680 |
||
681 |
||
31962 | 682 |
(** declaring executable ingredients **) |
683 |
||
33940
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
684 |
(* constant signatures *) |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
685 |
|
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
686 |
fun add_type tyco thy = |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
687 |
case Symtab.lookup ((snd o #types o Type.rep_tsig o Sign.tsig_of) thy) tyco |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
688 |
of SOME (Type.Abbreviation (vs, _, _)) => |
34173
458ced35abb8
reduced code generator cache to the baremost minimum
haftmann
parents:
33977
diff
changeset
|
689 |
(map_exec_purge o map_signatures o apfst) |
33940
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
690 |
(Symtab.update (tyco, length vs)) thy |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
691 |
| _ => error ("No such type abbreviation: " ^ quote tyco); |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
692 |
|
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
693 |
fun add_type_cmd s thy = add_type (Sign.intern_type thy s) thy; |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
694 |
|
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
695 |
fun gen_add_signature prep_const prep_signature (raw_c, raw_ty) thy = |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
696 |
let |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
697 |
val c = prep_const thy raw_c; |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
698 |
val ty = prep_signature thy raw_ty; |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
699 |
val ty' = expand_signature thy ty; |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
700 |
val ty'' = Sign.the_const_type thy c; |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
701 |
val _ = if typ_equiv (ty', ty'') then () else |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
702 |
error ("Illegal constant signature: " ^ Syntax.string_of_typ_global thy ty); |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
703 |
in |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
704 |
thy |
34173
458ced35abb8
reduced code generator cache to the baremost minimum
haftmann
parents:
33977
diff
changeset
|
705 |
|> (map_exec_purge o map_signatures o apsnd) (Symtab.update (c, ty)) |
33940
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
706 |
end; |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
707 |
|
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
708 |
val add_signature = gen_add_signature (K I) cert_signature; |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
709 |
val add_signature_cmd = gen_add_signature read_const read_signature; |
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
710 |
|
317933ce3712
crude support for type aliasses and corresponding constant signatures
haftmann
parents:
33756
diff
changeset
|
711 |
|
31962 | 712 |
(* datatypes *) |
31090
3be41b271023
clarified matter of "proper" flag in code equations
haftmann
parents:
31088
diff
changeset
|
713 |
|
33314 | 714 |
structure Type_Interpretation = |
715 |
Interpretation(type T = string * serial val eq = eq_snd (op =) : T * T -> bool); |
|
25462 | 716 |
|
24423
ae9cd0e92423
overloaded definitions accompanied by explicit constants
haftmann
parents:
24283
diff
changeset
|
717 |
fun add_datatype raw_cs thy = |
24219 | 718 |
let |
25597
34860182b250
moved instance parameter management from class.ML to axclass.ML
haftmann
parents:
25501
diff
changeset
|
719 |
val cs = map (fn c_ty as (_, ty) => (AxClass.unoverload_const thy c_ty, ty)) raw_cs; |
31156 | 720 |
val (tyco, vs_cos) = constrset_of_consts thy cs; |
30076 | 721 |
val old_cs = (map fst o snd o get_datatype thy) tyco; |
722 |
fun drop_outdated_cases cases = fold Symtab.delete_safe |
|
723 |
(Symtab.fold (fn (c, (_, (_, cos))) => |
|
724 |
if exists (member (op =) old_cs) cos |
|
725 |
then insert (op =) c else I) cases []) cases; |
|
24219 | 726 |
in |
727 |
thy |
|
31091
8316d22f10f5
corrected deletetion of code equations for constructors
haftmann
parents:
31090
diff
changeset
|
728 |
|> fold (del_eqns o fst) cs |
34173
458ced35abb8
reduced code generator cache to the baremost minimum
haftmann
parents:
33977
diff
changeset
|
729 |
|> map_exec_purge |
28695 | 730 |
((map_dtyps o Symtab.map_default (tyco, [])) (cons (serial (), vs_cos)) |
30076 | 731 |
#> (map_cases o apfst) drop_outdated_cases) |
31962 | 732 |
|> Type_Interpretation.data (tyco, serial ()) |
24219 | 733 |
end; |
734 |
||
31962 | 735 |
fun type_interpretation f = Type_Interpretation.interpretation |
25485 | 736 |
(fn (tyco, _) => fn thy => f (tyco, get_datatype thy tyco) thy); |
737 |
||
24423
ae9cd0e92423
overloaded definitions accompanied by explicit constants
haftmann
parents:
24283
diff
changeset
|
738 |
fun add_datatype_cmd raw_cs thy = |
ae9cd0e92423
overloaded definitions accompanied by explicit constants
haftmann
parents:
24283
diff
changeset
|
739 |
let |
31156 | 740 |
val cs = map (read_bare_const thy) raw_cs; |
24423
ae9cd0e92423
overloaded definitions accompanied by explicit constants
haftmann
parents:
24283
diff
changeset
|
741 |
in add_datatype cs thy end; |
24219 | 742 |
|
31962 | 743 |
|
744 |
(* code equations *) |
|
745 |
||
33075 | 746 |
fun gen_add_eqn default (thm, proper) thy = |
747 |
let |
|
748 |
val thm' = Thm.close_derivation thm; |
|
749 |
val c = const_eqn thy thm'; |
|
750 |
in change_eqns false c (add_thm thy default (thm', proper)) thy end; |
|
31962 | 751 |
|
752 |
fun add_eqn thm thy = |
|
753 |
gen_add_eqn false (mk_eqn thy (thm, true)) thy; |
|
754 |
||
755 |
fun add_warning_eqn thm thy = |
|
756 |
case mk_eqn_warning thy thm |
|
757 |
of SOME eqn => gen_add_eqn false eqn thy |
|
758 |
| NONE => thy; |
|
759 |
||
760 |
fun add_default_eqn thm thy = |
|
761 |
case mk_eqn_liberal thy thm |
|
762 |
of SOME eqn => gen_add_eqn true eqn thy |
|
763 |
| NONE => thy; |
|
764 |
||
765 |
fun add_nbe_eqn thm thy = |
|
766 |
gen_add_eqn false (mk_eqn thy (thm, false)) thy; |
|
767 |
||
768 |
val add_default_eqn_attribute = Thm.declaration_attribute |
|
769 |
(fn thm => Context.mapping (add_default_eqn thm) I); |
|
770 |
val add_default_eqn_attrib = Attrib.internal (K add_default_eqn_attribute); |
|
771 |
||
772 |
fun del_eqn thm thy = case mk_eqn_liberal thy thm |
|
773 |
of SOME (thm, _) => change_eqns true (const_eqn thy thm) (del_thm thm) thy |
|
774 |
| NONE => thy; |
|
775 |
||
32070 | 776 |
(* c.f. src/HOL/Tools/recfun_codegen.ML *) |
777 |
||
33522 | 778 |
structure Code_Target_Attr = Theory_Data |
779 |
( |
|
31998
2c7a24f74db9
code attributes use common underscore convention
haftmann
parents:
31971
diff
changeset
|
780 |
type T = (string -> thm -> theory -> theory) option; |
2c7a24f74db9
code attributes use common underscore convention
haftmann
parents:
31971
diff
changeset
|
781 |
val empty = NONE; |
2c7a24f74db9
code attributes use common underscore convention
haftmann
parents:
31971
diff
changeset
|
782 |
val extend = I; |
33522 | 783 |
fun merge (f1, f2) = if is_some f1 then f1 else f2; |
31998
2c7a24f74db9
code attributes use common underscore convention
haftmann
parents:
31971
diff
changeset
|
784 |
); |
2c7a24f74db9
code attributes use common underscore convention
haftmann
parents:
31971
diff
changeset
|
785 |
|
32070 | 786 |
fun set_code_target_attr f = Code_Target_Attr.map (K (SOME f)); |
787 |
||
788 |
fun code_target_attr prefix thm thy = |
|
789 |
let |
|
790 |
val attr = the_default ((K o K) I) (Code_Target_Attr.get thy); |
|
791 |
in thy |> add_warning_eqn thm |> attr prefix thm end; |
|
792 |
||
793 |
(* setup *) |
|
31998
2c7a24f74db9
code attributes use common underscore convention
haftmann
parents:
31971
diff
changeset
|
794 |
|
31962 | 795 |
val _ = Context.>> (Context.map_theory |
796 |
(let |
|
797 |
fun mk_attribute f = Thm.declaration_attribute (fn thm => Context.mapping (f thm) I); |
|
31998
2c7a24f74db9
code attributes use common underscore convention
haftmann
parents:
31971
diff
changeset
|
798 |
val code_attribute_parser = |
2c7a24f74db9
code attributes use common underscore convention
haftmann
parents:
31971
diff
changeset
|
799 |
Args.del |-- Scan.succeed (mk_attribute del_eqn) |
2c7a24f74db9
code attributes use common underscore convention
haftmann
parents:
31971
diff
changeset
|
800 |
|| Args.$$$ "nbe" |-- Scan.succeed (mk_attribute add_nbe_eqn) |
2c7a24f74db9
code attributes use common underscore convention
haftmann
parents:
31971
diff
changeset
|
801 |
|| (Args.$$$ "target" |-- Args.colon |-- Args.name >> |
32070 | 802 |
(mk_attribute o code_target_attr)) |
31998
2c7a24f74db9
code attributes use common underscore convention
haftmann
parents:
31971
diff
changeset
|
803 |
|| Scan.succeed (mk_attribute add_warning_eqn); |
31962 | 804 |
in |
805 |
Type_Interpretation.init |
|
31998
2c7a24f74db9
code attributes use common underscore convention
haftmann
parents:
31971
diff
changeset
|
806 |
#> Attrib.setup (Binding.name "code") (Scan.lift code_attribute_parser) |
2c7a24f74db9
code attributes use common underscore convention
haftmann
parents:
31971
diff
changeset
|
807 |
"declare theorems for code generation" |
31962 | 808 |
end)); |
809 |
||
810 |
||
811 |
(* cases *) |
|
812 |
||
24844
98c006a30218
certificates for code generator case expressions
haftmann
parents:
24837
diff
changeset
|
813 |
fun add_case thm thy = |
98c006a30218
certificates for code generator case expressions
haftmann
parents:
24837
diff
changeset
|
814 |
let |
31156 | 815 |
val (c, (k, case_pats)) = case_cert thm; |
31088 | 816 |
val _ = case filter_out (is_constr thy) case_pats |
30076 | 817 |
of [] => () |
818 |
| cs => error ("Non-constructor(s) in case certificate: " ^ commas (map quote cs)); |
|
819 |
val entry = (1 + Int.max (1, length case_pats), (k, case_pats)) |
|
34173
458ced35abb8
reduced code generator cache to the baremost minimum
haftmann
parents:
33977
diff
changeset
|
820 |
in (map_exec_purge o map_cases o apfst) (Symtab.update (c, entry)) thy end; |
24844
98c006a30218
certificates for code generator case expressions
haftmann
parents:
24837
diff
changeset
|
821 |
|
98c006a30218
certificates for code generator case expressions
haftmann
parents:
24837
diff
changeset
|
822 |
fun add_undefined c thy = |
34173
458ced35abb8
reduced code generator cache to the baremost minimum
haftmann
parents:
33977
diff
changeset
|
823 |
(map_exec_purge o map_cases o apsnd) (Symtab.update (c, ())) thy; |
24844
98c006a30218
certificates for code generator case expressions
haftmann
parents:
24837
diff
changeset
|
824 |
|
24219 | 825 |
end; (*struct*) |
826 |
||
827 |
||
32661
f4d179d91af2
experimenting to add some useful interface for definitions
bulwahn
parents:
32640
diff
changeset
|
828 |
(** type-safe interfaces for data dependent on executable code **) |
24219 | 829 |
|
34173
458ced35abb8
reduced code generator cache to the baremost minimum
haftmann
parents:
33977
diff
changeset
|
830 |
functor Code_Data(Data: CODE_DATA_ARGS): CODE_DATA = |
24219 | 831 |
struct |
832 |
||
833 |
type T = Data.T; |
|
834 |
exception Data of T; |
|
835 |
fun dest (Data x) = x |
|
836 |
||
34173
458ced35abb8
reduced code generator cache to the baremost minimum
haftmann
parents:
33977
diff
changeset
|
837 |
val kind = Code.declare_data (Data Data.empty); |
24219 | 838 |
|
839 |
val data_op = (kind, Data, dest); |
|
840 |
||
841 |
val change = Code.change_data data_op; |
|
842 |
fun change_yield thy = Code.change_yield_data data_op thy; |
|
843 |
||
844 |
end; |
|
845 |
||
28143 | 846 |
structure Code : CODE = struct open Code; end; |