author | paulson |
Wed, 08 May 1996 17:57:05 +0200 | |
changeset 1736 | fe0b459273f2 |
parent 1627 | 64ee96ebf32a |
child 2148 | 7ef2987da18f |
permissions | -rw-r--r-- |
256 | 1 |
(* Title: Pure/type.ML |
0 | 2 |
ID: $Id$ |
416 | 3 |
Author: Tobias Nipkow & Lawrence C Paulson |
0 | 4 |
|
416 | 5 |
Type classes and sorts. Type signatures. Type unification and inference. |
256 | 6 |
|
7 |
TODO: |
|
1257 | 8 |
improve nonempty_sort! |
416 | 9 |
move type unification and inference to type_unify.ML (TypeUnify) (?) |
0 | 10 |
*) |
11 |
||
12 |
signature TYPE = |
|
1504 | 13 |
sig |
14 |
exception TUNIFY |
|
15 |
exception TYPE_MATCH |
|
621 | 16 |
val no_tvars: typ -> typ |
17 |
val varifyT: typ -> typ |
|
18 |
val unvarifyT: typ -> typ |
|
19 |
val varify: term * string list -> term |
|
416 | 20 |
val str_of_sort: sort -> string |
21 |
val str_of_arity: string * sort list * sort -> string |
|
0 | 22 |
type type_sig |
200 | 23 |
val rep_tsig: type_sig -> |
256 | 24 |
{classes: class list, |
25 |
subclass: (class * class list) list, |
|
26 |
default: sort, |
|
963 | 27 |
tycons: (string * int) list, |
621 | 28 |
abbrs: (string * (string list * typ)) list, |
963 | 29 |
arities: (string * (class * sort list) list) list} |
0 | 30 |
val defaultS: type_sig -> sort |
416 | 31 |
val tsig0: type_sig |
256 | 32 |
val logical_types: type_sig -> string list |
621 | 33 |
val ext_tsig_classes: type_sig -> (class * class list) list -> type_sig |
422 | 34 |
val ext_tsig_subclass: type_sig -> (class * class) list -> type_sig |
35 |
val ext_tsig_defsort: type_sig -> sort -> type_sig |
|
582 | 36 |
val ext_tsig_types: type_sig -> (string * int) list -> type_sig |
621 | 37 |
val ext_tsig_abbrs: type_sig -> (string * string list * typ) list -> type_sig |
963 | 38 |
val ext_tsig_arities: type_sig -> (string * sort list * sort)list -> type_sig |
256 | 39 |
val merge_tsigs: type_sig * type_sig -> type_sig |
416 | 40 |
val subsort: type_sig -> sort * sort -> bool |
41 |
val norm_sort: type_sig -> sort -> sort |
|
42 |
val rem_sorts: typ -> typ |
|
1239 | 43 |
val nonempty_sort: type_sig -> sort list -> sort -> bool |
256 | 44 |
val cert_typ: type_sig -> typ -> typ |
45 |
val norm_typ: type_sig -> typ -> typ |
|
949
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
46 |
val freeze: term -> term |
0 | 47 |
val freeze_vars: typ -> typ |
949
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
48 |
val infer_types: type_sig * (string -> typ option) * |
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
49 |
(indexname -> typ option) * (indexname -> sort option) * |
1392
1b4ae50e0e0a
infer_types now takes a term list and a type list as argument. It
paulson
parents:
1257
diff
changeset
|
50 |
string list * bool * typ list * term list |
1b4ae50e0e0a
infer_types now takes a term list and a type list as argument. It
paulson
parents:
1257
diff
changeset
|
51 |
-> term list * (indexname * typ) list |
256 | 52 |
val inst_term_tvars: type_sig * (indexname * typ) list -> term -> term |
0 | 53 |
val thaw_vars: typ -> typ |
256 | 54 |
val typ_errors: type_sig -> typ * string list -> string list |
0 | 55 |
val typ_instance: type_sig * typ * typ -> bool |
256 | 56 |
val typ_match: type_sig -> (indexname * typ) list * (typ * typ) |
57 |
-> (indexname * typ) list |
|
1435
aefcd255ed4a
Removed bug in type unification. Negative indexes are not used any longer.
nipkow
parents:
1392
diff
changeset
|
58 |
val unify: type_sig -> int -> (indexname * typ) list -> (typ * typ) |
aefcd255ed4a
Removed bug in type unification. Negative indexes are not used any longer.
nipkow
parents:
1392
diff
changeset
|
59 |
-> (indexname * typ) list * int |
450 | 60 |
val raw_unify: typ * typ -> bool |
1504 | 61 |
end; |
0 | 62 |
|
1504 | 63 |
structure Type : TYPE = |
0 | 64 |
struct |
65 |
||
621 | 66 |
(*** TFrees vs TVars ***) |
67 |
||
68 |
(*disallow TVars*) |
|
69 |
fun no_tvars T = |
|
70 |
if null (typ_tvars T) then T |
|
71 |
else raise_type "Illegal schematic type variable(s)" [T] []; |
|
72 |
||
73 |
(*turn TFrees into TVars to allow types & axioms to be written without "?"*) |
|
949
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
74 |
val varifyT = map_type_tfree (fn (a, S) => TVar((a, 0), S)); |
621 | 75 |
|
76 |
(*inverse of varifyT*) |
|
77 |
fun unvarifyT (Type (a, Ts)) = Type (a, map unvarifyT Ts) |
|
78 |
| unvarifyT (TVar ((a, 0), S)) = TFree (a, S) |
|
79 |
| unvarifyT T = T; |
|
80 |
||
81 |
(*turn TFrees except those in fixed into new TVars*) |
|
82 |
fun varify (t, fixed) = |
|
83 |
let |
|
84 |
val fs = add_term_tfree_names (t, []) \\ fixed; |
|
85 |
val ixns = add_term_tvar_ixns (t, []); |
|
86 |
val fmap = fs ~~ variantlist (fs, map #1 ixns) |
|
949
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
87 |
fun thaw(f as (a,S)) = case assoc (fmap, a) of |
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
88 |
None => TFree(f) |
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
89 |
| Some b => TVar((b, 0), S) |
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
90 |
in map_term_types (map_type_tfree thaw) t end; |
621 | 91 |
|
92 |
||
93 |
||
416 | 94 |
(*** type classes and sorts ***) |
95 |
||
96 |
(* |
|
97 |
Classes denote (possibly empty) collections of types (e.g. sets of types) |
|
98 |
and are partially ordered by 'inclusion'. They are represented by strings. |
|
99 |
||
100 |
Sorts are intersections of finitely many classes. They are represented by |
|
101 |
lists of classes. |
|
102 |
*) |
|
0 | 103 |
|
104 |
type domain = sort list; |
|
416 | 105 |
|
106 |
||
107 |
(* print sorts and arities *) |
|
0 | 108 |
|
416 | 109 |
fun str_of_sort [c] = c |
565 | 110 |
| str_of_sort cs = enclose "{" "}" (commas cs); |
416 | 111 |
|
565 | 112 |
fun str_of_dom dom = enclose "(" ")" (commas (map str_of_sort dom)); |
416 | 113 |
|
114 |
fun str_of_arity (t, [], S) = t ^ " :: " ^ str_of_sort S |
|
115 |
| str_of_arity (t, SS, S) = |
|
116 |
t ^ " :: " ^ str_of_dom SS ^ " " ^ str_of_sort S; |
|
256 | 117 |
|
118 |
||
119 |
||
416 | 120 |
(*** type signatures ***) |
256 | 121 |
|
122 |
(* |
|
123 |
classes: |
|
124 |
a list of all declared classes; |
|
0 | 125 |
|
256 | 126 |
subclass: |
416 | 127 |
an association list representing the subclass relation; (c, cs) is |
256 | 128 |
interpreted as "c is a proper subclass of all elemenst of cs"; note that |
129 |
c itself is not a memeber of cs; |
|
130 |
||
131 |
default: |
|
132 |
the default sort attached to all unconstrained type vars; |
|
133 |
||
963 | 134 |
tycons: |
256 | 135 |
an association list of all declared types with the number of their |
136 |
arguments; |
|
137 |
||
138 |
abbrs: |
|
139 |
an association list of type abbreviations; |
|
140 |
||
963 | 141 |
arities: |
256 | 142 |
a two-fold association list of all type arities; (t, al) means that type |
143 |
constructor t has the arities in al; an element (c, ss) of al represents |
|
144 |
the arity (ss)c; |
|
0 | 145 |
*) |
146 |
||
256 | 147 |
datatype type_sig = |
148 |
TySg of { |
|
149 |
classes: class list, |
|
150 |
subclass: (class * class list) list, |
|
151 |
default: sort, |
|
963 | 152 |
tycons: (string * int) list, |
621 | 153 |
abbrs: (string * (string list * typ)) list, |
963 | 154 |
arities: (string * (class * domain) list) list}; |
256 | 155 |
|
189 | 156 |
fun rep_tsig (TySg comps) = comps; |
0 | 157 |
|
256 | 158 |
fun defaultS (TySg {default, ...}) = default; |
159 |
||
160 |
||
582 | 161 |
(* error messages *) |
256 | 162 |
|
416 | 163 |
fun undcl_class c = "Undeclared class " ^ quote c; |
256 | 164 |
val err_undcl_class = error o undcl_class; |
0 | 165 |
|
422 | 166 |
fun err_dup_classes cs = |
167 |
error ("Duplicate declaration of class(es) " ^ commas_quote cs); |
|
416 | 168 |
|
169 |
fun undcl_type c = "Undeclared type constructor " ^ quote c; |
|
256 | 170 |
val err_undcl_type = error o undcl_type; |
171 |
||
582 | 172 |
fun err_neg_args c = |
173 |
error ("Negative number of arguments of type constructor " ^ quote c); |
|
174 |
||
416 | 175 |
fun err_dup_tycon c = |
176 |
error ("Duplicate declaration of type constructor " ^ quote c); |
|
177 |
||
621 | 178 |
fun dup_tyabbrs ts = |
179 |
"Duplicate declaration of type abbreviation(s) " ^ commas_quote ts; |
|
416 | 180 |
|
181 |
fun ty_confl c = "Conflicting type constructor and abbreviation " ^ quote c; |
|
182 |
val err_ty_confl = error o ty_confl; |
|
0 | 183 |
|
184 |
||
185 |
(* 'leq' checks the partial order on classes according to the |
|
621 | 186 |
statements in the association list 'a' (i.e. 'subclass') |
0 | 187 |
*) |
188 |
||
256 | 189 |
fun less a (C, D) = case assoc (a, C) of |
621 | 190 |
Some ss => D mem ss |
191 |
| None => err_undcl_class C; |
|
0 | 192 |
|
256 | 193 |
fun leq a (C, D) = C = D orelse less a (C, D); |
0 | 194 |
|
195 |
||
416 | 196 |
(* logical_types *) |
0 | 197 |
|
416 | 198 |
(*return all logical types of tsig, i.e. all types t with some arity t::(ss)c |
199 |
and c <= logic*) |
|
0 | 200 |
|
416 | 201 |
fun logical_types tsig = |
202 |
let |
|
963 | 203 |
val TySg {subclass, arities, tycons, ...} = tsig; |
416 | 204 |
|
205 |
fun log_class c = leq subclass (c, logicC); |
|
963 | 206 |
fun log_type t = exists (log_class o #1) (assocs arities t); |
416 | 207 |
in |
963 | 208 |
filter log_type (map #1 tycons) |
0 | 209 |
end; |
210 |
||
162 | 211 |
|
256 | 212 |
(* 'sortorder' checks the ordering on sets of classes, i.e. on sorts: |
213 |
S1 <= S2 , iff for every class C2 in S2 there exists a class C1 in S1 |
|
0 | 214 |
with C1 <= C2 (according to an association list 'a') |
215 |
*) |
|
216 |
||
256 | 217 |
fun sortorder a (S1, S2) = |
218 |
forall (fn C2 => exists (fn C1 => leq a (C1, C2)) S1) S2; |
|
0 | 219 |
|
220 |
||
221 |
(* 'inj' inserts a new class C into a given class set S (i.e.sort) only if |
|
222 |
there exists no class in S which is <= C; |
|
223 |
the resulting set is minimal if S was minimal |
|
224 |
*) |
|
225 |
||
256 | 226 |
fun inj a (C, S) = |
0 | 227 |
let fun inj1 [] = [C] |
256 | 228 |
| inj1 (D::T) = if leq a (D, C) then D::T |
229 |
else if leq a (C, D) then inj1 T |
|
0 | 230 |
else D::(inj1 T) |
231 |
in inj1 S end; |
|
232 |
||
233 |
||
234 |
(* 'union_sort' forms the minimal union set of two sorts S1 and S2 |
|
235 |
under the assumption that S2 is minimal *) |
|
256 | 236 |
(* FIXME rename to inter_sort (?) *) |
0 | 237 |
|
238 |
fun union_sort a = foldr (inj a); |
|
239 |
||
240 |
||
241 |
(* 'elementwise_union' forms elementwise the minimal union set of two |
|
242 |
sort lists under the assumption that the two lists have the same length |
|
256 | 243 |
*) |
0 | 244 |
|
256 | 245 |
fun elementwise_union a (Ss1, Ss2) = map (union_sort a) (Ss1~~Ss2); |
246 |
||
0 | 247 |
|
248 |
(* 'lew' checks for two sort lists the ordering for all corresponding list |
|
249 |
elements (i.e. sorts) *) |
|
250 |
||
256 | 251 |
fun lew a (w1, w2) = forall (sortorder a) (w1~~w2); |
252 |
||
0 | 253 |
|
256 | 254 |
(* 'is_min' checks if a class C is minimal in a given sort S under the |
255 |
assumption that S contains C *) |
|
0 | 256 |
|
256 | 257 |
fun is_min a S C = not (exists (fn (D) => less a (D, C)) S); |
0 | 258 |
|
259 |
||
260 |
(* 'min_sort' reduces a sort to its minimal classes *) |
|
261 |
||
262 |
fun min_sort a S = distinct(filter (is_min a S) S); |
|
263 |
||
264 |
||
265 |
(* 'min_domain' minimizes the domain sorts of type declarationsl; |
|
256 | 266 |
the function will be applied on the type declarations in extensions *) |
0 | 267 |
|
268 |
fun min_domain subclass = |
|
256 | 269 |
let fun one_min (f, (doms, ran)) = (f, (map (min_sort subclass) doms, ran)) |
0 | 270 |
in map one_min end; |
271 |
||
272 |
||
273 |
(* 'min_filter' filters a list 'ars' consisting of arities (domain * class) |
|
256 | 274 |
and gives back a list of those range classes whose domains meet the |
0 | 275 |
predicate 'pred' *) |
256 | 276 |
|
0 | 277 |
fun min_filter a pred ars = |
256 | 278 |
let fun filt ([], l) = l |
279 |
| filt ((c, x)::xs, l) = if pred(x) then filt (xs, inj a (c, l)) |
|
280 |
else filt (xs, l) |
|
281 |
in filt (ars, []) end; |
|
0 | 282 |
|
283 |
||
284 |
(* 'cod_above' filters all arities whose domains are elementwise >= than |
|
256 | 285 |
a given domain 'w' and gives back a list of the corresponding range |
0 | 286 |
classes *) |
287 |
||
256 | 288 |
fun cod_above (a, w, ars) = min_filter a (fn w' => lew a (w, w')) ars; |
289 |
||
290 |
||
0 | 291 |
|
200 | 292 |
(*Instantiation of type variables in types*) |
293 |
(*Pre: instantiations obey restrictions! *) |
|
294 |
fun inst_typ tye = |
|
949
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
295 |
let fun inst(var as (v, _)) = case assoc(tye, v) of |
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
296 |
Some U => inst_typ tye U |
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
297 |
| None => TVar(var) |
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
298 |
in map_type_tvar inst end; |
0 | 299 |
|
300 |
(* 'least_sort' returns for a given type its maximum sort: |
|
301 |
- type variables, free types: the sort brought with |
|
302 |
- type constructors: recursive determination of the maximum sort of the |
|
963 | 303 |
arguments if the type is declared in 'arities' of the |
256 | 304 |
given type signature *) |
0 | 305 |
|
963 | 306 |
fun least_sort (tsig as TySg{subclass, arities, ...}) = |
256 | 307 |
let fun ls(T as Type(a, Ts)) = |
963 | 308 |
(case assoc (arities, a) of |
256 | 309 |
Some(ars) => cod_above(subclass, map ls Ts, ars) |
310 |
| None => raise TYPE(undcl_type a, [T], [])) |
|
311 |
| ls(TFree(a, S)) = S |
|
312 |
| ls(TVar(a, S)) = S |
|
0 | 313 |
in ls end; |
314 |
||
315 |
||
963 | 316 |
fun check_has_sort(tsig as TySg{subclass, arities, ...}, T, S) = |
256 | 317 |
if sortorder subclass ((least_sort tsig T), S) then () |
318 |
else raise TYPE("Type not of sort " ^ (str_of_sort S), [T], []) |
|
0 | 319 |
|
320 |
||
321 |
(*Instantiation of type variables in types *) |
|
256 | 322 |
fun inst_typ_tvars(tsig, tye) = |
949
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
323 |
let fun inst(var as (v, S)) = case assoc(tye, v) of |
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
324 |
Some U => (check_has_sort(tsig, U, S); U) |
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
325 |
| None => TVar(var) |
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
326 |
in map_type_tvar inst end; |
0 | 327 |
|
328 |
(*Instantiation of type variables in terms *) |
|
256 | 329 |
fun inst_term_tvars(tsig, tye) = map_term_types (inst_typ_tvars(tsig, tye)); |
200 | 330 |
|
331 |
||
1484 | 332 |
(* norm_typ *) |
200 | 333 |
|
1484 | 334 |
fun norm_typ (TySg {abbrs, ...}) ty = |
256 | 335 |
let |
621 | 336 |
val idx = maxidx_of_typ ty + 1; |
337 |
||
338 |
fun expand (Type (a, Ts)) = |
|
256 | 339 |
(case assoc (abbrs, a) of |
621 | 340 |
Some (vs, U) => |
341 |
expand (inst_typ (map (rpair idx) vs ~~ Ts) (incr_tvar idx U)) |
|
342 |
| None => Type (a, map expand Ts)) |
|
343 |
| expand T = T |
|
256 | 344 |
in |
621 | 345 |
expand ty |
256 | 346 |
end; |
347 |
||
348 |
||
349 |
(** type matching **) |
|
200 | 350 |
|
0 | 351 |
exception TYPE_MATCH; |
352 |
||
256 | 353 |
(*typ_match (s, (U, T)) = s' <==> s'(U) = T and s' is an extension of s*) |
354 |
fun typ_match tsig = |
|
355 |
let |
|
356 |
fun match (subs, (TVar (v, S), T)) = |
|
357 |
(case assoc (subs, v) of |
|
358 |
None => ((v, (check_has_sort (tsig, T, S); T)) :: subs |
|
359 |
handle TYPE _ => raise TYPE_MATCH) |
|
422 | 360 |
| Some U => if U = T then subs else raise TYPE_MATCH) |
256 | 361 |
| match (subs, (Type (a, Ts), Type (b, Us))) = |
362 |
if a <> b then raise TYPE_MATCH |
|
363 |
else foldl match (subs, Ts ~~ Us) |
|
422 | 364 |
| match (subs, (TFree x, TFree y)) = |
256 | 365 |
if x = y then subs else raise TYPE_MATCH |
366 |
| match _ = raise TYPE_MATCH; |
|
367 |
in match end; |
|
0 | 368 |
|
369 |
||
256 | 370 |
fun typ_instance (tsig, T, U) = |
371 |
(typ_match tsig ([], (U, T)); true) handle TYPE_MATCH => false; |
|
372 |
||
373 |
||
374 |
||
375 |
(** build type signatures **) |
|
376 |
||
963 | 377 |
fun make_tsig (classes, subclass, default, tycons, abbrs, arities) = |
416 | 378 |
TySg {classes = classes, subclass = subclass, default = default, |
963 | 379 |
tycons = tycons, abbrs = abbrs, arities = arities}; |
416 | 380 |
|
381 |
val tsig0 = make_tsig ([], [], [], [], [], []); |
|
256 | 382 |
|
0 | 383 |
|
401 | 384 |
(* sorts *) |
385 |
||
416 | 386 |
fun subsort (TySg {subclass, ...}) (S1, S2) = |
387 |
sortorder subclass (S1, S2); |
|
388 |
||
401 | 389 |
fun norm_sort (TySg {subclass, ...}) S = |
390 |
sort_strings (min_sort subclass S); |
|
391 |
||
416 | 392 |
fun rem_sorts (Type (a, tys)) = Type (a, map rem_sorts tys) |
393 |
| rem_sorts (TFree (x, _)) = TFree (x, []) |
|
394 |
| rem_sorts (TVar (xi, _)) = TVar (xi, []); |
|
401 | 395 |
|
396 |
||
1215
a206f722bef9
added nonempty_sort (a somewhat braindead version!);
wenzelm
parents:
963
diff
changeset
|
397 |
(* nonempty_sort *) |
a206f722bef9
added nonempty_sort (a somewhat braindead version!);
wenzelm
parents:
963
diff
changeset
|
398 |
|
a206f722bef9
added nonempty_sort (a somewhat braindead version!);
wenzelm
parents:
963
diff
changeset
|
399 |
(* FIXME improve: proper sorts; non-base, non-ground types (vars from hyps) *) |
a206f722bef9
added nonempty_sort (a somewhat braindead version!);
wenzelm
parents:
963
diff
changeset
|
400 |
fun nonempty_sort _ _ [] = true |
a206f722bef9
added nonempty_sort (a somewhat braindead version!);
wenzelm
parents:
963
diff
changeset
|
401 |
| nonempty_sort (tsig as TySg {arities, ...}) hyps S = |
a206f722bef9
added nonempty_sort (a somewhat braindead version!);
wenzelm
parents:
963
diff
changeset
|
402 |
exists (exists (fn (c, ss) => [c] = S andalso null ss) o snd) arities |
1239 | 403 |
orelse exists (fn S' => subsort tsig (S', S)) hyps; |
1215
a206f722bef9
added nonempty_sort (a somewhat braindead version!);
wenzelm
parents:
963
diff
changeset
|
404 |
|
a206f722bef9
added nonempty_sort (a somewhat braindead version!);
wenzelm
parents:
963
diff
changeset
|
405 |
|
a206f722bef9
added nonempty_sort (a somewhat braindead version!);
wenzelm
parents:
963
diff
changeset
|
406 |
|
416 | 407 |
(* typ_errors *) |
256 | 408 |
|
416 | 409 |
(*check validity of (not necessarily normal) type; accumulate error messages*) |
256 | 410 |
|
416 | 411 |
fun typ_errors tsig (typ, errors) = |
256 | 412 |
let |
963 | 413 |
val TySg {classes, tycons, abbrs, ...} = tsig; |
416 | 414 |
|
415 |
fun class_err (errs, c) = |
|
416 |
if c mem classes then errs |
|
417 |
else undcl_class c ins errs; |
|
256 | 418 |
|
419 |
val sort_err = foldl class_err; |
|
0 | 420 |
|
256 | 421 |
fun typ_errs (Type (c, Us), errs) = |
422 |
let |
|
423 |
val errs' = foldr typ_errs (Us, errs); |
|
424 |
fun nargs n = |
|
425 |
if n = length Us then errs' |
|
416 | 426 |
else ("Wrong number of arguments: " ^ quote c) ins errs'; |
256 | 427 |
in |
963 | 428 |
(case assoc (tycons, c) of |
256 | 429 |
Some n => nargs n |
430 |
| None => |
|
431 |
(case assoc (abbrs, c) of |
|
432 |
Some (vs, _) => nargs (length vs) |
|
416 | 433 |
| None => undcl_type c ins errs)) |
256 | 434 |
end |
435 |
| typ_errs (TFree (_, S), errs) = sort_err (errs, S) |
|
416 | 436 |
| typ_errs (TVar ((x, i), S), errs) = |
437 |
if i < 0 then |
|
438 |
("Negative index for TVar " ^ quote x) ins sort_err (errs, S) |
|
439 |
else sort_err (errs, S); |
|
256 | 440 |
in |
416 | 441 |
typ_errs (typ, errors) |
256 | 442 |
end; |
443 |
||
444 |
||
445 |
(* cert_typ *) |
|
446 |
||
447 |
(*check and normalize typ wrt. tsig; errors are indicated by exception TYPE*) |
|
448 |
||
449 |
fun cert_typ tsig ty = |
|
450 |
(case typ_errors tsig (ty, []) of |
|
451 |
[] => norm_typ tsig ty |
|
452 |
| errs => raise_type (cat_lines errs) [ty] []); |
|
453 |
||
454 |
||
455 |
||
422 | 456 |
(** merge type signatures **) |
256 | 457 |
|
422 | 458 |
(*'assoc_union' merges two association lists if the contents associated |
459 |
the keys are lists*) |
|
0 | 460 |
|
422 | 461 |
fun assoc_union (as1, []) = as1 |
462 |
| assoc_union (as1, (key, l2) :: as2) = |
|
463 |
(case assoc (as1, key) of |
|
464 |
Some l1 => assoc_union (overwrite (as1, (key, l1 union l2)), as2) |
|
465 |
| None => assoc_union ((key, l2) :: as1, as2)); |
|
0 | 466 |
|
467 |
||
422 | 468 |
(* merge subclass *) |
0 | 469 |
|
422 | 470 |
fun merge_subclass (subclass1, subclass2) = |
471 |
let val subclass = transitive_closure (assoc_union (subclass1, subclass2)) in |
|
472 |
if exists (op mem) subclass then |
|
473 |
error ("Cyclic class structure!") (* FIXME improve msg, raise TERM *) |
|
474 |
else subclass |
|
416 | 475 |
end; |
476 |
||
477 |
||
422 | 478 |
(* coregularity *) |
0 | 479 |
|
480 |
(* 'is_unique_decl' checks if there exists just one declaration t:(Ss)C *) |
|
481 |
||
963 | 482 |
fun is_unique_decl ars (t,(C,w)) = case assoc (ars, C) of |
0 | 483 |
Some(w1) => if w = w1 then () else |
256 | 484 |
error("There are two declarations\n" ^ |
963 | 485 |
str_of_arity(t, w, [C]) ^ " and\n" ^ |
486 |
str_of_arity(t, w1, [C]) ^ "\n" ^ |
|
0 | 487 |
"with the same result class.") |
488 |
| None => (); |
|
489 |
||
963 | 490 |
(* 'coreg' checks if there are two declarations t:(Ss1)C1 and t:(Ss2)C2 |
0 | 491 |
such that C1 >= C2 then Ss1 >= Ss2 (elementwise) *) |
492 |
||
963 | 493 |
fun coreg_err(t, (C1,w1), (C2,w2)) = |
494 |
error("Declarations " ^ str_of_arity(t, w1, [C1]) ^ " and " |
|
495 |
^ str_of_arity(t, w2, [C2]) ^ " are in conflict"); |
|
0 | 496 |
|
963 | 497 |
fun coreg subclass (t, Cw1) = |
498 |
let fun check1(Cw1 as (C1,w1), Cw2 as (C2,w2)) = |
|
499 |
if leq subclass (C1,C2) |
|
500 |
then if lew subclass (w1,w2) then () else coreg_err(t, Cw1, Cw2) |
|
501 |
else () |
|
502 |
fun check(Cw2) = (check1(Cw1,Cw2); check1(Cw2,Cw1)) |
|
503 |
in seq check end; |
|
0 | 504 |
|
963 | 505 |
fun add_arity subclass ars (tCw as (_,Cw)) = |
506 |
(is_unique_decl ars tCw; coreg subclass tCw ars; Cw ins ars); |
|
0 | 507 |
|
256 | 508 |
fun varying_decls t = |
509 |
error ("Type constructor " ^ quote t ^ " has varying number of arguments"); |
|
0 | 510 |
|
511 |
||
963 | 512 |
(* 'merge_arities' builds the union of two 'arities' lists; |
422 | 513 |
it only checks the two restriction conditions and inserts afterwards |
514 |
all elements of the second list into the first one *) |
|
515 |
||
963 | 516 |
fun merge_arities subclass = |
517 |
let fun test_ar t (ars1, sw) = add_arity subclass ars1 (t,sw); |
|
422 | 518 |
|
963 | 519 |
fun merge_c (arities1, (c as (t, ars2))) = case assoc (arities1, t) of |
520 |
Some(ars1) => |
|
521 |
let val ars = foldl (test_ar t) (ars1, ars2) |
|
522 |
in overwrite (arities1, (t,ars)) end |
|
523 |
| None => c::arities1 |
|
422 | 524 |
in foldl merge_c end; |
525 |
||
963 | 526 |
fun add_tycons (tycons, tn as (t,n)) = |
527 |
(case assoc (tycons, t) of |
|
528 |
Some m => if m = n then tycons else varying_decls t |
|
529 |
| None => tn :: tycons); |
|
422 | 530 |
|
531 |
fun merge_abbrs (abbrs1, abbrs2) = |
|
621 | 532 |
let val abbrs = abbrs1 union abbrs2 in |
533 |
(case gen_duplicates eq_fst abbrs of |
|
422 | 534 |
[] => abbrs |
621 | 535 |
| dups => raise_term (dup_tyabbrs (map fst dups)) []) |
422 | 536 |
end; |
537 |
||
538 |
||
539 |
(* 'merge_tsigs' takes the above declared functions to merge two type |
|
540 |
signatures *) |
|
541 |
||
963 | 542 |
fun merge_tsigs(TySg{classes=classes1, default=default1, subclass=subclass1, |
543 |
tycons=tycons1, arities=arities1, abbrs=abbrs1}, |
|
544 |
TySg{classes=classes2, default=default2, subclass=subclass2, |
|
545 |
tycons=tycons2, arities=arities2, abbrs=abbrs2}) = |
|
422 | 546 |
let val classes' = classes1 union classes2; |
547 |
val subclass' = merge_subclass (subclass1, subclass2); |
|
963 | 548 |
val tycons' = foldl add_tycons (tycons1, tycons2) |
549 |
val arities' = merge_arities subclass' (arities1, arities2); |
|
422 | 550 |
val default' = min_sort subclass' (default1 @ default2); |
551 |
val abbrs' = merge_abbrs(abbrs1, abbrs2); |
|
963 | 552 |
in make_tsig(classes', subclass', default', tycons', abbrs', arities') end; |
422 | 553 |
|
554 |
||
555 |
||
556 |
(*** extend type signatures ***) |
|
557 |
||
621 | 558 |
(** add classes and subclass relations**) |
422 | 559 |
|
560 |
fun add_classes classes cs = |
|
561 |
(case cs inter classes of |
|
562 |
[] => cs @ classes |
|
563 |
| dups => err_dup_classes cs); |
|
564 |
||
565 |
||
566 |
(*'add_subclass' adds a tuple consisting of a new class (the new class has |
|
567 |
already been inserted into the 'classes' list) and its superclasses (they |
|
568 |
must be declared in 'classes' too) to the 'subclass' list of the given type |
|
569 |
signature; furthermore all inherited superclasses according to the |
|
570 |
superclasses brought with are inserted and there is a check that there are |
|
571 |
no cycles (i.e. C <= D <= C, with C <> D);*) |
|
572 |
||
573 |
fun add_subclass classes (subclass, (s, ges)) = |
|
621 | 574 |
let |
575 |
fun upd (subclass, s') = |
|
576 |
if s' mem classes then |
|
422 | 577 |
let val ges' = the (assoc (subclass, s)) |
578 |
in case assoc (subclass, s') of |
|
579 |
Some sups => if s mem sups |
|
580 |
then error(" Cycle :" ^ s^" <= "^ s'^" <= "^ s ) |
|
581 |
else overwrite (subclass, (s, sups union ges')) |
|
582 |
| None => subclass |
|
621 | 583 |
end |
584 |
else err_undcl_class s' |
|
585 |
in foldl upd (subclass @ [(s, ges)], ges) end; |
|
422 | 586 |
|
587 |
||
588 |
(* 'extend_classes' inserts all new classes into the corresponding |
|
589 |
lists ('classes', 'subclass') if possible *) |
|
590 |
||
621 | 591 |
fun extend_classes (classes, subclass, new_classes) = |
592 |
let |
|
593 |
val classes' = add_classes classes (map fst new_classes); |
|
594 |
val subclass' = foldl (add_subclass classes') (subclass, new_classes); |
|
422 | 595 |
in (classes', subclass') end; |
596 |
||
597 |
||
621 | 598 |
(* ext_tsig_classes *) |
599 |
||
600 |
fun ext_tsig_classes tsig new_classes = |
|
601 |
let |
|
963 | 602 |
val TySg {classes, subclass, default, tycons, abbrs, arities} = tsig; |
603 |
val (classes',subclass') = extend_classes (classes,subclass,new_classes); |
|
621 | 604 |
in |
963 | 605 |
make_tsig (classes', subclass', default, tycons, abbrs, arities) |
621 | 606 |
end; |
607 |
||
608 |
||
422 | 609 |
(* ext_tsig_subclass *) |
610 |
||
611 |
fun ext_tsig_subclass tsig pairs = |
|
612 |
let |
|
963 | 613 |
val TySg {classes, subclass, default, tycons, abbrs, arities} = tsig; |
422 | 614 |
|
615 |
(* FIXME clean! *) |
|
616 |
val subclass' = |
|
617 |
merge_subclass (subclass, map (fn (c1, c2) => (c1, [c2])) pairs); |
|
618 |
in |
|
963 | 619 |
make_tsig (classes, subclass', default, tycons, abbrs, arities) |
422 | 620 |
end; |
621 |
||
622 |
||
623 |
(* ext_tsig_defsort *) |
|
624 |
||
963 | 625 |
fun ext_tsig_defsort(TySg{classes,subclass,tycons,abbrs,arities,...}) default = |
626 |
make_tsig (classes, subclass, default, tycons, abbrs, arities); |
|
422 | 627 |
|
628 |
||
629 |
||
621 | 630 |
(** add types **) |
582 | 631 |
|
963 | 632 |
fun ext_tsig_types (TySg {classes, subclass, default, tycons, abbrs, arities}) ts = |
582 | 633 |
let |
634 |
fun check_type (c, n) = |
|
635 |
if n < 0 then err_neg_args c |
|
963 | 636 |
else if is_some (assoc (tycons, c)) then err_dup_tycon c |
582 | 637 |
else if is_some (assoc (abbrs, c)) then err_ty_confl c |
638 |
else (); |
|
639 |
in |
|
640 |
seq check_type ts; |
|
963 | 641 |
make_tsig (classes, subclass, default, ts @ tycons, abbrs, |
642 |
map (rpair [] o #1) ts @ arities) |
|
582 | 643 |
end; |
644 |
||
645 |
||
646 |
||
647 |
(** add type abbreviations **) |
|
648 |
||
649 |
fun abbr_errors tsig (a, (lhs_vs, rhs)) = |
|
650 |
let |
|
963 | 651 |
val TySg {tycons, abbrs, ...} = tsig; |
621 | 652 |
val rhs_vs = map (#1 o #1) (typ_tvars rhs); |
582 | 653 |
|
654 |
val dup_lhs_vars = |
|
655 |
(case duplicates lhs_vs of |
|
656 |
[] => [] |
|
621 | 657 |
| vs => ["Duplicate variables on lhs: " ^ commas_quote vs]); |
582 | 658 |
|
659 |
val extra_rhs_vars = |
|
660 |
(case gen_rems (op =) (rhs_vs, lhs_vs) of |
|
661 |
[] => [] |
|
621 | 662 |
| vs => ["Extra variables on rhs: " ^ commas_quote vs]); |
582 | 663 |
|
664 |
val tycon_confl = |
|
963 | 665 |
if is_none (assoc (tycons, a)) then [] |
582 | 666 |
else [ty_confl a]; |
667 |
||
668 |
val dup_abbr = |
|
669 |
if is_none (assoc (abbrs, a)) then [] |
|
670 |
else ["Duplicate declaration of abbreviation"]; |
|
671 |
in |
|
672 |
dup_lhs_vars @ extra_rhs_vars @ tycon_confl @ dup_abbr @ |
|
673 |
typ_errors tsig (rhs, []) |
|
674 |
end; |
|
675 |
||
621 | 676 |
fun prep_abbr tsig (a, vs, raw_rhs) = |
677 |
let |
|
678 |
fun err msgs = (seq writeln msgs; |
|
679 |
error ("The error(s) above occurred in type abbreviation " ^ quote a)); |
|
680 |
||
681 |
val rhs = rem_sorts (varifyT (no_tvars raw_rhs)) |
|
682 |
handle TYPE (msg, _, _) => err [msg]; |
|
683 |
val abbr = (a, (vs, rhs)); |
|
684 |
in |
|
582 | 685 |
(case abbr_errors tsig abbr of |
621 | 686 |
[] => abbr |
687 |
| msgs => err msgs) |
|
582 | 688 |
end; |
689 |
||
963 | 690 |
fun add_abbr (tsig as TySg{classes,subclass,default,tycons,arities,abbrs}, |
691 |
abbr) = |
|
621 | 692 |
make_tsig |
963 | 693 |
(classes,subclass,default,tycons, prep_abbr tsig abbr :: abbrs, arities); |
621 | 694 |
|
695 |
fun ext_tsig_abbrs tsig raw_abbrs = foldl add_abbr (tsig, raw_abbrs); |
|
582 | 696 |
|
697 |
||
698 |
||
422 | 699 |
(** add arities **) |
700 |
||
0 | 701 |
(* 'coregular' checks |
963 | 702 |
- the two restrictions 'is_unique_decl' and 'coreg' |
256 | 703 |
- if the classes in the new type declarations are known in the |
0 | 704 |
given type signature |
705 |
- if one type constructor has always the same number of arguments; |
|
256 | 706 |
if one type declaration has passed all checks it is inserted into |
963 | 707 |
the 'arities' association list of the given type signatrure *) |
0 | 708 |
|
963 | 709 |
fun coregular (classes, subclass, tycons) = |
256 | 710 |
let fun ex C = if C mem classes then () else err_undcl_class(C); |
0 | 711 |
|
963 | 712 |
fun addar(arities, (t, (w, C))) = case assoc(tycons, t) of |
0 | 713 |
Some(n) => if n <> length w then varying_decls(t) else |
963 | 714 |
((seq o seq) ex w; ex C; |
715 |
let val ars = the (assoc(arities, t)) |
|
716 |
val ars' = add_arity subclass ars (t,(C,w)) |
|
717 |
in overwrite(arities, (t,ars')) end) |
|
256 | 718 |
| None => err_undcl_type(t); |
0 | 719 |
|
963 | 720 |
in addar end; |
0 | 721 |
|
722 |
||
963 | 723 |
(* 'close' extends the 'arities' association list after all new type |
0 | 724 |
declarations have been inserted successfully: |
725 |
for every declaration t:(Ss)C , for all classses D with C <= D: |
|
726 |
if there is no declaration t:(Ss')C' with C < C' and C' <= D |
|
963 | 727 |
then insert the declaration t:(Ss)D into 'arities' |
0 | 728 |
this means, if there exists a declaration t:(Ss)C and there is |
729 |
no declaration t:(Ss')D with C <=D then the declaration holds |
|
256 | 730 |
for all range classes more general than C *) |
731 |
||
963 | 732 |
fun close subclass arities = |
256 | 733 |
let fun check sl (l, (s, dom)) = case assoc (subclass, s) of |
621 | 734 |
Some sups => |
256 | 735 |
let fun close_sup (l, sup) = |
736 |
if exists (fn s'' => less subclass (s, s'') andalso |
|
737 |
leq subclass (s'', sup)) sl |
|
0 | 738 |
then l |
256 | 739 |
else (sup, dom)::l |
740 |
in foldl close_sup (l, sups) end |
|
0 | 741 |
| None => l; |
256 | 742 |
fun ext (s, l) = (s, foldl (check (map #1 l)) (l, l)); |
963 | 743 |
in map ext arities end; |
0 | 744 |
|
422 | 745 |
|
621 | 746 |
(* ext_tsig_arities *) |
256 | 747 |
|
621 | 748 |
fun ext_tsig_arities tsig sarities = |
416 | 749 |
let |
963 | 750 |
val TySg {classes, subclass, default, tycons, arities, abbrs} = tsig; |
751 |
val arities1 = |
|
752 |
flat (map (fn (t, ss, cs) => map (fn c => (t, (ss, c))) cs) sarities); |
|
753 |
val arities2 = foldl (coregular (classes, subclass, tycons)) |
|
754 |
(arities, min_domain subclass arities1) |
|
621 | 755 |
|> close subclass; |
416 | 756 |
in |
963 | 757 |
make_tsig (classes, subclass, default, tycons, abbrs, arities2) |
416 | 758 |
end; |
0 | 759 |
|
760 |
||
416 | 761 |
|
762 |
(*** type unification and inference ***) |
|
0 | 763 |
|
764 |
(* |
|
621 | 765 |
Input: |
766 |
- a 'raw' term which contains only dummy types and some explicit type |
|
767 |
constraints encoded as terms. |
|
768 |
- the expected type of the term. |
|
0 | 769 |
|
621 | 770 |
Output: |
771 |
- the correctly typed term |
|
772 |
- the substitution needed to unify the actual type of the term with its |
|
773 |
expected type; only the TVars in the expected type are included. |
|
0 | 774 |
|
1435
aefcd255ed4a
Removed bug in type unification. Negative indexes are not used any longer.
nipkow
parents:
1392
diff
changeset
|
775 |
During type inference all TVars in the term have index > maxidx, where |
aefcd255ed4a
Removed bug in type unification. Negative indexes are not used any longer.
nipkow
parents:
1392
diff
changeset
|
776 |
maxidx is the max. index in the expected type of the term (T). This keeps |
aefcd255ed4a
Removed bug in type unification. Negative indexes are not used any longer.
nipkow
parents:
1392
diff
changeset
|
777 |
them apart, because at the end the type of the term is unified with T. |
0 | 778 |
|
621 | 779 |
1. Add initial type information to the term (attach_types). |
780 |
This freezes (freeze_vars) TVars in explicitly provided types (eg |
|
781 |
constraints or defaults) by turning them into TFrees. |
|
1435
aefcd255ed4a
Removed bug in type unification. Negative indexes are not used any longer.
nipkow
parents:
1392
diff
changeset
|
782 |
2. Carry out type inference. |
621 | 783 |
3. Unify actual and expected type. |
1435
aefcd255ed4a
Removed bug in type unification. Negative indexes are not used any longer.
nipkow
parents:
1392
diff
changeset
|
784 |
4. Turn all local (i.e. > maxidx) TVars into unique new TFrees (freeze). |
621 | 785 |
5. Thaw all TVars frozen in step 1 (thaw_vars). |
0 | 786 |
*) |
787 |
||
788 |
(*Raised if types are not unifiable*) |
|
789 |
exception TUNIFY; |
|
790 |
||
1435
aefcd255ed4a
Removed bug in type unification. Negative indexes are not used any longer.
nipkow
parents:
1392
diff
changeset
|
791 |
val tyvar_count = ref 0; |
0 | 792 |
|
1435
aefcd255ed4a
Removed bug in type unification. Negative indexes are not used any longer.
nipkow
parents:
1392
diff
changeset
|
793 |
fun tyinit(i) = (tyvar_count := i); |
0 | 794 |
|
1435
aefcd255ed4a
Removed bug in type unification. Negative indexes are not used any longer.
nipkow
parents:
1392
diff
changeset
|
795 |
fun new_tvar_inx () = (tyvar_count := !tyvar_count + 1; !tyvar_count) |
0 | 796 |
|
797 |
(* |
|
1435
aefcd255ed4a
Removed bug in type unification. Negative indexes are not used any longer.
nipkow
parents:
1392
diff
changeset
|
798 |
Generate new TVar. Index is > maxidx+1 to distinguish it from TVars |
aefcd255ed4a
Removed bug in type unification. Negative indexes are not used any longer.
nipkow
parents:
1392
diff
changeset
|
799 |
generated from variable names (see id_type). |
aefcd255ed4a
Removed bug in type unification. Negative indexes are not used any longer.
nipkow
parents:
1392
diff
changeset
|
800 |
Name is arbitrary because index is new. |
0 | 801 |
*) |
802 |
||
256 | 803 |
fun gen_tyvar(S) = TVar(("'a", new_tvar_inx()), S); |
0 | 804 |
|
805 |
(*Occurs check: type variable occurs in type?*) |
|
806 |
fun occ v tye = |
|
256 | 807 |
let fun occ(Type(_, Ts)) = exists occ Ts |
0 | 808 |
| occ(TFree _) = false |
256 | 809 |
| occ(TVar(w, _)) = v=w orelse |
810 |
(case assoc(tye, w) of |
|
0 | 811 |
None => false |
812 |
| Some U => occ U); |
|
813 |
in occ end; |
|
814 |
||
256 | 815 |
(*Chase variable assignments in tye. |
816 |
If devar (T, tye) returns a type var then it must be unassigned.*) |
|
817 |
fun devar (T as TVar(v, _), tye) = (case assoc(tye, v) of |
|
818 |
Some U => devar (U, tye) |
|
0 | 819 |
| None => T) |
256 | 820 |
| devar (T, tye) = T; |
0 | 821 |
|
1627 | 822 |
(* use add_to_tye(t,tye) instead of t::tye |
823 |
to avoid chains of the form 'a |-> 'b |-> 'c ... *) |
|
824 |
||
825 |
fun add_to_tye(p,[]) = [p] |
|
826 |
| add_to_tye(vT as (v,T),(xU as (x,TVar(w,S)))::ps) = |
|
827 |
(if v=w then (x,T) else xU) :: (add_to_tye(vT,ps)) |
|
828 |
| add_to_tye(v,x::xs) = x::(add_to_tye(v,xs)); |
|
0 | 829 |
|
830 |
(* 'dom' returns for a type constructor t the list of those domains |
|
831 |
which deliver a given range class C *) |
|
832 |
||
963 | 833 |
fun dom arities t C = case assoc2 (arities, (t, C)) of |
0 | 834 |
Some(Ss) => Ss |
835 |
| None => raise TUNIFY; |
|
836 |
||
837 |
||
838 |
(* 'Dom' returns the union of all domain lists of 'dom' for a given sort S |
|
839 |
(i.e. a set of range classes ); the union is carried out elementwise |
|
840 |
for the seperate sorts in the domains *) |
|
841 |
||
963 | 842 |
fun Dom (subclass, arities) (t, S) = |
843 |
let val domlist = map (dom arities t) S; |
|
0 | 844 |
in if null domlist then [] |
256 | 845 |
else foldl (elementwise_union subclass) (hd domlist, tl domlist) |
0 | 846 |
end; |
847 |
||
848 |
||
963 | 849 |
fun W ((T, S), tsig as TySg{subclass, arities, ...}, tye) = |
256 | 850 |
let fun Wd ((T, S), tye) = W ((devar (T, tye), S), tsig, tye) |
851 |
fun Wk(T as TVar(v, S')) = |
|
852 |
if sortorder subclass (S', S) then tye |
|
1627 | 853 |
else add_to_tye((v, gen_tyvar(union_sort subclass (S', S))),tye) |
256 | 854 |
| Wk(T as TFree(v, S')) = if sortorder subclass (S', S) then tye |
855 |
else raise TUNIFY |
|
856 |
| Wk(T as Type(f, Ts)) = |
|
857 |
if null S then tye |
|
963 | 858 |
else foldr Wd (Ts~~(Dom (subclass, arities) (f, S)) , tye) |
0 | 859 |
in Wk(T) end; |
860 |
||
861 |
||
862 |
(* Order-sorted Unification of Types (U) *) |
|
863 |
||
864 |
(* Precondition: both types are well-formed w.r.t. type constructor arities *) |
|
1435
aefcd255ed4a
Removed bug in type unification. Negative indexes are not used any longer.
nipkow
parents:
1392
diff
changeset
|
865 |
fun unify1 (tsig as TySg{subclass, arities, ...}) = |
256 | 866 |
let fun unif ((T, U), tye) = |
867 |
case (devar(T, tye), devar(U, tye)) of |
|
868 |
(T as TVar(v, S1), U as TVar(w, S2)) => |
|
0 | 869 |
if v=w then tye else |
1627 | 870 |
if sortorder subclass (S1, S2) then add_to_tye((w, T),tye) else |
871 |
if sortorder subclass (S2, S1) then add_to_tye((v, U),tye) |
|
256 | 872 |
else let val nu = gen_tyvar (union_sort subclass (S1, S2)) |
1627 | 873 |
in add_to_tye((v, nu),add_to_tye((w, nu),tye)) end |
256 | 874 |
| (T as TVar(v, S), U) => |
1627 | 875 |
if occ v tye U then raise TUNIFY else W ((U,S), tsig, add_to_tye((v, U),tye)) |
256 | 876 |
| (U, T as TVar (v, S)) => |
1627 | 877 |
if occ v tye U then raise TUNIFY else W ((U,S), tsig, add_to_tye((v, U),tye)) |
256 | 878 |
| (Type(a, Ts), Type(b, Us)) => |
879 |
if a<>b then raise TUNIFY else foldr unif (Ts~~Us, tye) |
|
880 |
| (T, U) => if T=U then tye else raise TUNIFY |
|
0 | 881 |
in unif end; |
882 |
||
1435
aefcd255ed4a
Removed bug in type unification. Negative indexes are not used any longer.
nipkow
parents:
1392
diff
changeset
|
883 |
fun unify tsig maxidx tye TU = |
aefcd255ed4a
Removed bug in type unification. Negative indexes are not used any longer.
nipkow
parents:
1392
diff
changeset
|
884 |
(tyinit maxidx; (unify1 tsig (TU,tye), !tyvar_count) ); |
0 | 885 |
|
450 | 886 |
(* raw_unify (ignores sorts) *) |
887 |
||
888 |
fun raw_unify (ty1, ty2) = |
|
1435
aefcd255ed4a
Removed bug in type unification. Negative indexes are not used any longer.
nipkow
parents:
1392
diff
changeset
|
889 |
(unify tsig0 0 [] (rem_sorts ty1, rem_sorts ty2); true) |
450 | 890 |
handle TUNIFY => false; |
891 |
||
892 |
||
0 | 893 |
(*Type inference for polymorphic term*) |
894 |
fun infer tsig = |
|
256 | 895 |
let fun inf(Ts, Const (_, T), tye) = (T, tye) |
896 |
| inf(Ts, Free (_, T), tye) = (T, tye) |
|
897 |
| inf(Ts, Bound i, tye) = ((nth_elem(i, Ts) , tye) |
|
0 | 898 |
handle LIST _=> raise TYPE ("loose bound variable", [], [Bound i])) |
256 | 899 |
| inf(Ts, Var (_, T), tye) = (T, tye) |
900 |
| inf(Ts, Abs (_, T, body), tye) = |
|
901 |
let val (U, tye') = inf(T::Ts, body, tye) in (T-->U, tye') end |
|
0 | 902 |
| inf(Ts, f$u, tye) = |
256 | 903 |
let val (U, tyeU) = inf(Ts, u, tye); |
904 |
val (T, tyeT) = inf(Ts, f, tyeU); |
|
0 | 905 |
fun err s = |
906 |
raise TYPE(s, [inst_typ tyeT T, inst_typ tyeT U], [f$u]) |
|
1460 | 907 |
val msg = "function type is incompatible with argument type" |
256 | 908 |
in case T of |
909 |
Type("fun", [T1, T2]) => |
|
1435
aefcd255ed4a
Removed bug in type unification. Negative indexes are not used any longer.
nipkow
parents:
1392
diff
changeset
|
910 |
( (T2, unify1 tsig ((T1, U), tyeT)) |
1392
1b4ae50e0e0a
infer_types now takes a term list and a type list as argument. It
paulson
parents:
1257
diff
changeset
|
911 |
handle TUNIFY => err msg) |
256 | 912 |
| TVar _ => |
0 | 913 |
let val T2 = gen_tyvar([]) |
1435
aefcd255ed4a
Removed bug in type unification. Negative indexes are not used any longer.
nipkow
parents:
1392
diff
changeset
|
914 |
in (T2, unify1 tsig ((T, U-->T2), tyeT)) |
1392
1b4ae50e0e0a
infer_types now takes a term list and a type list as argument. It
paulson
parents:
1257
diff
changeset
|
915 |
handle TUNIFY => err msg |
0 | 916 |
end |
1392
1b4ae50e0e0a
infer_types now takes a term list and a type list as argument. It
paulson
parents:
1257
diff
changeset
|
917 |
| _ => err"function type is expected in application" |
0 | 918 |
end |
919 |
in inf end; |
|
920 |
||
949
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
921 |
val freeze_vars = |
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
922 |
map_type_tvar (fn (v, S) => TFree(Syntax.string_of_vname v, S)); |
0 | 923 |
|
924 |
(* Attach a type to a constant *) |
|
256 | 925 |
fun type_const (a, T) = Const(a, incr_tvar (new_tvar_inx()) T); |
0 | 926 |
|
927 |
(*Find type of ident. If not in table then use ident's name for tyvar |
|
928 |
to get consistent typing.*) |
|
256 | 929 |
fun new_id_type a = TVar(("'"^a, new_tvar_inx()), []); |
1435
aefcd255ed4a
Removed bug in type unification. Negative indexes are not used any longer.
nipkow
parents:
1392
diff
changeset
|
930 |
|
aefcd255ed4a
Removed bug in type unification. Negative indexes are not used any longer.
nipkow
parents:
1392
diff
changeset
|
931 |
fun type_of_ixn(types, ixn as (a, _),maxidx1) = |
aefcd255ed4a
Removed bug in type unification. Negative indexes are not used any longer.
nipkow
parents:
1392
diff
changeset
|
932 |
case types ixn of Some T => freeze_vars T |
aefcd255ed4a
Removed bug in type unification. Negative indexes are not used any longer.
nipkow
parents:
1392
diff
changeset
|
933 |
| None => TVar(("'"^a, maxidx1), []); |
565 | 934 |
|
935 |
fun constrain (term, T) = Const (Syntax.constrainC, T --> T) $ term; |
|
0 | 936 |
|
565 | 937 |
fun constrainAbs (Abs (a, _, body), T) = Abs (a, T, body) |
938 |
| constrainAbs _ = sys_error "constrainAbs"; |
|
256 | 939 |
|
0 | 940 |
|
565 | 941 |
(* attach_types *) |
942 |
||
0 | 943 |
(* |
256 | 944 |
Attach types to a term. Input is a "parse tree" containing dummy types. |
945 |
Type constraints are translated and checked for validity wrt tsig. TVars in |
|
946 |
constraints are frozen. |
|
0 | 947 |
|
256 | 948 |
The atoms in the resulting term satisfy the following spec: |
0 | 949 |
|
256 | 950 |
Const (a, T): |
1435
aefcd255ed4a
Removed bug in type unification. Negative indexes are not used any longer.
nipkow
parents:
1392
diff
changeset
|
951 |
T is a renamed copy of the generic type of a; renaming increases index of |
aefcd255ed4a
Removed bug in type unification. Negative indexes are not used any longer.
nipkow
parents:
1392
diff
changeset
|
952 |
all TVars by new_tvar_inx(), which is > maxidx+1. |
0 | 953 |
|
256 | 954 |
Free (a, T), Var (ixn, T): |
1435
aefcd255ed4a
Removed bug in type unification. Negative indexes are not used any longer.
nipkow
parents:
1392
diff
changeset
|
955 |
T is either the frozen default type of a or TVar (("'"^a, maxidx+1), []) |
0 | 956 |
|
256 | 957 |
Abs (a, T, _): |
958 |
T is either a type constraint or TVar (("'" ^ a, i), []), where i is |
|
959 |
generated by new_tvar_inx(). Thus different abstractions can have the |
|
960 |
bound variables of the same name but different types. |
|
0 | 961 |
*) |
962 |
||
1257 | 963 |
(* FIXME consistency of sort_env / sorts (!?) *) |
256 | 964 |
|
1435
aefcd255ed4a
Removed bug in type unification. Negative indexes are not used any longer.
nipkow
parents:
1392
diff
changeset
|
965 |
fun attach_types (tsig, const_type, types, sorts, maxidx1) tm = |
256 | 966 |
let |
565 | 967 |
val sort_env = Syntax.raw_term_sorts tm; |
968 |
fun def_sort xi = if_none (sorts xi) (defaultS tsig); |
|
256 | 969 |
|
565 | 970 |
fun prepareT t = |
971 |
freeze_vars (cert_typ tsig (Syntax.typ_of_term sort_env def_sort t)); |
|
256 | 972 |
|
973 |
fun add (Const (a, _)) = |
|
565 | 974 |
(case const_type a of |
256 | 975 |
Some T => type_const (a, T) |
976 |
| None => raise_type ("No such constant: " ^ quote a) [] []) |
|
977 |
| add (Free (a, _)) = |
|
565 | 978 |
(case const_type a of |
256 | 979 |
Some T => type_const (a, T) |
1435
aefcd255ed4a
Removed bug in type unification. Negative indexes are not used any longer.
nipkow
parents:
1392
diff
changeset
|
980 |
| None => Free (a, type_of_ixn (types,(a,~1),maxidx1))) |
aefcd255ed4a
Removed bug in type unification. Negative indexes are not used any longer.
nipkow
parents:
1392
diff
changeset
|
981 |
| add (Var (ixn, _)) = Var (ixn, type_of_ixn (types, ixn, maxidx1)) |
565 | 982 |
| add (Bound i) = Bound i |
256 | 983 |
| add (Abs (a, _, body)) = Abs (a, new_id_type a, add body) |
984 |
| add ((f as Const (a, _) $ t1) $ t2) = |
|
985 |
if a = Syntax.constrainC then |
|
986 |
constrain (add t1, prepareT t2) |
|
987 |
else if a = Syntax.constrainAbsC then |
|
988 |
constrainAbs (add t1, prepareT t2) |
|
989 |
else add f $ add t2 |
|
990 |
| add (f $ t) = add f $ add t; |
|
565 | 991 |
in add tm end; |
0 | 992 |
|
993 |
||
994 |
(* Post-Processing *) |
|
995 |
||
996 |
(*Instantiation of type variables in terms*) |
|
997 |
fun inst_types tye = map_term_types (inst_typ tye); |
|
998 |
||
999 |
(*Delete explicit constraints -- occurrences of "_constrain" *) |
|
256 | 1000 |
fun unconstrain (Abs(a, T, t)) = Abs(a, T, unconstrain t) |
1001 |
| unconstrain ((f as Const(a, _)) $ t) = |
|
0 | 1002 |
if a=Syntax.constrainC then unconstrain t |
1003 |
else unconstrain f $ unconstrain t |
|
1004 |
| unconstrain (f$t) = unconstrain f $ unconstrain t |
|
1005 |
| unconstrain (t) = t; |
|
1006 |
||
949
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
1007 |
fun nextname(pref,c) = if c="z" then (pref^"a", "a") else (pref,chr(ord(c)+1)); |
0 | 1008 |
|
949
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
1009 |
fun newtvars used = |
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
1010 |
let fun new([],_,vmap) = vmap |
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
1011 |
| new(ixn::ixns,p as (pref,c),vmap) = |
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
1012 |
let val nm = pref ^ c |
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
1013 |
in if nm mem used then new(ixn::ixns,nextname p, vmap) |
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
1014 |
else new(ixns, nextname p, (ixn,nm)::vmap) |
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
1015 |
end |
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
1016 |
in new end; |
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
1017 |
|
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
1018 |
(* |
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
1019 |
Turn all TVars which satisfy p into new (if freeze then TFrees else TVars). |
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
1020 |
Note that if t contains frozen TVars there is the possibility that a TVar is |
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
1021 |
turned into one of those. This is sound but not complete. |
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
1022 |
*) |
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
1023 |
fun convert used freeze p t = |
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
1024 |
let val used = if freeze then add_term_tfree_names(t, used) |
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
1025 |
else used union |
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
1026 |
(map #1 (filter_out p (add_term_tvar_ixns(t, [])))) |
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
1027 |
val ixns = filter p (add_term_tvar_ixns(t, [])); |
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
1028 |
val vmap = newtvars used (ixns,("'","a"),[]); |
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
1029 |
fun conv(var as (ixn,S)) = case assoc(vmap,ixn) of |
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
1030 |
None => TVar(var) | |
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
1031 |
Some(a) => if freeze then TFree(a,S) else TVar((a,0),S); |
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
1032 |
in map_term_types (map_type_tvar conv) t end; |
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
1033 |
|
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
1034 |
fun freeze t = convert (add_term_tfree_names(t,[])) true (K true) t; |
0 | 1035 |
|
1036 |
(* Thaw all TVars that were frozen in freeze_vars *) |
|
949
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
1037 |
val thaw_vars = |
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
1038 |
let fun thaw(f as (a, S)) = (case explode a of |
256 | 1039 |
"?"::"'"::vn => let val ((b, i), _) = Syntax.scan_varname vn |
1040 |
in TVar(("'"^b, i), S) end |
|
949
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
1041 |
| _ => TFree f) |
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
1042 |
in map_type_tfree thaw end; |
0 | 1043 |
|
1044 |
||
1435
aefcd255ed4a
Removed bug in type unification. Negative indexes are not used any longer.
nipkow
parents:
1392
diff
changeset
|
1045 |
fun restrict maxidx1 tye = |
256 | 1046 |
let fun clean(tye1, ((a, i), T)) = |
1435
aefcd255ed4a
Removed bug in type unification. Negative indexes are not used any longer.
nipkow
parents:
1392
diff
changeset
|
1047 |
if i >= maxidx1 then tye1 else ((a, i), inst_typ tye T) :: tye1 |
256 | 1048 |
in foldl clean ([], tye) end |
0 | 1049 |
|
1050 |
||
1392
1b4ae50e0e0a
infer_types now takes a term list and a type list as argument. It
paulson
parents:
1257
diff
changeset
|
1051 |
(*Infer types for terms. Given Ts=[T1,...,Tn] and ts=[t1,...,tn], ensure that |
1460 | 1052 |
the type of ti unifies with Ti (i=1,...,n). |
1392
1b4ae50e0e0a
infer_types now takes a term list and a type list as argument. It
paulson
parents:
1257
diff
changeset
|
1053 |
types is a partial map from indexnames to types (constrains Free, Var). |
1b4ae50e0e0a
infer_types now takes a term list and a type list as argument. It
paulson
parents:
1257
diff
changeset
|
1054 |
sorts is a partial map from indexnames to sorts (constrains TFree, TVar). |
1b4ae50e0e0a
infer_types now takes a term list and a type list as argument. It
paulson
parents:
1257
diff
changeset
|
1055 |
used is the list of already used type variables. |
1b4ae50e0e0a
infer_types now takes a term list and a type list as argument. It
paulson
parents:
1257
diff
changeset
|
1056 |
If freeze then internal TVars are turned into TFrees, else TVars.*) |
1435
aefcd255ed4a
Removed bug in type unification. Negative indexes are not used any longer.
nipkow
parents:
1392
diff
changeset
|
1057 |
fun infer_types (tsig, const_type, types, sorts, used, freeze, Ts, ts) = |
565 | 1058 |
let |
1435
aefcd255ed4a
Removed bug in type unification. Negative indexes are not used any longer.
nipkow
parents:
1392
diff
changeset
|
1059 |
val maxidx1 = max(map maxidx_of_typ Ts)+1; |
aefcd255ed4a
Removed bug in type unification. Negative indexes are not used any longer.
nipkow
parents:
1392
diff
changeset
|
1060 |
val () = tyinit(maxidx1+1); |
aefcd255ed4a
Removed bug in type unification. Negative indexes are not used any longer.
nipkow
parents:
1392
diff
changeset
|
1061 |
val us = map (attach_types (tsig, const_type, types, sorts, maxidx1)) ts; |
1392
1b4ae50e0e0a
infer_types now takes a term list and a type list as argument. It
paulson
parents:
1257
diff
changeset
|
1062 |
val u = list_comb(Const("",Ts ---> propT),us) |
1b4ae50e0e0a
infer_types now takes a term list and a type list as argument. It
paulson
parents:
1257
diff
changeset
|
1063 |
val (_, tye) = infer tsig ([], u, []); |
565 | 1064 |
val uu = unconstrain u; |
1435
aefcd255ed4a
Removed bug in type unification. Negative indexes are not used any longer.
nipkow
parents:
1392
diff
changeset
|
1065 |
val Ttye = restrict maxidx1 tye (*restriction to TVars in Ts*) |
1392
1b4ae50e0e0a
infer_types now takes a term list and a type list as argument. It
paulson
parents:
1257
diff
changeset
|
1066 |
val all = Const("", Type("", map snd Ttye)) $ (inst_types tye uu) |
565 | 1067 |
(*all is a dummy term which contains all exported TVars*) |
1392
1b4ae50e0e0a
infer_types now takes a term list and a type list as argument. It
paulson
parents:
1257
diff
changeset
|
1068 |
val Const(_, Type(_, Us)) $ u'' = |
1435
aefcd255ed4a
Removed bug in type unification. Negative indexes are not used any longer.
nipkow
parents:
1392
diff
changeset
|
1069 |
map_term_types thaw_vars (convert used freeze (fn (_,i) => i >= maxidx1) all) |
949
83c588d6fee9
Changed treatment of during type inference internally generated type
nipkow
parents:
621
diff
changeset
|
1070 |
(*convert all internally generated TVars into TFrees or TVars |
565 | 1071 |
and thaw all initially frozen TVars*) |
1072 |
in |
|
1392
1b4ae50e0e0a
infer_types now takes a term list and a type list as argument. It
paulson
parents:
1257
diff
changeset
|
1073 |
(snd(strip_comb u''), (map fst Ttye) ~~ Us) |
565 | 1074 |
end; |
0 | 1075 |
|
1076 |
end; |