author | wenzelm |
Mon, 27 May 2013 16:52:39 +0200 | |
changeset 52179 | 3b9c31867707 |
parent 52128 | 7f3549a316f4 |
child 52220 | c4264f71dc3b |
permissions | -rw-r--r-- |
15797 | 1 |
(* Title: Pure/unify.ML |
16425
2427be27cc60
accomodate identification of type Sign.sg and theory;
wenzelm
parents:
15797
diff
changeset
|
2 |
Author: Lawrence C Paulson, Cambridge University Computer Laboratory |
0 | 3 |
Copyright Cambridge University 1992 |
4 |
||
16425
2427be27cc60
accomodate identification of type Sign.sg and theory;
wenzelm
parents:
15797
diff
changeset
|
5 |
Higher-Order Unification. |
0 | 6 |
|
16425
2427be27cc60
accomodate identification of type Sign.sg and theory;
wenzelm
parents:
15797
diff
changeset
|
7 |
Types as well as terms are unified. The outermost functions assume |
2427be27cc60
accomodate identification of type Sign.sg and theory;
wenzelm
parents:
15797
diff
changeset
|
8 |
the terms to be unified already have the same type. In resolution, |
2427be27cc60
accomodate identification of type Sign.sg and theory;
wenzelm
parents:
15797
diff
changeset
|
9 |
this is assured because both have type "prop". |
0 | 10 |
*) |
11 |
||
16425
2427be27cc60
accomodate identification of type Sign.sg and theory;
wenzelm
parents:
15797
diff
changeset
|
12 |
signature UNIFY = |
2427be27cc60
accomodate identification of type Sign.sg and theory;
wenzelm
parents:
15797
diff
changeset
|
13 |
sig |
39163
4d701c0388c3
more explicit indication of Config.raw options, which are only needed for bootstrapping Pure;
wenzelm
parents:
39116
diff
changeset
|
14 |
val trace_bound_raw: Config.raw |
24178
4ff1dc2aa18d
turned Unify flags into configuration options (global only);
wenzelm
parents:
23178
diff
changeset
|
15 |
val trace_bound: int Config.T |
39163
4d701c0388c3
more explicit indication of Config.raw options, which are only needed for bootstrapping Pure;
wenzelm
parents:
39116
diff
changeset
|
16 |
val search_bound_raw: Config.raw |
24178
4ff1dc2aa18d
turned Unify flags into configuration options (global only);
wenzelm
parents:
23178
diff
changeset
|
17 |
val search_bound: int Config.T |
39163
4d701c0388c3
more explicit indication of Config.raw options, which are only needed for bootstrapping Pure;
wenzelm
parents:
39116
diff
changeset
|
18 |
val trace_simp_raw: Config.raw |
24178
4ff1dc2aa18d
turned Unify flags into configuration options (global only);
wenzelm
parents:
23178
diff
changeset
|
19 |
val trace_simp: bool Config.T |
39163
4d701c0388c3
more explicit indication of Config.raw options, which are only needed for bootstrapping Pure;
wenzelm
parents:
39116
diff
changeset
|
20 |
val trace_types_raw: Config.raw |
24178
4ff1dc2aa18d
turned Unify flags into configuration options (global only);
wenzelm
parents:
23178
diff
changeset
|
21 |
val trace_types: bool Config.T |
52126 | 22 |
val hounifiers: theory * Envir.env * ((term * term) list) -> |
23 |
(Envir.env * (term * term) list) Seq.seq |
|
16425
2427be27cc60
accomodate identification of type Sign.sg and theory;
wenzelm
parents:
15797
diff
changeset
|
24 |
val unifiers: theory * Envir.env * ((term * term) list) -> |
2427be27cc60
accomodate identification of type Sign.sg and theory;
wenzelm
parents:
15797
diff
changeset
|
25 |
(Envir.env * (term * term) list) Seq.seq |
19864 | 26 |
val smash_unifiers: theory -> (term * term) list -> Envir.env -> Envir.env Seq.seq |
27 |
val matchers: theory -> (term * term) list -> Envir.env Seq.seq |
|
28 |
val matches_list: theory -> term list -> term list -> bool |
|
16425
2427be27cc60
accomodate identification of type Sign.sg and theory;
wenzelm
parents:
15797
diff
changeset
|
29 |
end |
0 | 30 |
|
19864 | 31 |
structure Unify : UNIFY = |
0 | 32 |
struct |
33 |
||
34 |
(*Unification options*) |
|
35 |
||
24178
4ff1dc2aa18d
turned Unify flags into configuration options (global only);
wenzelm
parents:
23178
diff
changeset
|
36 |
(*tracing starts above this depth, 0 for full*) |
39163
4d701c0388c3
more explicit indication of Config.raw options, which are only needed for bootstrapping Pure;
wenzelm
parents:
39116
diff
changeset
|
37 |
val trace_bound_raw = Config.declare_global "unify_trace_bound" (K (Config.Int 50)); |
4d701c0388c3
more explicit indication of Config.raw options, which are only needed for bootstrapping Pure;
wenzelm
parents:
39116
diff
changeset
|
38 |
val trace_bound = Config.int trace_bound_raw; |
24178
4ff1dc2aa18d
turned Unify flags into configuration options (global only);
wenzelm
parents:
23178
diff
changeset
|
39 |
|
4ff1dc2aa18d
turned Unify flags into configuration options (global only);
wenzelm
parents:
23178
diff
changeset
|
40 |
(*unification quits above this depth*) |
39163
4d701c0388c3
more explicit indication of Config.raw options, which are only needed for bootstrapping Pure;
wenzelm
parents:
39116
diff
changeset
|
41 |
val search_bound_raw = Config.declare_global "unify_search_bound" (K (Config.Int 60)); |
4d701c0388c3
more explicit indication of Config.raw options, which are only needed for bootstrapping Pure;
wenzelm
parents:
39116
diff
changeset
|
42 |
val search_bound = Config.int search_bound_raw; |
24178
4ff1dc2aa18d
turned Unify flags into configuration options (global only);
wenzelm
parents:
23178
diff
changeset
|
43 |
|
4ff1dc2aa18d
turned Unify flags into configuration options (global only);
wenzelm
parents:
23178
diff
changeset
|
44 |
(*print dpairs before calling SIMPL*) |
39163
4d701c0388c3
more explicit indication of Config.raw options, which are only needed for bootstrapping Pure;
wenzelm
parents:
39116
diff
changeset
|
45 |
val trace_simp_raw = Config.declare_global "unify_trace_simp" (K (Config.Bool false)); |
4d701c0388c3
more explicit indication of Config.raw options, which are only needed for bootstrapping Pure;
wenzelm
parents:
39116
diff
changeset
|
46 |
val trace_simp = Config.bool trace_simp_raw; |
24178
4ff1dc2aa18d
turned Unify flags into configuration options (global only);
wenzelm
parents:
23178
diff
changeset
|
47 |
|
4ff1dc2aa18d
turned Unify flags into configuration options (global only);
wenzelm
parents:
23178
diff
changeset
|
48 |
(*announce potential incompleteness of type unification*) |
39163
4d701c0388c3
more explicit indication of Config.raw options, which are only needed for bootstrapping Pure;
wenzelm
parents:
39116
diff
changeset
|
49 |
val trace_types_raw = Config.declare_global "unify_trace_types" (K (Config.Bool false)); |
4d701c0388c3
more explicit indication of Config.raw options, which are only needed for bootstrapping Pure;
wenzelm
parents:
39116
diff
changeset
|
50 |
val trace_types = Config.bool trace_types_raw; |
24178
4ff1dc2aa18d
turned Unify flags into configuration options (global only);
wenzelm
parents:
23178
diff
changeset
|
51 |
|
0 | 52 |
|
52126 | 53 |
type binderlist = (string * typ) list; |
0 | 54 |
|
55 |
type dpair = binderlist * term * term; |
|
56 |
||
12231
4a25f04bea61
Moved head_norm and fastype from unify.ML to envir.ML
berghofe
parents:
8406
diff
changeset
|
57 |
fun fastype env (Ts, t) = Envir.fastype env (map snd Ts) t; |
0 | 58 |
|
59 |
||
32032 | 60 |
(* eta normal form *) |
61 |
||
62 |
fun eta_norm env = |
|
63 |
let |
|
64 |
val tyenv = Envir.type_env env; |
|
65 |
fun etif (Type ("fun", [T, U]), t) = |
|
66 |
Abs ("", T, etif (U, incr_boundvars 1 t $ Bound 0)) |
|
67 |
| etif (TVar v, t) = |
|
68 |
(case Type.lookup tyenv v of |
|
69 |
NONE => t |
|
70 |
| SOME T => etif (T, t)) |
|
71 |
| etif (_, t) = t; |
|
72 |
fun eta_nm (rbinder, Abs (a, T, body)) = |
|
73 |
Abs (a, T, eta_nm ((a, T) :: rbinder, body)) |
|
74 |
| eta_nm (rbinder, t) = etif (fastype env (rbinder, t), t); |
|
0 | 75 |
in eta_nm end; |
76 |
||
77 |
||
78 |
(*OCCURS CHECK |
|
19864 | 79 |
Does the uvar occur in the term t? |
0 | 80 |
two forms of search, for whether there is a rigid path to the current term. |
81 |
"seen" is list of variables passed thru, is a memo variable for sharing. |
|
15797 | 82 |
This version searches for nonrigid occurrence, returns true if found. |
83 |
Since terms may contain variables with same name and different types, |
|
84 |
the occurs check must ignore the types of variables. This avoids |
|
85 |
that ?x::?'a is unified with f(?x::T), which may lead to a cyclic |
|
86 |
substitution when ?'a is instantiated with T later. *) |
|
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
87 |
fun occurs_terms (seen: indexname list Unsynchronized.ref, |
19864 | 88 |
env: Envir.env, v: indexname, ts: term list): bool = |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
89 |
let |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
90 |
fun occurs [] = false |
37636 | 91 |
| occurs (t :: ts) = occur t orelse occurs ts |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
92 |
and occur (Const _) = false |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
93 |
| occur (Bound _) = false |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
94 |
| occur (Free _) = false |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
95 |
| occur (Var (w, T)) = |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
96 |
if member (op =) (!seen) w then false |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
97 |
else if Term.eq_ix (v, w) then true |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
98 |
(*no need to lookup: v has no assignment*) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
99 |
else |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
100 |
(seen := w :: !seen; |
51700 | 101 |
case Envir.lookup env (w, T) of |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
102 |
NONE => false |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
103 |
| SOME t => occur t) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
104 |
| occur (Abs (_, _, body)) = occur body |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
105 |
| occur (f $ t) = occur t orelse occur f; |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
106 |
in occurs ts end; |
0 | 107 |
|
108 |
||
52126 | 109 |
(* f a1 ... an ----> f using the assignments*) |
110 |
fun head_of_in env t = |
|
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
111 |
(case t of |
52126 | 112 |
f $ _ => head_of_in env f |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
113 |
| Var vT => |
51700 | 114 |
(case Envir.lookup env vT of |
52126 | 115 |
SOME u => head_of_in env u |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
116 |
| NONE => t) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
117 |
| _ => t); |
0 | 118 |
|
119 |
||
120 |
datatype occ = NoOcc | Nonrigid | Rigid; |
|
121 |
||
122 |
(* Rigid occur check |
|
123 |
Returns Rigid if it finds a rigid occurrence of the variable, |
|
124 |
Nonrigid if it finds a nonrigid path to the variable. |
|
125 |
NoOcc otherwise. |
|
126 |
Continues searching for a rigid occurrence even if it finds a nonrigid one. |
|
127 |
||
128 |
Condition for detecting non-unifable terms: [ section 5.3 of Huet (1975) ] |
|
129 |
a rigid path to the variable, appearing with no arguments. |
|
130 |
Here completeness is sacrificed in order to reduce danger of divergence: |
|
131 |
reject ALL rigid paths to the variable. |
|
19864 | 132 |
Could check for rigid paths to bound variables that are out of scope. |
0 | 133 |
Not necessary because the assignment test looks at variable's ENTIRE rbinder. |
134 |
||
135 |
Treatment of head(arg1,...,argn): |
|
136 |
If head is a variable then no rigid path, switch to nonrigid search |
|
19864 | 137 |
for arg1,...,argn. |
138 |
If head is an abstraction then possibly no rigid path (head could be a |
|
0 | 139 |
constant function) so again use nonrigid search. Happens only if |
19864 | 140 |
term is not in normal form. |
0 | 141 |
|
142 |
Warning: finds a rigid occurrence of ?f in ?f(t). |
|
143 |
Should NOT be called in this case: there is a flex-flex unifier |
|
144 |
*) |
|
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
145 |
fun rigid_occurs_term (seen: indexname list Unsynchronized.ref, env, v: indexname, t) = |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
146 |
let |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
147 |
fun nonrigid t = |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
148 |
if occurs_terms (seen, env, v, [t]) then Nonrigid |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
149 |
else NoOcc |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
150 |
fun occurs [] = NoOcc |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
151 |
| occurs (t :: ts) = |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
152 |
(case occur t of |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
153 |
Rigid => Rigid |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
154 |
| oc => (case occurs ts of NoOcc => oc | oc2 => oc2)) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
155 |
and occomb (f $ t) = |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
156 |
(case occur t of |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
157 |
Rigid => Rigid |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
158 |
| oc => (case occomb f of NoOcc => oc | oc2 => oc2)) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
159 |
| occomb t = occur t |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
160 |
and occur (Const _) = NoOcc |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
161 |
| occur (Bound _) = NoOcc |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
162 |
| occur (Free _) = NoOcc |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
163 |
| occur (Var (w, T)) = |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
164 |
if member (op =) (!seen) w then NoOcc |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
165 |
else if Term.eq_ix (v, w) then Rigid |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
166 |
else |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
167 |
(seen := w :: !seen; |
51700 | 168 |
case Envir.lookup env (w, T) of |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
169 |
NONE => NoOcc |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
170 |
| SOME t => occur t) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
171 |
| occur (Abs (_, _, body)) = occur body |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
172 |
| occur (t as f $ _) = (*switch to nonrigid search?*) |
52126 | 173 |
(case head_of_in env f of |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
174 |
Var (w,_) => (*w is not assigned*) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
175 |
if Term.eq_ix (v, w) then Rigid |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
176 |
else nonrigid t |
37636 | 177 |
| Abs _ => nonrigid t (*not in normal form*) |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
178 |
| _ => occomb t) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
179 |
in occur t end; |
0 | 180 |
|
181 |
||
19864 | 182 |
exception CANTUNIFY; (*Signals non-unifiability. Does not signal errors!*) |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
183 |
exception ASSIGN; (*Raised if not an assignment*) |
0 | 184 |
|
185 |
||
52127
a40dfe02dd83
re-use Pattern.unify_types, including its trace_unify_fail option;
wenzelm
parents:
52126
diff
changeset
|
186 |
fun unify_types thy TU env = |
a40dfe02dd83
re-use Pattern.unify_types, including its trace_unify_fail option;
wenzelm
parents:
52126
diff
changeset
|
187 |
Pattern.unify_types thy TU env handle Pattern.Unif => raise CANTUNIFY; |
0 | 188 |
|
52179
3b9c31867707
more thorough type unification: treat equal Vars like other atoms, otherwise unify type of term pair (not just accidental body_type of its head Vars);
wenzelm
parents:
52128
diff
changeset
|
189 |
fun unify_types_of thy (rbinder, t, u) env = |
3b9c31867707
more thorough type unification: treat equal Vars like other atoms, otherwise unify type of term pair (not just accidental body_type of its head Vars);
wenzelm
parents:
52128
diff
changeset
|
190 |
unify_types thy (fastype env (rbinder, t), fastype env (rbinder, u)) env; |
3b9c31867707
more thorough type unification: treat equal Vars like other atoms, otherwise unify type of term pair (not just accidental body_type of its head Vars);
wenzelm
parents:
52128
diff
changeset
|
191 |
|
52126 | 192 |
fun test_unify_types thy (T, U) env = |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
193 |
let |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
194 |
val str_of = Syntax.string_of_typ_global thy; |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
195 |
fun warn () = tracing ("Potential loss of completeness: " ^ str_of U ^ " = " ^ str_of T); |
52126 | 196 |
val env' = unify_types thy (T, U) env; |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
197 |
in if is_TVar T orelse is_TVar U then warn () else (); env' end; |
0 | 198 |
|
199 |
(*Is the term eta-convertible to a single variable with the given rbinder? |
|
200 |
Examples: ?a ?f(B.0) ?g(B.1,B.0) |
|
201 |
Result is var a for use in SIMPL. *) |
|
52179
3b9c31867707
more thorough type unification: treat equal Vars like other atoms, otherwise unify type of term pair (not just accidental body_type of its head Vars);
wenzelm
parents:
52128
diff
changeset
|
202 |
fun get_eta_var [] n (Var vT) = (n, vT) |
3b9c31867707
more thorough type unification: treat equal Vars like other atoms, otherwise unify type of term pair (not just accidental body_type of its head Vars);
wenzelm
parents:
52128
diff
changeset
|
203 |
| get_eta_var (_ :: rbinder) n (f $ Bound i) = |
3b9c31867707
more thorough type unification: treat equal Vars like other atoms, otherwise unify type of term pair (not just accidental body_type of its head Vars);
wenzelm
parents:
52128
diff
changeset
|
204 |
if n = i then get_eta_var rbinder (n + 1) f |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
205 |
else raise ASSIGN |
52179
3b9c31867707
more thorough type unification: treat equal Vars like other atoms, otherwise unify type of term pair (not just accidental body_type of its head Vars);
wenzelm
parents:
52128
diff
changeset
|
206 |
| get_eta_var _ _ _ = raise ASSIGN; |
0 | 207 |
|
208 |
||
209 |
(*Solve v=u by assignment -- "fixedpoint" to Huet -- if v not in u. |
|
210 |
If v occurs rigidly then nonunifiable. |
|
211 |
If v occurs nonrigidly then must use full algorithm. *) |
|
52126 | 212 |
fun assignment thy (rbinder, t, u) env = |
52179
3b9c31867707
more thorough type unification: treat equal Vars like other atoms, otherwise unify type of term pair (not just accidental body_type of its head Vars);
wenzelm
parents:
52128
diff
changeset
|
213 |
let val (n, (v, T)) = get_eta_var rbinder 0 t in |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
214 |
(case rigid_occurs_term (Unsynchronized.ref [], env, v, u) of |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
215 |
NoOcc => |
52179
3b9c31867707
more thorough type unification: treat equal Vars like other atoms, otherwise unify type of term pair (not just accidental body_type of its head Vars);
wenzelm
parents:
52128
diff
changeset
|
216 |
let val env = unify_types thy (Envir.body_type env n T, fastype env (rbinder, u)) env |
3b9c31867707
more thorough type unification: treat equal Vars like other atoms, otherwise unify type of term pair (not just accidental body_type of its head Vars);
wenzelm
parents:
52128
diff
changeset
|
217 |
in Envir.update ((v, T), Logic.rlist_abs (rbinder, u)) env end |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
218 |
| Nonrigid => raise ASSIGN |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
219 |
| Rigid => raise CANTUNIFY) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
220 |
end; |
0 | 221 |
|
222 |
||
223 |
(*Extends an rbinder with a new disagreement pair, if both are abstractions. |
|
224 |
Checks that binders have same length, since terms should be eta-normal; |
|
225 |
if not, raises TERM, probably indicating type mismatch. |
|
19864 | 226 |
Uses variable a (unless the null string) to preserve user's naming.*) |
52126 | 227 |
fun new_dpair thy (rbinder, Abs (a, T, body1), Abs (b, U, body2)) env = |
52179
3b9c31867707
more thorough type unification: treat equal Vars like other atoms, otherwise unify type of term pair (not just accidental body_type of its head Vars);
wenzelm
parents:
52128
diff
changeset
|
228 |
let val c = if a = "" then b else a |
3b9c31867707
more thorough type unification: treat equal Vars like other atoms, otherwise unify type of term pair (not just accidental body_type of its head Vars);
wenzelm
parents:
52128
diff
changeset
|
229 |
in new_dpair thy ((c, T) :: rbinder, body1, body2) env end |
52126 | 230 |
| new_dpair _ (_, Abs _, _) _ = raise TERM ("new_dpair", []) |
231 |
| new_dpair _ (_, _, Abs _) _ = raise TERM ("new_dpair", []) |
|
232 |
| new_dpair _ (rbinder, t1, t2) env = ((rbinder, t1, t2), env); |
|
0 | 233 |
|
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
234 |
fun head_norm_dpair thy (env, (rbinder, t, u)) : dpair * Envir.env = |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
235 |
new_dpair thy (rbinder, |
19864 | 236 |
eta_norm env (rbinder, Envir.head_norm env t), |
52126 | 237 |
eta_norm env (rbinder, Envir.head_norm env u)) env; |
0 | 238 |
|
239 |
||
240 |
(*flexflex: the flex-flex pairs, flexrigid: the flex-rigid pairs |
|
241 |
Does not perform assignments for flex-flex pairs: |
|
646 | 242 |
may create nonrigid paths, which prevent other assignments. |
243 |
Does not even identify Vars in dpairs such as ?a =?= ?b; an attempt to |
|
244 |
do so caused numerous problems with no compensating advantage. |
|
245 |
*) |
|
48263 | 246 |
fun SIMPL0 thy dp0 (env,flexflex,flexrigid) : Envir.env * dpair list * dpair list = |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
247 |
let |
52179
3b9c31867707
more thorough type unification: treat equal Vars like other atoms, otherwise unify type of term pair (not just accidental body_type of its head Vars);
wenzelm
parents:
52128
diff
changeset
|
248 |
val (dp as (rbinder, t, u), env) = |
3b9c31867707
more thorough type unification: treat equal Vars like other atoms, otherwise unify type of term pair (not just accidental body_type of its head Vars);
wenzelm
parents:
52128
diff
changeset
|
249 |
head_norm_dpair thy (unify_types_of thy dp0 env, dp0); |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
250 |
fun SIMRANDS (f $ t, g $ u, env) = |
48263 | 251 |
SIMPL0 thy (rbinder, t, u) (SIMRANDS (f, g, env)) |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
252 |
| SIMRANDS (t as _$_, _, _) = |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
253 |
raise TERM ("SIMPL: operands mismatch", [t, u]) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
254 |
| SIMRANDS (t, u as _ $ _, _) = |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
255 |
raise TERM ("SIMPL: operands mismatch", [t, u]) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
256 |
| SIMRANDS (_, _, env) = (env, flexflex, flexrigid); |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
257 |
in |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
258 |
(case (head_of t, head_of u) of |
52179
3b9c31867707
more thorough type unification: treat equal Vars like other atoms, otherwise unify type of term pair (not just accidental body_type of its head Vars);
wenzelm
parents:
52128
diff
changeset
|
259 |
(Var (v, T), Var (w, U)) => |
3b9c31867707
more thorough type unification: treat equal Vars like other atoms, otherwise unify type of term pair (not just accidental body_type of its head Vars);
wenzelm
parents:
52128
diff
changeset
|
260 |
let val env' = if v = w then unify_types thy (T, U) env else env |
3b9c31867707
more thorough type unification: treat equal Vars like other atoms, otherwise unify type of term pair (not just accidental body_type of its head Vars);
wenzelm
parents:
52128
diff
changeset
|
261 |
in (env', dp :: flexflex, flexrigid) end |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
262 |
| (Var _, _) => |
52126 | 263 |
((assignment thy (rbinder,t,u) env, flexflex, flexrigid) |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
264 |
handle ASSIGN => (env, flexflex, dp :: flexrigid)) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
265 |
| (_, Var _) => |
52126 | 266 |
((assignment thy (rbinder, u, t) env, flexflex, flexrigid) |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
267 |
handle ASSIGN => (env, flexflex, (rbinder, u, t) :: flexrigid)) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
268 |
| (Const (a, T), Const (b, U)) => |
52126 | 269 |
if a = b then SIMRANDS (t, u, unify_types thy (T, U) env) |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
270 |
else raise CANTUNIFY |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
271 |
| (Bound i, Bound j) => |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
272 |
if i = j then SIMRANDS (t, u, env) else raise CANTUNIFY |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
273 |
| (Free (a, T), Free (b, U)) => |
52126 | 274 |
if a = b then SIMRANDS (t, u, unify_types thy (T, U) env) |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
275 |
else raise CANTUNIFY |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
276 |
| _ => raise CANTUNIFY) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
277 |
end; |
0 | 278 |
|
279 |
||
280 |
(* changed(env,t) checks whether the head of t is a variable assigned in env*) |
|
52126 | 281 |
fun changed env (f $ _) = changed env f |
282 |
| changed env (Var v) = (case Envir.lookup env v of NONE => false | _ => true) |
|
283 |
| changed _ _ = false; |
|
0 | 284 |
|
285 |
||
286 |
(*Recursion needed if any of the 'head variables' have been updated |
|
287 |
Clever would be to re-do just the affected dpairs*) |
|
16664 | 288 |
fun SIMPL thy (env,dpairs) : Envir.env * dpair list * dpair list = |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
289 |
let |
48263 | 290 |
val all as (env', flexflex, flexrigid) = fold_rev (SIMPL0 thy) dpairs (env, [], []); |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
291 |
val dps = flexrigid @ flexflex; |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
292 |
in |
52126 | 293 |
if exists (fn (_, t, u) => changed env' t orelse changed env' u) dps |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
294 |
then SIMPL thy (env', dps) else all |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
295 |
end; |
0 | 296 |
|
297 |
||
19864 | 298 |
(*Makes the terms E1,...,Em, where Ts = [T...Tm]. |
0 | 299 |
Each Ei is ?Gi(B.(n-1),...,B.0), and has type Ti |
300 |
The B.j are bound vars of binder. |
|
19864 | 301 |
The terms are not made in eta-normal-form, SIMPL does that later. |
0 | 302 |
If done here, eta-expansion must be recursive in the arguments! *) |
37636 | 303 |
fun make_args _ (_, env, []) = (env, []) (*frequent case*) |
0 | 304 |
| make_args name (binder: typ list, env, Ts) : Envir.env * term list = |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
305 |
let |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
306 |
fun funtype T = binder ---> T; |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
307 |
val (env', vars) = Envir.genvars name (env, map funtype Ts); |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
308 |
in (env', map (fn var => Logic.combound (var, 0, length binder)) vars) end; |
0 | 309 |
|
310 |
||
46219
426ed18eba43
discontinued old-style Term.list_abs in favour of plain Term.abs;
wenzelm
parents:
42279
diff
changeset
|
311 |
(*Abstraction over a list of types*) |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
312 |
fun types_abs ([], u) = u |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
313 |
| types_abs (T :: Ts, u) = Abs ("", T, types_abs (Ts, u)); |
0 | 314 |
|
315 |
(*Abstraction over the binder of a type*) |
|
52128
7f3549a316f4
tuned signature -- slightly more general operations (cf. term.ML);
wenzelm
parents:
52127
diff
changeset
|
316 |
fun type_abs (env, T, t) = types_abs (Envir.binder_types env ~1 T, t); |
0 | 317 |
|
318 |
||
319 |
(*MATCH taking "big steps". |
|
320 |
Copies u into the Var v, using projection on targs or imitation. |
|
321 |
A projection is allowed unless SIMPL raises an exception. |
|
322 |
Allocates new variables in projection on a higher-order argument, |
|
323 |
or if u is a variable (flex-flex dpair). |
|
324 |
Returns long sequence of every way of copying u, for backtracking |
|
325 |
For example, projection in ?b'(?a) may be wrong if other dpairs constrain ?a. |
|
19864 | 326 |
The order for trying projections is crucial in ?b'(?a) |
0 | 327 |
NB "vname" is only used in the call to make_args!! *) |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
328 |
fun matchcopy thy vname = |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
329 |
let |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
330 |
fun mc (rbinder, targs, u, ed as (env, dpairs)) : (term * (Envir.env * dpair list)) Seq.seq = |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
331 |
let |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
332 |
val trace_tps = Config.get_global thy trace_types; |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
333 |
(*Produce copies of uarg and cons them in front of uargs*) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
334 |
fun copycons uarg (uargs, (env, dpairs)) = |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
335 |
Seq.map (fn (uarg', ed') => (uarg' :: uargs, ed')) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
336 |
(mc (rbinder, targs,eta_norm env (rbinder, Envir.head_norm env uarg), |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
337 |
(env, dpairs))); |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
338 |
(*Produce sequence of all possible ways of copying the arg list*) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
339 |
fun copyargs [] = Seq.cons ([], ed) Seq.empty |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
340 |
| copyargs (uarg :: uargs) = Seq.maps (copycons uarg) (copyargs uargs); |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
341 |
val (uhead, uargs) = strip_comb u; |
52128
7f3549a316f4
tuned signature -- slightly more general operations (cf. term.ML);
wenzelm
parents:
52127
diff
changeset
|
342 |
val base = Envir.body_type env ~1 (fastype env (rbinder, uhead)); |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
343 |
fun joinargs (uargs', ed') = (list_comb (uhead, uargs'), ed'); |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
344 |
(*attempt projection on argument with given typ*) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
345 |
val Ts = map (curry (fastype env) rbinder) targs; |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
346 |
fun projenv (head, (Us, bary), targ, tail) = |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
347 |
let |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
348 |
val env = |
52126 | 349 |
if trace_tps then test_unify_types thy (base, bary) env |
350 |
else unify_types thy (base, bary) env |
|
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
351 |
in |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
352 |
Seq.make (fn () => |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
353 |
let |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
354 |
val (env', args) = make_args vname (Ts, env, Us); |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
355 |
(*higher-order projection: plug in targs for bound vars*) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
356 |
fun plugin arg = list_comb (head_of arg, targs); |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
357 |
val dp = (rbinder, list_comb (targ, map plugin args), u); |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
358 |
val (env2, frigid, fflex) = SIMPL thy (env', dp :: dpairs); |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
359 |
(*may raise exception CANTUNIFY*) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
360 |
in |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
361 |
SOME ((list_comb (head, args), (env2, frigid @ fflex)), tail) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
362 |
end handle CANTUNIFY => Seq.pull tail) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
363 |
end handle CANTUNIFY => tail; |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
364 |
(*make a list of projections*) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
365 |
fun make_projs (T::Ts, targ::targs) = |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
366 |
(Bound(length Ts), T, targ) :: make_projs (Ts,targs) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
367 |
| make_projs ([],[]) = [] |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
368 |
| make_projs _ = raise TERM ("make_projs", u::targs); |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
369 |
(*try projections and imitation*) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
370 |
fun matchfun ((bvar,T,targ)::projs) = |
52128
7f3549a316f4
tuned signature -- slightly more general operations (cf. term.ML);
wenzelm
parents:
52127
diff
changeset
|
371 |
(projenv(bvar, Envir.strip_type env ~1 T, targ, matchfun projs)) |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
372 |
| matchfun [] = (*imitation last of all*) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
373 |
(case uhead of |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
374 |
Const _ => Seq.map joinargs (copyargs uargs) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
375 |
| Free _ => Seq.map joinargs (copyargs uargs) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
376 |
| _ => Seq.empty) (*if Var, would be a loop!*) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
377 |
in |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
378 |
(case uhead of |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
379 |
Abs (a, T, body) => |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
380 |
Seq.map (fn (body', ed') => (Abs (a, T, body'), ed')) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
381 |
(mc ((a, T) :: rbinder, (map (incr_boundvars 1) targs) @ [Bound 0], body, ed)) |
37636 | 382 |
| Var (w, _) => |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
383 |
(*a flex-flex dpair: make variable for t*) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
384 |
let |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
385 |
val (env', newhd) = Envir.genvar (#1 w) (env, Ts ---> base); |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
386 |
val tabs = Logic.combound (newhd, 0, length Ts); |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
387 |
val tsub = list_comb (newhd, targs); |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
388 |
in Seq.single (tabs, (env', (rbinder, tsub, u) :: dpairs)) end |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
389 |
| _ => matchfun (rev (make_projs (Ts, targs)))) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
390 |
end; |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
391 |
in mc end; |
0 | 392 |
|
393 |
||
394 |
(*Call matchcopy to produce assignments to the variable in the dpair*) |
|
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
395 |
fun MATCH thy (env, (rbinder, t, u), dpairs) : (Envir.env * dpair list) Seq.seq = |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
396 |
let |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
397 |
val (Var (vT as (v, T)), targs) = strip_comb t; |
52128
7f3549a316f4
tuned signature -- slightly more general operations (cf. term.ML);
wenzelm
parents:
52127
diff
changeset
|
398 |
val Ts = Envir.binder_types env ~1 T; |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
399 |
fun new_dset (u', (env', dpairs')) = |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
400 |
(*if v was updated to s, must unify s with u' *) |
51700 | 401 |
(case Envir.lookup env' vT of |
402 |
NONE => (Envir.update (vT, types_abs (Ts, u')) env', dpairs') |
|
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
403 |
| SOME s => (env', ([], s, types_abs (Ts, u')) :: dpairs')); |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
404 |
in |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
405 |
Seq.map new_dset (matchcopy thy (#1 v) (rbinder, targs, u, (env, dpairs))) |
0 | 406 |
end; |
407 |
||
408 |
||
409 |
||
410 |
(**** Flex-flex processing ****) |
|
411 |
||
19864 | 412 |
(*At end of unification, do flex-flex assignments like ?a -> ?f(?b) |
0 | 413 |
Attempts to update t with u, raising ASSIGN if impossible*) |
19864 | 414 |
fun ff_assign thy (env, rbinder, t, u) : Envir.env = |
52179
3b9c31867707
more thorough type unification: treat equal Vars like other atoms, otherwise unify type of term pair (not just accidental body_type of its head Vars);
wenzelm
parents:
52128
diff
changeset
|
415 |
let val (n, (v, T)) = get_eta_var rbinder 0 t in |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
416 |
if occurs_terms (Unsynchronized.ref [], env, v, [u]) then raise ASSIGN |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
417 |
else |
52179
3b9c31867707
more thorough type unification: treat equal Vars like other atoms, otherwise unify type of term pair (not just accidental body_type of its head Vars);
wenzelm
parents:
52128
diff
changeset
|
418 |
let val env = unify_types thy (Envir.body_type env n T, fastype env (rbinder, u)) env |
3b9c31867707
more thorough type unification: treat equal Vars like other atoms, otherwise unify type of term pair (not just accidental body_type of its head Vars);
wenzelm
parents:
52128
diff
changeset
|
419 |
in Envir.vupdate ((v, T), Logic.rlist_abs (rbinder, u)) env end |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
420 |
end; |
0 | 421 |
|
422 |
||
37720
50a9e2fa4f6b
Unification (flexflex) bug fix; making "auto" deterministic
paulson
parents:
37637
diff
changeset
|
423 |
(*If an argument contains a banned Bound, then it should be deleted. |
50a9e2fa4f6b
Unification (flexflex) bug fix; making "auto" deterministic
paulson
parents:
37637
diff
changeset
|
424 |
But if the only path is flexible, this is difficult; the code gives up! |
50a9e2fa4f6b
Unification (flexflex) bug fix; making "auto" deterministic
paulson
parents:
37637
diff
changeset
|
425 |
In %x y.?a(x) =?= %x y.?b(?c(y)) should we instantiate ?b or ?c *) |
50a9e2fa4f6b
Unification (flexflex) bug fix; making "auto" deterministic
paulson
parents:
37637
diff
changeset
|
426 |
exception CHANGE_FAIL; (*flexible occurrence of banned variable, or other reason to quit*) |
50a9e2fa4f6b
Unification (flexflex) bug fix; making "auto" deterministic
paulson
parents:
37637
diff
changeset
|
427 |
|
50a9e2fa4f6b
Unification (flexflex) bug fix; making "auto" deterministic
paulson
parents:
37637
diff
changeset
|
428 |
|
0 | 429 |
(*Flex argument: a term, its type, and the index that refers to it.*) |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
430 |
type flarg = {t: term, T: typ, j: int}; |
0 | 431 |
|
432 |
(*Form the arguments into records for deletion/sorting.*) |
|
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
433 |
fun flexargs ([], [], []) = [] : flarg list |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
434 |
| flexargs (j :: js, t :: ts, T :: Ts) = {j = j, t = t, T = T} :: flexargs (js, ts, Ts) |
37720
50a9e2fa4f6b
Unification (flexflex) bug fix; making "auto" deterministic
paulson
parents:
37637
diff
changeset
|
435 |
| flexargs _ = raise CHANGE_FAIL; |
41422
8a765db7e0f8
uniform treatment of type vs. term environment (cf. b654fa27fbc4);
wenzelm
parents:
39997
diff
changeset
|
436 |
(*We give up if we see a variable of function type not applied to a full list of |
8a765db7e0f8
uniform treatment of type vs. term environment (cf. b654fa27fbc4);
wenzelm
parents:
39997
diff
changeset
|
437 |
arguments (remember, this code assumes that terms are fully eta-expanded). This situation |
37720
50a9e2fa4f6b
Unification (flexflex) bug fix; making "auto" deterministic
paulson
parents:
37637
diff
changeset
|
438 |
can occur if a type variable is instantiated with a function type. |
50a9e2fa4f6b
Unification (flexflex) bug fix; making "auto" deterministic
paulson
parents:
37637
diff
changeset
|
439 |
*) |
0 | 440 |
|
651
4b0455fbcc49
Pure/Unify/IMPROVING "CLEANING" OF FLEX-FLEX PAIRS: Old code would refuse
lcp
parents:
646
diff
changeset
|
441 |
(*Check whether the 'banned' bound var indices occur rigidly in t*) |
19864 | 442 |
fun rigid_bound (lev, banned) t = |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
443 |
let val (head,args) = strip_comb t in |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
444 |
(case head of |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
445 |
Bound i => |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
446 |
member (op =) banned (i - lev) orelse exists (rigid_bound (lev, banned)) args |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
447 |
| Var _ => false (*no rigid occurrences here!*) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
448 |
| Abs (_, _, u) => |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
449 |
rigid_bound (lev + 1, banned) u orelse |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
450 |
exists (rigid_bound (lev, banned)) args |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
451 |
| _ => exists (rigid_bound (lev, banned)) args) |
0 | 452 |
end; |
453 |
||
651
4b0455fbcc49
Pure/Unify/IMPROVING "CLEANING" OF FLEX-FLEX PAIRS: Old code would refuse
lcp
parents:
646
diff
changeset
|
454 |
(*Squash down indices at level >=lev to delete the banned from a term.*) |
4b0455fbcc49
Pure/Unify/IMPROVING "CLEANING" OF FLEX-FLEX PAIRS: Old code would refuse
lcp
parents:
646
diff
changeset
|
455 |
fun change_bnos banned = |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
456 |
let |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
457 |
fun change lev (Bound i) = |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
458 |
if i < lev then Bound i |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
459 |
else if member (op =) banned (i - lev) then |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
460 |
raise CHANGE_FAIL (**flexible occurrence: give up**) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
461 |
else Bound (i - length (filter (fn j => j < i - lev) banned)) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
462 |
| change lev (Abs (a, T, t)) = Abs (a, T, change(lev + 1) t) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
463 |
| change lev (t $ u) = change lev t $ change lev u |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
464 |
| change lev t = t; |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
465 |
in change 0 end; |
0 | 466 |
|
467 |
(*Change indices, delete the argument if it contains a banned Bound*) |
|
48263 | 468 |
fun change_arg banned {j, t, T} args : flarg list = |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
469 |
if rigid_bound (0, banned) t then args (*delete argument!*) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
470 |
else {j = j, t = change_bnos banned t, T = T} :: args; |
0 | 471 |
|
472 |
||
473 |
(*Sort the arguments to create assignments if possible: |
|
48262
a0d8abca8d7a
back to naive insertion sort before 1997 to accommodate peculiar less_arg relation -- NB: make_ord arg_less was not a quasi-order and thus inappropriate for generic sort (cf. de74b549f976, ecfeff48bf0c);
wenzelm
parents:
46219
diff
changeset
|
474 |
create eta-terms like ?g B.1 B.0*) |
a0d8abca8d7a
back to naive insertion sort before 1997 to accommodate peculiar less_arg relation -- NB: make_ord arg_less was not a quasi-order and thus inappropriate for generic sort (cf. de74b549f976, ecfeff48bf0c);
wenzelm
parents:
46219
diff
changeset
|
475 |
local |
a0d8abca8d7a
back to naive insertion sort before 1997 to accommodate peculiar less_arg relation -- NB: make_ord arg_less was not a quasi-order and thus inappropriate for generic sort (cf. de74b549f976, ecfeff48bf0c);
wenzelm
parents:
46219
diff
changeset
|
476 |
fun less_arg ({t = Bound i1, ...}, {t = Bound i2, ...}) = (i2 < i1) |
a0d8abca8d7a
back to naive insertion sort before 1997 to accommodate peculiar less_arg relation -- NB: make_ord arg_less was not a quasi-order and thus inappropriate for generic sort (cf. de74b549f976, ecfeff48bf0c);
wenzelm
parents:
46219
diff
changeset
|
477 |
| less_arg (_: flarg, _: flarg) = false; |
a0d8abca8d7a
back to naive insertion sort before 1997 to accommodate peculiar less_arg relation -- NB: make_ord arg_less was not a quasi-order and thus inappropriate for generic sort (cf. de74b549f976, ecfeff48bf0c);
wenzelm
parents:
46219
diff
changeset
|
478 |
|
a0d8abca8d7a
back to naive insertion sort before 1997 to accommodate peculiar less_arg relation -- NB: make_ord arg_less was not a quasi-order and thus inappropriate for generic sort (cf. de74b549f976, ecfeff48bf0c);
wenzelm
parents:
46219
diff
changeset
|
479 |
fun ins_arg x [] = [x] |
a0d8abca8d7a
back to naive insertion sort before 1997 to accommodate peculiar less_arg relation -- NB: make_ord arg_less was not a quasi-order and thus inappropriate for generic sort (cf. de74b549f976, ecfeff48bf0c);
wenzelm
parents:
46219
diff
changeset
|
480 |
| ins_arg x (y :: ys) = |
a0d8abca8d7a
back to naive insertion sort before 1997 to accommodate peculiar less_arg relation -- NB: make_ord arg_less was not a quasi-order and thus inappropriate for generic sort (cf. de74b549f976, ecfeff48bf0c);
wenzelm
parents:
46219
diff
changeset
|
481 |
if less_arg (y, x) then y :: ins_arg x ys else x :: y :: ys; |
a0d8abca8d7a
back to naive insertion sort before 1997 to accommodate peculiar less_arg relation -- NB: make_ord arg_less was not a quasi-order and thus inappropriate for generic sort (cf. de74b549f976, ecfeff48bf0c);
wenzelm
parents:
46219
diff
changeset
|
482 |
in |
a0d8abca8d7a
back to naive insertion sort before 1997 to accommodate peculiar less_arg relation -- NB: make_ord arg_less was not a quasi-order and thus inappropriate for generic sort (cf. de74b549f976, ecfeff48bf0c);
wenzelm
parents:
46219
diff
changeset
|
483 |
fun sort_args [] = [] |
a0d8abca8d7a
back to naive insertion sort before 1997 to accommodate peculiar less_arg relation -- NB: make_ord arg_less was not a quasi-order and thus inappropriate for generic sort (cf. de74b549f976, ecfeff48bf0c);
wenzelm
parents:
46219
diff
changeset
|
484 |
| sort_args (x :: xs) = ins_arg x (sort_args xs); |
a0d8abca8d7a
back to naive insertion sort before 1997 to accommodate peculiar less_arg relation -- NB: make_ord arg_less was not a quasi-order and thus inappropriate for generic sort (cf. de74b549f976, ecfeff48bf0c);
wenzelm
parents:
46219
diff
changeset
|
485 |
end; |
0 | 486 |
|
487 |
(*Test whether the new term would be eta-equivalent to a variable -- |
|
488 |
if so then there is no point in creating a new variable*) |
|
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
489 |
fun decreasing n ([]: flarg list) = (n = 0) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
490 |
| decreasing n ({j, ...} :: args) = j = n - 1 andalso decreasing (n - 1) args; |
0 | 491 |
|
492 |
(*Delete banned indices in the term, simplifying it. |
|
493 |
Force an assignment, if possible, by sorting the arguments. |
|
494 |
Update its head; squash indices in arguments. *) |
|
495 |
fun clean_term banned (env,t) = |
|
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
496 |
let |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
497 |
val (Var (v, T), ts) = strip_comb t; |
52128
7f3549a316f4
tuned signature -- slightly more general operations (cf. term.ML);
wenzelm
parents:
52127
diff
changeset
|
498 |
val (Ts, U) = Envir.strip_type env ~1 T |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
499 |
and js = length ts - 1 downto 0; |
48263 | 500 |
val args = sort_args (fold_rev (change_arg banned) (flexargs (js, ts, Ts)) []) |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
501 |
val ts' = map #t args; |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
502 |
in |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
503 |
if decreasing (length Ts) args then (env, (list_comb (Var (v, T), ts'))) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
504 |
else |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
505 |
let |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
506 |
val (env', v') = Envir.genvar (#1 v) (env, map #T args ---> U); |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
507 |
val body = list_comb (v', map (Bound o #j) args); |
51700 | 508 |
val env2 = Envir.vupdate ((v, T), types_abs (Ts, body)) env'; |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
509 |
(*the vupdate affects ts' if they contain v*) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
510 |
in (env2, Envir.norm_term env2 (list_comb (v', ts'))) end |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
511 |
end; |
0 | 512 |
|
513 |
||
514 |
(*Add tpair if not trivial or already there. |
|
515 |
Should check for swapped pairs??*) |
|
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
516 |
fun add_tpair (rbinder, (t0, u0), tpairs) : (term * term) list = |
19864 | 517 |
if t0 aconv u0 then tpairs |
0 | 518 |
else |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
519 |
let |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
520 |
val t = Logic.rlist_abs (rbinder, t0) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
521 |
and u = Logic.rlist_abs (rbinder, u0); |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
522 |
fun same (t', u') = (t aconv t') andalso (u aconv u') |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
523 |
in if exists same tpairs then tpairs else (t, u) :: tpairs end; |
0 | 524 |
|
525 |
||
526 |
(*Simplify both terms and check for assignments. |
|
527 |
Bound vars in the binder are "banned" unless used in both t AND u *) |
|
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
528 |
fun clean_ffpair thy ((rbinder, t, u), (env, tpairs)) = |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
529 |
let |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
530 |
val loot = loose_bnos t and loou = loose_bnos u |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
531 |
fun add_index (j, (a, T)) (bnos, newbinder) = |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
532 |
if member (op =) loot j andalso member (op =) loou j |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
533 |
then (bnos, (a, T) :: newbinder) (*needed by both: keep*) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
534 |
else (j :: bnos, newbinder); (*remove*) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
535 |
val (banned, rbin') = fold_rev add_index ((0 upto (length rbinder - 1)) ~~ rbinder) ([], []); |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
536 |
val (env', t') = clean_term banned (env, t); |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
537 |
val (env'',u') = clean_term banned (env',u); |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
538 |
in |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
539 |
(ff_assign thy (env'', rbin', t', u'), tpairs) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
540 |
handle ASSIGN => |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
541 |
(ff_assign thy (env'', rbin', u', t'), tpairs) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
542 |
handle ASSIGN => (env'', add_tpair (rbin', (t', u'), tpairs)) |
0 | 543 |
end |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
544 |
handle CHANGE_FAIL => (env, add_tpair (rbinder, (t, u), tpairs)); |
0 | 545 |
|
546 |
||
547 |
(*IF the flex-flex dpair is an assignment THEN do it ELSE put in tpairs |
|
548 |
eliminates trivial tpairs like t=t, as well as repeated ones |
|
19864 | 549 |
trivial tpairs can easily escape SIMPL: ?A=t, ?A=?B, ?B=t gives t=t |
0 | 550 |
Resulting tpairs MAY NOT be in normal form: assignments may occur here.*) |
48263 | 551 |
fun add_ffpair thy (rbinder,t0,u0) (env,tpairs) : Envir.env * (term * term) list = |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
552 |
let |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
553 |
val t = Envir.norm_term env t0 |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
554 |
and u = Envir.norm_term env u0; |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
555 |
in |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
556 |
(case (head_of t, head_of u) of |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
557 |
(Var (v, T), Var (w, U)) => (*Check for identical variables...*) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
558 |
if Term.eq_ix (v, w) then (*...occur check would falsely return true!*) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
559 |
if T = U then (env, add_tpair (rbinder, (t, u), tpairs)) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
560 |
else raise TERM ("add_ffpair: Var name confusion", [t, u]) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
561 |
else if Term_Ord.indexname_ord (v, w) = LESS then (*prefer to update the LARGER variable*) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
562 |
clean_ffpair thy ((rbinder, u, t), (env, tpairs)) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
563 |
else clean_ffpair thy ((rbinder, t, u), (env, tpairs)) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
564 |
| _ => raise TERM ("add_ffpair: Vars expected", [t, u])) |
0 | 565 |
end; |
566 |
||
567 |
||
568 |
(*Print a tracing message + list of dpairs. |
|
569 |
In t==u print u first because it may be rigid or flexible -- |
|
570 |
t is always flexible.*) |
|
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
571 |
fun print_dpairs thy msg (env, dpairs) = |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
572 |
let |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
573 |
fun pdp (rbinder, t, u) = |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
574 |
let |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
575 |
fun termT t = |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
576 |
Syntax.pretty_term_global thy (Envir.norm_term env (Logic.rlist_abs (rbinder, t))); |
42279
6da43a5018e2
constant =?= no longer exists (cf. 8c09e1fa24a7);
wenzelm
parents:
41422
diff
changeset
|
577 |
val bsymbs = [termT u, Pretty.str " =?=", Pretty.brk 1, termT t]; |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
578 |
in tracing (Pretty.string_of (Pretty.blk (0, bsymbs))) end; |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
579 |
in tracing msg; List.app pdp dpairs end; |
0 | 580 |
|
581 |
||
582 |
(*Unify the dpairs in the environment. |
|
19864 | 583 |
Returns flex-flex disagreement pairs NOT IN normal form. |
0 | 584 |
SIMPL may raise exception CANTUNIFY. *) |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
585 |
fun hounifiers (thy, env, tus : (term * term) list) : (Envir.env * (term * term) list) Seq.seq = |
24178
4ff1dc2aa18d
turned Unify flags into configuration options (global only);
wenzelm
parents:
23178
diff
changeset
|
586 |
let |
36787
f60e4dd6d76f
renamed Config.get_thy to Config.get_global etc. to indicate that this is not the real thing;
wenzelm
parents:
36001
diff
changeset
|
587 |
val trace_bnd = Config.get_global thy trace_bound; |
f60e4dd6d76f
renamed Config.get_thy to Config.get_global etc. to indicate that this is not the real thing;
wenzelm
parents:
36001
diff
changeset
|
588 |
val search_bnd = Config.get_global thy search_bound; |
f60e4dd6d76f
renamed Config.get_thy to Config.get_global etc. to indicate that this is not the real thing;
wenzelm
parents:
36001
diff
changeset
|
589 |
val trace_smp = Config.get_global thy trace_simp; |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
590 |
fun add_unify tdepth ((env, dpairs), reseq) = |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
591 |
Seq.make (fn () => |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
592 |
let |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
593 |
val (env', flexflex, flexrigid) = |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
594 |
(if tdepth > trace_bnd andalso trace_smp |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
595 |
then print_dpairs thy "Enter SIMPL" (env, dpairs) else (); |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
596 |
SIMPL thy (env, dpairs)); |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
597 |
in |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
598 |
(case flexrigid of |
48263 | 599 |
[] => SOME (fold_rev (add_ffpair thy) flexflex (env', []), reseq) |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
600 |
| dp :: frigid' => |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
601 |
if tdepth > search_bnd then |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
602 |
(warning "Unification bound exceeded"; Seq.pull reseq) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
603 |
else |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
604 |
(if tdepth > trace_bnd then |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
605 |
print_dpairs thy "Enter MATCH" (env',flexrigid@flexflex) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
606 |
else (); |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
607 |
Seq.pull (Seq.it_right |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
608 |
(add_unify (tdepth + 1)) (MATCH thy (env',dp, frigid'@flexflex), reseq)))) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
609 |
end |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
610 |
handle CANTUNIFY => |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
611 |
(if tdepth > trace_bnd then tracing"Failure node" else (); |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
612 |
Seq.pull reseq)); |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
613 |
val dps = map (fn (t, u) => ([], t, u)) tus; |
16425
2427be27cc60
accomodate identification of type Sign.sg and theory;
wenzelm
parents:
15797
diff
changeset
|
614 |
in add_unify 1 ((env, dps), Seq.empty) end; |
0 | 615 |
|
18184 | 616 |
fun unifiers (params as (thy, env, tus)) = |
19473 | 617 |
Seq.cons (fold (Pattern.unify thy) tus env, []) Seq.empty |
16425
2427be27cc60
accomodate identification of type Sign.sg and theory;
wenzelm
parents:
15797
diff
changeset
|
618 |
handle Pattern.Unif => Seq.empty |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
619 |
| Pattern.Pattern => hounifiers params; |
0 | 620 |
|
621 |
||
622 |
(*For smash_flexflex1*) |
|
623 |
fun var_head_of (env,t) : indexname * typ = |
|
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
624 |
(case head_of (strip_abs_body (Envir.norm_term env t)) of |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
625 |
Var (v, T) => (v, T) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
626 |
| _ => raise CANTUNIFY); (*not flexible, cannot use trivial substitution*) |
0 | 627 |
|
628 |
||
629 |
(*Eliminate a flex-flex pair by the trivial substitution, see Huet (1975) |
|
630 |
Unifies ?f(t1...rm) with ?g(u1...un) by ?f -> %x1...xm.?a, ?g -> %x1...xn.?a |
|
19864 | 631 |
Unfortunately, unifies ?f(t,u) with ?g(t,u) by ?f, ?g -> %(x,y)?a, |
632 |
though just ?g->?f is a more general unifier. |
|
0 | 633 |
Unlike Huet (1975), does not smash together all variables of same type -- |
634 |
requires more work yet gives a less general unifier (fewer variables). |
|
635 |
Handles ?f(t1...rm) with ?f(u1...um) to avoid multiple updates. *) |
|
48263 | 636 |
fun smash_flexflex1 (t, u) env : Envir.env = |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
637 |
let |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
638 |
val vT as (v, T) = var_head_of (env, t) |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
639 |
and wU as (w, U) = var_head_of (env, u); |
52128
7f3549a316f4
tuned signature -- slightly more general operations (cf. term.ML);
wenzelm
parents:
52127
diff
changeset
|
640 |
val (env', var) = Envir.genvar (#1 v) (env, Envir.body_type env ~1 T); |
51700 | 641 |
val env'' = Envir.vupdate (wU, type_abs (env', U, var)) env'; |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
642 |
in |
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
643 |
if vT = wU then env'' (*the other update would be identical*) |
51700 | 644 |
else Envir.vupdate (vT, type_abs (env', T, var)) env'' |
0 | 645 |
end; |
646 |
||
647 |
||
648 |
(*Smash all flex-flexpairs. Should allow selection of pairs by a predicate?*) |
|
37636 | 649 |
fun smash_flexflex (env, tpairs) : Envir.env = |
48263 | 650 |
fold_rev smash_flexflex1 tpairs env; |
0 | 651 |
|
652 |
(*Returns unifiers with no remaining disagreement pairs*) |
|
19864 | 653 |
fun smash_unifiers thy tus env = |
37635
484efa650907
recovered some indentation from the depths of time;
wenzelm
parents:
36787
diff
changeset
|
654 |
Seq.map smash_flexflex (unifiers (thy, env, tus)); |
0 | 655 |
|
19864 | 656 |
|
657 |
(*Pattern matching*) |
|
32032 | 658 |
fun first_order_matchers thy pairs (Envir.Envir {maxidx, tenv, tyenv}) = |
20020
9e7d3d06c643
matchers: fall back on plain first_order_matchers, not pattern;
wenzelm
parents:
19920
diff
changeset
|
659 |
let val (tyenv', tenv') = fold (Pattern.first_order_match thy) pairs (tyenv, tenv) |
32032 | 660 |
in Seq.single (Envir.Envir {maxidx = maxidx, tenv = tenv', tyenv = tyenv'}) end |
19864 | 661 |
handle Pattern.MATCH => Seq.empty; |
662 |
||
41422
8a765db7e0f8
uniform treatment of type vs. term environment (cf. b654fa27fbc4);
wenzelm
parents:
39997
diff
changeset
|
663 |
(*General matching -- keep variables disjoint*) |
19864 | 664 |
fun matchers _ [] = Seq.single (Envir.empty ~1) |
665 |
| matchers thy pairs = |
|
666 |
let |
|
667 |
val maxidx = fold (Term.maxidx_term o #2) pairs ~1; |
|
668 |
val offset = maxidx + 1; |
|
669 |
val pairs' = map (apfst (Logic.incr_indexes ([], offset))) pairs; |
|
670 |
val maxidx' = fold (fn (t, u) => Term.maxidx_term t #> Term.maxidx_term u) pairs' ~1; |
|
671 |
||
672 |
val pat_tvars = fold (Term.add_tvars o #1) pairs' []; |
|
673 |
val pat_vars = fold (Term.add_vars o #1) pairs' []; |
|
674 |
||
675 |
val decr_indexesT = |
|
676 |
Term.map_atyps (fn T as TVar ((x, i), S) => |
|
677 |
if i > maxidx then TVar ((x, i - offset), S) else T | T => T); |
|
678 |
val decr_indexes = |
|
20548
8ef25fe585a8
renamed Term.map_term_types to Term.map_types (cf. Term.fold_types);
wenzelm
parents:
20098
diff
changeset
|
679 |
Term.map_types decr_indexesT #> |
19864 | 680 |
Term.map_aterms (fn t as Var ((x, i), T) => |
681 |
if i > maxidx then Var ((x, i - offset), T) else t | t => t); |
|
682 |
||
32032 | 683 |
fun norm_tvar env ((x, i), S) = |
41422
8a765db7e0f8
uniform treatment of type vs. term environment (cf. b654fa27fbc4);
wenzelm
parents:
39997
diff
changeset
|
684 |
let |
8a765db7e0f8
uniform treatment of type vs. term environment (cf. b654fa27fbc4);
wenzelm
parents:
39997
diff
changeset
|
685 |
val tyenv = Envir.type_env env; |
8a765db7e0f8
uniform treatment of type vs. term environment (cf. b654fa27fbc4);
wenzelm
parents:
39997
diff
changeset
|
686 |
val T' = Envir.norm_type tyenv (TVar ((x, i), S)); |
8a765db7e0f8
uniform treatment of type vs. term environment (cf. b654fa27fbc4);
wenzelm
parents:
39997
diff
changeset
|
687 |
in |
8a765db7e0f8
uniform treatment of type vs. term environment (cf. b654fa27fbc4);
wenzelm
parents:
39997
diff
changeset
|
688 |
if (case T' of TVar (v, _) => v = (x, i) | _ => false) then NONE |
8a765db7e0f8
uniform treatment of type vs. term environment (cf. b654fa27fbc4);
wenzelm
parents:
39997
diff
changeset
|
689 |
else SOME ((x, i - offset), (S, decr_indexesT T')) |
8a765db7e0f8
uniform treatment of type vs. term environment (cf. b654fa27fbc4);
wenzelm
parents:
39997
diff
changeset
|
690 |
end; |
8a765db7e0f8
uniform treatment of type vs. term environment (cf. b654fa27fbc4);
wenzelm
parents:
39997
diff
changeset
|
691 |
|
32032 | 692 |
fun norm_var env ((x, i), T) = |
19864 | 693 |
let |
32032 | 694 |
val tyenv = Envir.type_env env; |
19864 | 695 |
val T' = Envir.norm_type tyenv T; |
696 |
val t' = Envir.norm_term env (Var ((x, i), T')); |
|
41422
8a765db7e0f8
uniform treatment of type vs. term environment (cf. b654fa27fbc4);
wenzelm
parents:
39997
diff
changeset
|
697 |
in |
8a765db7e0f8
uniform treatment of type vs. term environment (cf. b654fa27fbc4);
wenzelm
parents:
39997
diff
changeset
|
698 |
if (case t' of Var (v, _) => v = (x, i) | _ => false) then NONE |
8a765db7e0f8
uniform treatment of type vs. term environment (cf. b654fa27fbc4);
wenzelm
parents:
39997
diff
changeset
|
699 |
else SOME ((x, i - offset), (decr_indexesT T', decr_indexes t')) |
8a765db7e0f8
uniform treatment of type vs. term environment (cf. b654fa27fbc4);
wenzelm
parents:
39997
diff
changeset
|
700 |
end; |
19864 | 701 |
|
702 |
fun result env = |
|
19876 | 703 |
if Envir.above env maxidx then (* FIXME proper handling of generated vars!? *) |
19864 | 704 |
SOME (Envir.Envir {maxidx = maxidx, |
41422
8a765db7e0f8
uniform treatment of type vs. term environment (cf. b654fa27fbc4);
wenzelm
parents:
39997
diff
changeset
|
705 |
tyenv = Vartab.make (map_filter (norm_tvar env) pat_tvars), |
8a765db7e0f8
uniform treatment of type vs. term environment (cf. b654fa27fbc4);
wenzelm
parents:
39997
diff
changeset
|
706 |
tenv = Vartab.make (map_filter (norm_var env) pat_vars)}) |
19866 | 707 |
else NONE; |
19864 | 708 |
|
709 |
val empty = Envir.empty maxidx'; |
|
710 |
in |
|
19876 | 711 |
Seq.append |
19920
8257e52164a1
matchers: try pattern_matchers only *after* general matching (The
wenzelm
parents:
19876
diff
changeset
|
712 |
(Seq.map_filter result (smash_unifiers thy pairs' empty)) |
20020
9e7d3d06c643
matchers: fall back on plain first_order_matchers, not pattern;
wenzelm
parents:
19920
diff
changeset
|
713 |
(first_order_matchers thy pairs empty) |
19864 | 714 |
end; |
715 |
||
716 |
fun matches_list thy ps os = |
|
717 |
length ps = length os andalso is_some (Seq.pull (matchers thy (ps ~~ os))); |
|
718 |
||
0 | 719 |
end; |