author | nipkow |
Wed, 06 May 2009 09:58:24 +0200 | |
changeset 31043 | df5ade763445 |
parent 30970 | 3fe2e418a071 |
child 31049 | 396d4d6a1594 |
permissions | -rw-r--r-- |
24590 | 1 |
(* Title: Tools/nbe.ML |
24155 | 2 |
Authors: Klaus Aehlig, LMU Muenchen; Tobias Nipkow, Florian Haftmann, TU Muenchen |
3 |
||
24839 | 4 |
Normalization by evaluation, based on generic code generator. |
24155 | 5 |
*) |
6 |
||
7 |
signature NBE = |
|
8 |
sig |
|
25101 | 9 |
val norm_conv: cterm -> thm |
30970
3fe2e418a071
generic postprocessing scheme for term evaluations
haftmann
parents:
30947
diff
changeset
|
10 |
val norm: theory -> term -> term |
25101 | 11 |
|
25204 | 12 |
datatype Univ = |
26064 | 13 |
Const of int * Univ list (*named (uninterpreted) constants*) |
25924 | 14 |
| Free of string * Univ list (*free (uninterpreted) variables*) |
15 |
| DFree of string * int (*free (uninterpreted) dictionary parameters*) |
|
24155 | 16 |
| BVar of int * Univ list |
28350 | 17 |
| Abs of (int * (Univ list -> Univ)) * Univ list |
25924 | 18 |
val apps: Univ -> Univ list -> Univ (*explicit applications*) |
25944 | 19 |
val abss: int -> (Univ list -> Univ) -> Univ |
28337 | 20 |
(*abstractions as closures*) |
28350 | 21 |
val same: Univ -> Univ -> bool |
24155 | 22 |
|
25204 | 23 |
val univs_ref: (unit -> Univ list -> Univ list) option ref |
24155 | 24 |
val trace: bool ref |
25924 | 25 |
|
26747
f32fa5f5bdd1
moved 'trivial classes' to foundation of code generator
haftmann
parents:
26739
diff
changeset
|
26 |
val setup: theory -> theory |
24155 | 27 |
end; |
28 |
||
29 |
structure Nbe: NBE = |
|
30 |
struct |
|
31 |
||
32 |
(* generic non-sense *) |
|
33 |
||
34 |
val trace = ref false; |
|
35 |
fun tracing f x = if !trace then (Output.tracing (f x); x) else x; |
|
36 |
||
37 |
||
38 |
(** the semantical universe **) |
|
39 |
||
40 |
(* |
|
41 |
Functions are given by their semantical function value. To avoid |
|
42 |
trouble with the ML-type system, these functions have the most |
|
43 |
generic type, that is "Univ list -> Univ". The calling convention is |
|
44 |
that the arguments come as a list, the last argument first. In |
|
45 |
other words, a function call that usually would look like |
|
46 |
||
47 |
f x_1 x_2 ... x_n or f(x_1,x_2, ..., x_n) |
|
48 |
||
49 |
would be in our convention called as |
|
50 |
||
51 |
f [x_n,..,x_2,x_1] |
|
52 |
||
53 |
Moreover, to handle functions that are still waiting for some |
|
54 |
arguments we have additionally a list of arguments collected to far |
|
55 |
and the number of arguments we're still waiting for. |
|
56 |
*) |
|
57 |
||
25204 | 58 |
datatype Univ = |
26064 | 59 |
Const of int * Univ list (*named (uninterpreted) constants*) |
24155 | 60 |
| Free of string * Univ list (*free variables*) |
25924 | 61 |
| DFree of string * int (*free (uninterpreted) dictionary parameters*) |
27499 | 62 |
| BVar of int * Univ list (*bound variables, named*) |
24155 | 63 |
| Abs of (int * (Univ list -> Univ)) * Univ list |
27499 | 64 |
(*abstractions as closures*); |
24155 | 65 |
|
28350 | 66 |
fun same (Const (k, xs)) (Const (l, ys)) = k = l andalso sames xs ys |
67 |
| same (Free (s, xs)) (Free (t, ys)) = s = t andalso sames xs ys |
|
68 |
| same (DFree (s, k)) (DFree (t, l)) = s = t andalso k = l |
|
69 |
| same (BVar (k, xs)) (BVar (l, ys)) = k = l andalso sames xs ys |
|
70 |
| same _ _ = false |
|
71 |
and sames xs ys = length xs = length ys andalso forall (uncurry same) (xs ~~ ys); |
|
72 |
||
24155 | 73 |
(* constructor functions *) |
74 |
||
25944 | 75 |
fun abss n f = Abs ((n, f), []); |
25924 | 76 |
fun apps (Abs ((n, f), xs)) ys = let val k = n - length ys in |
27499 | 77 |
case int_ord (k, 0) |
78 |
of EQUAL => f (ys @ xs) |
|
79 |
| LESS => let val (zs, ws) = chop (~ k) ys in apps (f (ws @ xs)) zs end |
|
80 |
| GREATER => Abs ((k, f), ys @ xs) (*note: reverse convention also for apps!*) |
|
81 |
end |
|
25924 | 82 |
| apps (Const (name, xs)) ys = Const (name, ys @ xs) |
83 |
| apps (Free (name, xs)) ys = Free (name, ys @ xs) |
|
27499 | 84 |
| apps (BVar (n, xs)) ys = BVar (n, ys @ xs); |
24155 | 85 |
|
86 |
||
87 |
(** assembling and compiling ML code from terms **) |
|
88 |
||
89 |
(* abstract ML syntax *) |
|
90 |
||
91 |
infix 9 `$` `$$`; |
|
92 |
fun e1 `$` e2 = "(" ^ e1 ^ " " ^ e2 ^ ")"; |
|
25101 | 93 |
fun e `$$` [] = e |
94 |
| e `$$` es = "(" ^ e ^ " " ^ space_implode " " es ^ ")"; |
|
24590 | 95 |
fun ml_abs v e = "(fn " ^ v ^ " => " ^ e ^ ")"; |
24155 | 96 |
|
97 |
fun ml_cases t cs = |
|
98 |
"(case " ^ t ^ " of " ^ space_implode " | " (map (fn (p, t) => p ^ " => " ^ t) cs) ^ ")"; |
|
25944 | 99 |
fun ml_Let d e = "let\n" ^ d ^ " in " ^ e ^ " end"; |
28337 | 100 |
fun ml_as v t = "(" ^ v ^ " as " ^ t ^ ")"; |
24155 | 101 |
|
28350 | 102 |
fun ml_and [] = "true" |
103 |
| ml_and [x] = x |
|
104 |
| ml_and xs = "(" ^ space_implode " andalso " xs ^ ")"; |
|
105 |
fun ml_if b x y = "(if " ^ b ^ " then " ^ x ^ " else " ^ y ^ ")"; |
|
106 |
||
24155 | 107 |
fun ml_list es = "[" ^ commas es ^ "]"; |
108 |
||
109 |
fun ml_fundefs ([(name, [([], e)])]) = |
|
110 |
"val " ^ name ^ " = " ^ e ^ "\n" |
|
111 |
| ml_fundefs (eqs :: eqss) = |
|
112 |
let |
|
113 |
fun fundef (name, eqs) = |
|
114 |
let |
|
115 |
fun eqn (es, e) = name ^ " " ^ space_implode " " es ^ " = " ^ e |
|
116 |
in space_implode "\n | " (map eqn eqs) end; |
|
117 |
in |
|
118 |
(prefix "fun " o fundef) eqs :: map (prefix "and " o fundef) eqss |
|
26931 | 119 |
|> cat_lines |
24155 | 120 |
|> suffix "\n" |
121 |
end; |
|
122 |
||
25944 | 123 |
(* nbe specific syntax and sandbox communication *) |
124 |
||
125 |
val univs_ref = ref (NONE : (unit -> Univ list -> Univ list) option); |
|
24155 | 126 |
|
127 |
local |
|
28350 | 128 |
val prefix = "Nbe."; |
129 |
val name_ref = prefix ^ "univs_ref"; |
|
130 |
val name_const = prefix ^ "Const"; |
|
131 |
val name_abss = prefix ^ "abss"; |
|
132 |
val name_apps = prefix ^ "apps"; |
|
133 |
val name_same = prefix ^ "same"; |
|
24155 | 134 |
in |
135 |
||
25944 | 136 |
val univs_cookie = (name_ref, univs_ref); |
137 |
||
28337 | 138 |
fun nbe_fun 0 "" = "nbe_value" |
139 |
| nbe_fun i c = "c_" ^ translate_string (fn "." => "_" | c => c) c ^ "_" ^ string_of_int i; |
|
25101 | 140 |
fun nbe_dict v n = "d_" ^ v ^ "_" ^ string_of_int n; |
24155 | 141 |
fun nbe_bound v = "v_" ^ v; |
28337 | 142 |
fun nbe_default v = "w_" ^ v; |
24155 | 143 |
|
25924 | 144 |
(*note: these three are the "turning spots" where proper argument order is established!*) |
145 |
fun nbe_apps t [] = t |
|
146 |
| nbe_apps t ts = name_apps `$$` [t, ml_list (rev ts)]; |
|
28337 | 147 |
fun nbe_apps_local i c ts = nbe_fun i c `$` ml_list (rev ts); |
148 |
fun nbe_apps_constr idx_of c ts = |
|
149 |
let |
|
150 |
val c' = if !trace then string_of_int (idx_of c) ^ " (*" ^ c ^ "*)" |
|
151 |
else string_of_int (idx_of c); |
|
152 |
in name_const `$` ("(" ^ c' ^ ", " ^ ml_list (rev ts) ^ ")") end; |
|
25924 | 153 |
|
24155 | 154 |
fun nbe_abss 0 f = f `$` ml_list [] |
25944 | 155 |
| nbe_abss n f = name_abss `$$` [string_of_int n, f]; |
24155 | 156 |
|
28350 | 157 |
fun nbe_same v1 v2 = "(" ^ name_same ^ " " ^ nbe_bound v1 ^ " " ^ nbe_bound v2 ^ ")"; |
158 |
||
24155 | 159 |
end; |
160 |
||
28054 | 161 |
open Basic_Code_Thingol; |
24155 | 162 |
|
25865 | 163 |
(* code generation *) |
24155 | 164 |
|
26064 | 165 |
fun assemble_eqnss idx_of deps eqnss = |
25944 | 166 |
let |
167 |
fun prep_eqns (c, (vs, eqns)) = |
|
25924 | 168 |
let |
25944 | 169 |
val dicts = maps (fn (v, sort) => map_index (nbe_dict v o fst) sort) vs; |
28337 | 170 |
val num_args = length dicts + ((length o fst o hd) eqns); |
25944 | 171 |
in (c, (num_args, (dicts, eqns))) end; |
172 |
val eqnss' = map prep_eqns eqnss; |
|
173 |
||
174 |
fun assemble_constapp c dss ts = |
|
175 |
let |
|
176 |
val ts' = (maps o map) assemble_idict dss @ ts; |
|
177 |
in case AList.lookup (op =) eqnss' c |
|
28337 | 178 |
of SOME (num_args, _) => if num_args <= length ts' |
179 |
then let val (ts1, ts2) = chop num_args ts' |
|
180 |
in nbe_apps (nbe_apps_local 0 c ts1) ts2 |
|
181 |
end else nbe_apps (nbe_abss num_args (nbe_fun 0 c)) ts' |
|
25944 | 182 |
| NONE => if member (op =) deps c |
28337 | 183 |
then nbe_apps (nbe_fun 0 c) ts' |
184 |
else nbe_apps_constr idx_of c ts' |
|
25924 | 185 |
end |
25944 | 186 |
and assemble_idict (DictConst (inst, dss)) = |
187 |
assemble_constapp inst dss [] |
|
188 |
| assemble_idict (DictVar (supers, (v, (n, _)))) = |
|
189 |
fold_rev (fn super => assemble_constapp super [] o single) supers (nbe_dict v n); |
|
25924 | 190 |
|
28350 | 191 |
fun assemble_iterm constapp = |
24155 | 192 |
let |
28350 | 193 |
fun of_iterm match_cont t = |
25944 | 194 |
let |
28054 | 195 |
val (t', ts) = Code_Thingol.unfold_app t |
28350 | 196 |
in of_iapp match_cont t' (fold_rev (cons o of_iterm NONE) ts []) end |
197 |
and of_iapp match_cont (IConst (c, (dss, _))) ts = constapp c dss ts |
|
198 |
| of_iapp match_cont (IVar v) ts = nbe_apps (nbe_bound v) ts |
|
199 |
| of_iapp match_cont ((v, _) `|-> t) ts = |
|
200 |
nbe_apps (nbe_abss 1 (ml_abs (ml_list [nbe_bound v]) (of_iterm NONE t))) ts |
|
201 |
| of_iapp match_cont (ICase (((t, _), cs), t0)) ts = |
|
202 |
nbe_apps (ml_cases (of_iterm NONE t) |
|
203 |
(map (fn (p, t) => (of_iterm NONE p, of_iterm match_cont t)) cs |
|
204 |
@ [("_", case match_cont of SOME s => s | NONE => of_iterm NONE t0)])) ts |
|
25944 | 205 |
in of_iterm end; |
24155 | 206 |
|
28350 | 207 |
fun subst_nonlin_vars args = |
208 |
let |
|
209 |
val vs = (fold o Code_Thingol.fold_varnames) |
|
210 |
(fn v => AList.map_default (op =) (v, 0) (curry (op +) 1)) args []; |
|
211 |
val names = Name.make_context (map fst vs); |
|
212 |
fun declare v k ctxt = let val vs = Name.invents ctxt v k |
|
213 |
in (vs, fold Name.declare vs ctxt) end; |
|
214 |
val (vs_renames, _) = fold_map (fn (v, k) => if k > 1 |
|
215 |
then declare v (k - 1) #>> (fn vs => (v, vs)) |
|
216 |
else pair (v, [])) vs names; |
|
217 |
val samepairs = maps (fn (v, vs) => map (pair v) vs) vs_renames; |
|
218 |
fun subst_vars (t as IConst _) samepairs = (t, samepairs) |
|
219 |
| subst_vars (t as IVar v) samepairs = (case AList.lookup (op =) samepairs v |
|
220 |
of SOME v' => (IVar v', AList.delete (op =) v samepairs) |
|
221 |
| NONE => (t, samepairs)) |
|
222 |
| subst_vars (t1 `$ t2) samepairs = samepairs |
|
223 |
|> subst_vars t1 |
|
224 |
||>> subst_vars t2 |
|
225 |
|>> (op `$) |
|
226 |
| subst_vars (ICase (_, t)) samepairs = subst_vars t samepairs; |
|
227 |
val (args', _) = fold_map subst_vars args samepairs; |
|
228 |
in (samepairs, args') end; |
|
229 |
||
28337 | 230 |
fun assemble_eqn c dicts default_args (i, (args, rhs)) = |
231 |
let |
|
232 |
val is_eval = (c = ""); |
|
233 |
val default_rhs = nbe_apps_local (i+1) c (dicts @ default_args); |
|
234 |
val match_cont = if is_eval then NONE else SOME default_rhs; |
|
28350 | 235 |
val assemble_arg = assemble_iterm |
236 |
(fn c => fn _ => fn ts => nbe_apps_constr idx_of c ts) NONE; |
|
237 |
val assemble_rhs = assemble_iterm assemble_constapp match_cont ; |
|
238 |
val (samepairs, args') = subst_nonlin_vars args; |
|
239 |
val s_args = map assemble_arg args'; |
|
240 |
val s_rhs = if null samepairs then assemble_rhs rhs |
|
241 |
else ml_if (ml_and (map (uncurry nbe_same) samepairs)) |
|
242 |
(assemble_rhs rhs) default_rhs; |
|
28337 | 243 |
val eqns = if is_eval then |
28350 | 244 |
[([ml_list (rev (dicts @ s_args))], s_rhs)] |
28337 | 245 |
else |
28350 | 246 |
[([ml_list (rev (dicts @ map2 ml_as default_args s_args))], s_rhs), |
28337 | 247 |
([ml_list (rev (dicts @ default_args))], default_rhs)] |
248 |
in (nbe_fun i c, eqns) end; |
|
249 |
||
25944 | 250 |
fun assemble_eqns (c, (num_args, (dicts, eqns))) = |
251 |
let |
|
28337 | 252 |
val default_args = map nbe_default |
253 |
(Name.invent_list [] "a" (num_args - length dicts)); |
|
254 |
val eqns' = map_index (assemble_eqn c dicts default_args) eqns |
|
255 |
@ (if c = "" then [] else [(nbe_fun (length eqns) c, |
|
256 |
[([ml_list (rev (dicts @ default_args))], |
|
257 |
nbe_apps_constr idx_of c (dicts @ default_args))])]); |
|
258 |
in (eqns', nbe_abss num_args (nbe_fun 0 c)) end; |
|
24155 | 259 |
|
25944 | 260 |
val (fun_vars, fun_vals) = map_split assemble_eqns eqnss'; |
28337 | 261 |
val deps_vars = ml_list (map (nbe_fun 0) deps); |
262 |
in ml_abs deps_vars (ml_Let (ml_fundefs (flat fun_vars)) (ml_list fun_vals)) end; |
|
25944 | 263 |
|
264 |
(* code compilation *) |
|
265 |
||
28274
9873697fa411
ML_Context.evaluate: proper context (for ML environment);
wenzelm
parents:
28227
diff
changeset
|
266 |
fun compile_eqnss _ gr raw_deps [] = [] |
9873697fa411
ML_Context.evaluate: proper context (for ML environment);
wenzelm
parents:
28227
diff
changeset
|
267 |
| compile_eqnss ctxt gr raw_deps eqnss = |
24155 | 268 |
let |
26064 | 269 |
val (deps, deps_vals) = split_list (map_filter |
270 |
(fn dep => Option.map (fn univ => (dep, univ)) (fst ((Graph.get_node gr dep)))) raw_deps); |
|
271 |
val idx_of = raw_deps |
|
272 |
|> map (fn dep => (dep, snd (Graph.get_node gr dep))) |
|
273 |
|> AList.lookup (op =) |
|
274 |
|> (fn f => the o f); |
|
275 |
val s = assemble_eqnss idx_of deps eqnss; |
|
24155 | 276 |
val cs = map fst eqnss; |
25944 | 277 |
in |
278 |
s |
|
279 |
|> tracing (fn s => "\n--- code to be evaluated:\n" ^ s) |
|
30672
beaadd5af500
more systematic type use_context, with particular values ML_Parse.global_context and ML_Context.local_context;
wenzelm
parents:
30288
diff
changeset
|
280 |
|> ML_Context.evaluate ctxt (!trace) univs_cookie |
25944 | 281 |
|> (fn f => f deps_vals) |
282 |
|> (fn univs => cs ~~ univs) |
|
283 |
end; |
|
25190 | 284 |
|
30672
beaadd5af500
more systematic type use_context, with particular values ML_Parse.global_context and ML_Context.local_context;
wenzelm
parents:
30288
diff
changeset
|
285 |
|
25944 | 286 |
(* preparing function equations *) |
24155 | 287 |
|
28663
bd8438543bf2
code identifier namings are no longer imperative
haftmann
parents:
28423
diff
changeset
|
288 |
fun eqns_of_stmt (_, Code_Thingol.Fun (_, (_, []))) = |
25101 | 289 |
[] |
28663
bd8438543bf2
code identifier namings are no longer imperative
haftmann
parents:
28423
diff
changeset
|
290 |
| eqns_of_stmt (const, Code_Thingol.Fun (_, ((vs, _), eqns))) = |
25101 | 291 |
[(const, (vs, map fst eqns))] |
28054 | 292 |
| eqns_of_stmt (_, Code_Thingol.Datatypecons _) = |
25101 | 293 |
[] |
28054 | 294 |
| eqns_of_stmt (_, Code_Thingol.Datatype _) = |
25101 | 295 |
[] |
28663
bd8438543bf2
code identifier namings are no longer imperative
haftmann
parents:
28423
diff
changeset
|
296 |
| eqns_of_stmt (class, Code_Thingol.Class (_, (v, (superclasses, classops)))) = |
25101 | 297 |
let |
298 |
val names = map snd superclasses @ map fst classops; |
|
299 |
val params = Name.invent_list [] "d" (length names); |
|
300 |
fun mk (k, name) = |
|
301 |
(name, ([(v, [])], |
|
302 |
[([IConst (class, ([], [])) `$$ map IVar params], IVar (nth params k))])); |
|
303 |
in map_index mk names end |
|
28054 | 304 |
| eqns_of_stmt (_, Code_Thingol.Classrel _) = |
25101 | 305 |
[] |
28054 | 306 |
| eqns_of_stmt (_, Code_Thingol.Classparam _) = |
25101 | 307 |
[] |
28054 | 308 |
| eqns_of_stmt (inst, Code_Thingol.Classinst ((class, (_, arities)), (superinsts, instops))) = |
25101 | 309 |
[(inst, (arities, [([], IConst (class, ([], [])) `$$ |
310 |
map (fn (_, (_, (inst, dicts))) => IConst (inst, (dicts, []))) superinsts |
|
311 |
@ map (IConst o snd o fst) instops)]))]; |
|
24155 | 312 |
|
28274
9873697fa411
ML_Context.evaluate: proper context (for ML environment);
wenzelm
parents:
28227
diff
changeset
|
313 |
fun compile_stmts ctxt stmts_deps = |
25101 | 314 |
let |
315 |
val names = map (fst o fst) stmts_deps; |
|
316 |
val names_deps = map (fn ((name, _), deps) => (name, deps)) stmts_deps; |
|
317 |
val eqnss = maps (eqns_of_stmt o fst) stmts_deps; |
|
26064 | 318 |
val refl_deps = names_deps |
25190 | 319 |
|> maps snd |
320 |
|> distinct (op =) |
|
26064 | 321 |
|> fold (insert (op =)) names; |
322 |
fun new_node name (gr, (maxidx, idx_tab)) = if can (Graph.get_node gr) name |
|
323 |
then (gr, (maxidx, idx_tab)) |
|
324 |
else (Graph.new_node (name, (NONE, maxidx)) gr, |
|
325 |
(maxidx + 1, Inttab.update_new (maxidx, name) idx_tab)); |
|
25190 | 326 |
fun compile gr = eqnss |
28274
9873697fa411
ML_Context.evaluate: proper context (for ML environment);
wenzelm
parents:
28227
diff
changeset
|
327 |
|> compile_eqnss ctxt gr refl_deps |
25190 | 328 |
|> rpair gr; |
25101 | 329 |
in |
26064 | 330 |
fold new_node refl_deps |
331 |
#> apfst (fold (fn (name, deps) => fold (curry Graph.add_edge name) deps) names_deps |
|
332 |
#> compile |
|
333 |
#-> fold (fn (name, univ) => (Graph.map_node name o apfst) (K (SOME univ)))) |
|
25101 | 334 |
end; |
24155 | 335 |
|
28706 | 336 |
fun ensure_stmts ctxt naming program = |
25101 | 337 |
let |
26064 | 338 |
fun add_stmts names (gr, (maxidx, idx_tab)) = if exists ((can o Graph.get_node) gr) names |
339 |
then (gr, (maxidx, idx_tab)) |
|
340 |
else (gr, (maxidx, idx_tab)) |
|
28274
9873697fa411
ML_Context.evaluate: proper context (for ML environment);
wenzelm
parents:
28227
diff
changeset
|
341 |
|> compile_stmts ctxt (map (fn name => ((name, Graph.get_node program name), |
27103 | 342 |
Graph.imm_succs program name)) names); |
28706 | 343 |
in |
344 |
fold_rev add_stmts (Graph.strong_conn program) |
|
345 |
#> pair naming |
|
346 |
end; |
|
24155 | 347 |
|
25944 | 348 |
|
349 |
(** evaluation **) |
|
350 |
||
351 |
(* term evaluation *) |
|
352 |
||
30947 | 353 |
fun eval_term ctxt gr deps (vs : (string * sort) list, t) = |
25924 | 354 |
let |
28054 | 355 |
val frees = Code_Thingol.fold_unbound_varnames (insert (op =)) t [] |
25924 | 356 |
val frees' = map (fn v => Free (v, [])) frees; |
357 |
val dict_frees = maps (fn (v, sort) => map_index (curry DFree v o fst) sort) vs; |
|
358 |
in |
|
25935 | 359 |
("", (vs, [(map IVar frees, t)])) |
28274
9873697fa411
ML_Context.evaluate: proper context (for ML environment);
wenzelm
parents:
28227
diff
changeset
|
360 |
|> singleton (compile_eqnss ctxt gr deps) |
25924 | 361 |
|> snd |
362 |
|> (fn t => apps t (rev (dict_frees @ frees'))) |
|
363 |
end; |
|
24155 | 364 |
|
24839 | 365 |
(* reification *) |
24155 | 366 |
|
30947 | 367 |
fun typ_of_itype program vs (ityco `%% itys) = |
368 |
let |
|
369 |
val Code_Thingol.Datatype (tyco, _) = Graph.get_node program ityco; |
|
370 |
in Type (tyco, map (typ_of_itype program vs) itys) end |
|
371 |
| typ_of_itype program vs (ITyVar v) = |
|
372 |
let |
|
373 |
val sort = (the o AList.lookup (op =) vs) v; |
|
374 |
in TFree ("'" ^ v, sort) end; |
|
375 |
||
28663
bd8438543bf2
code identifier namings are no longer imperative
haftmann
parents:
28423
diff
changeset
|
376 |
fun term_of_univ thy program idx_tab t = |
24155 | 377 |
let |
25101 | 378 |
fun take_until f [] = [] |
379 |
| take_until f (x::xs) = if f x then [] else x :: take_until f xs; |
|
28663
bd8438543bf2
code identifier namings are no longer imperative
haftmann
parents:
28423
diff
changeset
|
380 |
fun is_dict (Const (idx, _)) = (case (Graph.get_node program o the o Inttab.lookup idx_tab) idx |
bd8438543bf2
code identifier namings are no longer imperative
haftmann
parents:
28423
diff
changeset
|
381 |
of Code_Thingol.Class _ => true |
bd8438543bf2
code identifier namings are no longer imperative
haftmann
parents:
28423
diff
changeset
|
382 |
| Code_Thingol.Classrel _ => true |
bd8438543bf2
code identifier namings are no longer imperative
haftmann
parents:
28423
diff
changeset
|
383 |
| Code_Thingol.Classinst _ => true |
bd8438543bf2
code identifier namings are no longer imperative
haftmann
parents:
28423
diff
changeset
|
384 |
| _ => false) |
25101 | 385 |
| is_dict (DFree _) = true |
386 |
| is_dict _ = false; |
|
28663
bd8438543bf2
code identifier namings are no longer imperative
haftmann
parents:
28423
diff
changeset
|
387 |
fun const_of_idx idx = (case (Graph.get_node program o the o Inttab.lookup idx_tab) idx |
bd8438543bf2
code identifier namings are no longer imperative
haftmann
parents:
28423
diff
changeset
|
388 |
of Code_Thingol.Fun (c, _) => c |
bd8438543bf2
code identifier namings are no longer imperative
haftmann
parents:
28423
diff
changeset
|
389 |
| Code_Thingol.Datatypecons (c, _) => c |
bd8438543bf2
code identifier namings are no longer imperative
haftmann
parents:
28423
diff
changeset
|
390 |
| Code_Thingol.Classparam (c, _) => c); |
24155 | 391 |
fun of_apps bounds (t, ts) = |
392 |
fold_map (of_univ bounds) ts |
|
393 |
#>> (fn ts' => list_comb (t, rev ts')) |
|
26064 | 394 |
and of_univ bounds (Const (idx, ts)) typidx = |
24155 | 395 |
let |
25101 | 396 |
val ts' = take_until is_dict ts; |
28663
bd8438543bf2
code identifier namings are no longer imperative
haftmann
parents:
28423
diff
changeset
|
397 |
val c = const_of_idx idx; |
28423 | 398 |
val (_, T) = Code.default_typscheme thy c; |
30022
1d8b8fa19074
maintain order of constructors in datatypes; clarified conventions for type schemes
haftmann
parents:
29272
diff
changeset
|
399 |
val T' = map_type_tfree (fn (v, _) => TypeInfer.param typidx (v, [])) T; |
1d8b8fa19074
maintain order of constructors in datatypes; clarified conventions for type schemes
haftmann
parents:
29272
diff
changeset
|
400 |
val typidx' = typidx + 1; |
25101 | 401 |
in of_apps bounds (Term.Const (c, T'), ts') typidx' end |
24155 | 402 |
| of_univ bounds (Free (name, ts)) typidx = |
403 |
of_apps bounds (Term.Free (name, dummyT), ts) typidx |
|
27499 | 404 |
| of_univ bounds (BVar (n, ts)) typidx = |
405 |
of_apps bounds (Bound (bounds - n - 1), ts) typidx |
|
24155 | 406 |
| of_univ bounds (t as Abs _) typidx = |
407 |
typidx |
|
25924 | 408 |
|> of_univ (bounds + 1) (apps t [BVar (bounds, [])]) |
24155 | 409 |
|-> (fn t' => pair (Term.Abs ("u", dummyT, t'))) |
410 |
in of_univ 0 t 0 |> fst end; |
|
411 |
||
25101 | 412 |
(* function store *) |
413 |
||
414 |
structure Nbe_Functions = CodeDataFun |
|
415 |
( |
|
28706 | 416 |
type T = Code_Thingol.naming * ((Univ option * int) Graph.T * (int * string Inttab.table)); |
417 |
val empty = (Code_Thingol.empty_naming, (Graph.empty, (0, Inttab.empty))); |
|
418 |
fun purge thy cs (naming, (gr, (maxidx, idx_tab))) = |
|
27609 | 419 |
let |
28706 | 420 |
val names_delete = cs |
421 |
|> map_filter (Code_Thingol.lookup_const naming) |
|
422 |
|> filter (can (Graph.get_node gr)) |
|
423 |
|> Graph.all_preds gr; |
|
424 |
val gr' = Graph.del_nodes names_delete gr; |
|
425 |
in (naming, (gr', (maxidx, idx_tab))) end; |
|
25101 | 426 |
); |
427 |
||
428 |
(* compilation, evaluation and reification *) |
|
429 |
||
30947 | 430 |
fun compile_eval thy naming program vs_t deps = |
26064 | 431 |
let |
28274
9873697fa411
ML_Context.evaluate: proper context (for ML environment);
wenzelm
parents:
28227
diff
changeset
|
432 |
val ctxt = ProofContext.init thy; |
28706 | 433 |
val (_, (gr, (_, idx_tab))) = |
434 |
Nbe_Functions.change thy (ensure_stmts ctxt naming program o snd); |
|
26064 | 435 |
in |
30947 | 436 |
vs_t |
28274
9873697fa411
ML_Context.evaluate: proper context (for ML environment);
wenzelm
parents:
28227
diff
changeset
|
437 |
|> eval_term ctxt gr deps |
28663
bd8438543bf2
code identifier namings are no longer imperative
haftmann
parents:
28423
diff
changeset
|
438 |
|> term_of_univ thy program idx_tab |
26064 | 439 |
end; |
25101 | 440 |
|
24155 | 441 |
(* evaluation with type reconstruction *) |
442 |
||
30970
3fe2e418a071
generic postprocessing scheme for term evaluations
haftmann
parents:
30947
diff
changeset
|
443 |
fun normalize thy naming program (((vs0, (vs, ty)), fs), t) deps = |
24155 | 444 |
let |
26747
f32fa5f5bdd1
moved 'trivial classes' to foundation of code generator
haftmann
parents:
26739
diff
changeset
|
445 |
fun subst_const f = map_aterms (fn t as Term.Const (c, ty) => Term.Const (f c, ty) |
f32fa5f5bdd1
moved 'trivial classes' to foundation of code generator
haftmann
parents:
26739
diff
changeset
|
446 |
| t => t); |
30947 | 447 |
val resubst_triv_consts = subst_const (Code_Unit.resubst_alias thy); |
448 |
val ty' = typ_of_itype program vs0 ty; |
|
449 |
val fs' = (map o apsnd) (typ_of_itype program vs0) fs; |
|
450 |
val type_frees = Term.map_aterms (fn (t as Term.Free (s, _)) => |
|
451 |
Term.Free (s, (the o AList.lookup (op =) fs') s) | t => t); |
|
27264 | 452 |
fun type_infer t = |
453 |
singleton (TypeInfer.infer_types (Syntax.pp_global thy) (Sign.tsig_of thy) I |
|
454 |
(try (Type.strip_sorts o Sign.the_const_type thy)) (K NONE) Name.context 0) |
|
30947 | 455 |
(TypeInfer.constrain ty' t); |
29272 | 456 |
fun check_tvars t = if null (Term.add_tvars t []) then t else |
24155 | 457 |
error ("Illegal schematic type variables in normalized term: " |
26952
df36f4c52ee8
command 'normal_form': proper context via Variable.auto_fixes;
wenzelm
parents:
26931
diff
changeset
|
458 |
^ setmp show_types true (Syntax.string_of_term_global thy) t); |
df36f4c52ee8
command 'normal_form': proper context via Variable.auto_fixes;
wenzelm
parents:
26931
diff
changeset
|
459 |
val string_of_term = setmp show_types true (Syntax.string_of_term_global thy); |
24155 | 460 |
in |
30947 | 461 |
compile_eval thy naming program (vs, t) deps |
25167 | 462 |
|> tracing (fn t => "Normalized:\n" ^ string_of_term t) |
30947 | 463 |
|> resubst_triv_consts |
26739 | 464 |
|> type_frees |
25167 | 465 |
|> tracing (fn t => "Vars typed:\n" ^ string_of_term t) |
26739 | 466 |
|> type_infer |
25167 | 467 |
|> tracing (fn t => "Types inferred:\n" ^ string_of_term t) |
26739 | 468 |
|> check_tvars |
25101 | 469 |
|> tracing (fn t => "---\n") |
24155 | 470 |
end; |
471 |
||
472 |
(* evaluation oracle *) |
|
473 |
||
30947 | 474 |
fun add_triv_classes thy = curry (Sorts.inter_sort (Sign.classes_of thy)) |
475 |
(Code_Unit.triv_classes thy); |
|
476 |
||
477 |
fun mk_equals thy lhs raw_rhs = |
|
26747
f32fa5f5bdd1
moved 'trivial classes' to foundation of code generator
haftmann
parents:
26739
diff
changeset
|
478 |
let |
30947 | 479 |
val ty = Thm.typ_of (Thm.ctyp_of_term lhs); |
480 |
val eq = Thm.cterm_of thy (Term.Const ("==", ty --> ty --> propT)); |
|
481 |
val rhs = Thm.cterm_of thy raw_rhs; |
|
482 |
in Thm.mk_binop eq lhs rhs end; |
|
26747
f32fa5f5bdd1
moved 'trivial classes' to foundation of code generator
haftmann
parents:
26739
diff
changeset
|
483 |
|
30942
1e246776f876
diagnostic commands now in code_thingol; tuned code of funny continuations
haftmann
parents:
30672
diff
changeset
|
484 |
val (_, raw_norm_oracle) = Context.>>> (Context.map_theory_result |
30947 | 485 |
(Thm.add_oracle (Binding.name "norm", fn (thy, naming, program, vsp_ty_fs_t, deps, ct) => |
30970
3fe2e418a071
generic postprocessing scheme for term evaluations
haftmann
parents:
30947
diff
changeset
|
486 |
mk_equals thy ct (normalize thy naming program vsp_ty_fs_t deps)))); |
30942
1e246776f876
diagnostic commands now in code_thingol; tuned code of funny continuations
haftmann
parents:
30672
diff
changeset
|
487 |
|
30947 | 488 |
fun norm_oracle thy naming program vsp_ty_fs_t deps ct = |
489 |
raw_norm_oracle (thy, naming, program, vsp_ty_fs_t, deps, ct); |
|
30942
1e246776f876
diagnostic commands now in code_thingol; tuned code of funny continuations
haftmann
parents:
30672
diff
changeset
|
490 |
|
24839 | 491 |
fun norm_conv ct = |
24155 | 492 |
let |
493 |
val thy = Thm.theory_of_cterm ct; |
|
30942
1e246776f876
diagnostic commands now in code_thingol; tuned code of funny continuations
haftmann
parents:
30672
diff
changeset
|
494 |
in Code_Thingol.eval_conv thy (add_triv_classes thy) (norm_oracle thy) ct end; |
24155 | 495 |
|
30970
3fe2e418a071
generic postprocessing scheme for term evaluations
haftmann
parents:
30947
diff
changeset
|
496 |
fun norm thy = Code_Thingol.eval thy (add_triv_classes thy) I (normalize thy); |
24839 | 497 |
|
24155 | 498 |
(* evaluation command *) |
499 |
||
500 |
fun norm_print_term ctxt modes t = |
|
501 |
let |
|
502 |
val thy = ProofContext.theory_of ctxt; |
|
30970
3fe2e418a071
generic postprocessing scheme for term evaluations
haftmann
parents:
30947
diff
changeset
|
503 |
val t' = norm thy t; |
24839 | 504 |
val ty' = Term.type_of t'; |
26952
df36f4c52ee8
command 'normal_form': proper context via Variable.auto_fixes;
wenzelm
parents:
26931
diff
changeset
|
505 |
val ctxt' = Variable.auto_fixes t ctxt; |
24634 | 506 |
val p = PrintMode.with_modes modes (fn () => |
26952
df36f4c52ee8
command 'normal_form': proper context via Variable.auto_fixes;
wenzelm
parents:
26931
diff
changeset
|
507 |
Pretty.block [Pretty.quote (Syntax.pretty_term ctxt' t'), Pretty.fbrk, |
df36f4c52ee8
command 'normal_form': proper context via Variable.auto_fixes;
wenzelm
parents:
26931
diff
changeset
|
508 |
Pretty.str "::", Pretty.brk 1, Pretty.quote (Syntax.pretty_typ ctxt' ty')]) (); |
24155 | 509 |
in Pretty.writeln p end; |
510 |
||
511 |
||
512 |
(** Isar setup **) |
|
513 |
||
24508
c8b82fec6447
replaced ProofContext.read_term/prop by general Syntax.read_term/prop;
wenzelm
parents:
24493
diff
changeset
|
514 |
fun norm_print_term_cmd (modes, s) state = |
24155 | 515 |
let val ctxt = Toplevel.context_of state |
24508
c8b82fec6447
replaced ProofContext.read_term/prop by general Syntax.read_term/prop;
wenzelm
parents:
24493
diff
changeset
|
516 |
in norm_print_term ctxt modes (Syntax.read_term ctxt s) end; |
24155 | 517 |
|
30970
3fe2e418a071
generic postprocessing scheme for term evaluations
haftmann
parents:
30947
diff
changeset
|
518 |
val setup = Value.add_evaluator ("nbe", norm o ProofContext.theory_of); |
24155 | 519 |
|
520 |
local structure P = OuterParse and K = OuterKeyword in |
|
521 |
||
522 |
val opt_modes = Scan.optional (P.$$$ "(" |-- P.!!! (Scan.repeat1 P.xname --| P.$$$ ")")) []; |
|
523 |
||
24867 | 524 |
val _ = |
24155 | 525 |
OuterSyntax.improper_command "normal_form" "normalize term by evaluation" K.diag |
28227 | 526 |
(opt_modes -- P.term >> (Toplevel.keep o norm_print_term_cmd)); |
24155 | 527 |
|
528 |
end; |
|
529 |
||
530 |
end; |
|
28337 | 531 |