author | blanchet |
Fri, 20 Jul 2012 22:19:46 +0200 | |
changeset 48406 | b002cc16aa99 |
parent 48404 | 0a261b4aa093 |
child 48407 | 47fe0ca12fc2 |
permissions | -rw-r--r-- |
48380 | 1 |
(* Title: HOL/Tools/Sledgehammer/sledgehammer_mash.ML |
48248 | 2 |
Author: Jasmin Blanchette, TU Muenchen |
3 |
||
4 |
Sledgehammer's machine-learning-based relevance filter (MaSh). |
|
5 |
*) |
|
6 |
||
48381 | 7 |
signature SLEDGEHAMMER_MASH = |
48248 | 8 |
sig |
48251
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
9 |
type stature = ATP_Problem_Generate.stature |
48296
e7f01b7e244e
gracefully handle the case of empty theories when going up the accessibility chain
blanchet
parents:
48293
diff
changeset
|
10 |
type fact = Sledgehammer_Fact.fact |
e7f01b7e244e
gracefully handle the case of empty theories when going up the accessibility chain
blanchet
parents:
48293
diff
changeset
|
11 |
type fact_override = Sledgehammer_Fact.fact_override |
48251
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
12 |
type params = Sledgehammer_Provers.params |
48288
255c6e1fd505
rationalize relevance filter, slowing moving code from Iter to MaSh
blanchet
parents:
48251
diff
changeset
|
13 |
type relevance_fudge = Sledgehammer_Provers.relevance_fudge |
48251
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
14 |
type prover_result = Sledgehammer_Provers.prover_result |
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
15 |
|
48308 | 16 |
val trace : bool Config.T |
48319
340187063d84
use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents:
48318
diff
changeset
|
17 |
val MaShN : string |
48379
2b5ad61e2ccc
renamed "iter" fact filter to "MePo" (Meng--Paulson)
blanchet
parents:
48378
diff
changeset
|
18 |
val mepoN : string |
2b5ad61e2ccc
renamed "iter" fact filter to "MePo" (Meng--Paulson)
blanchet
parents:
48378
diff
changeset
|
19 |
val mashN : string |
48314
ee33ba3c0e05
added option to control which fact filter is used
blanchet
parents:
48313
diff
changeset
|
20 |
val meshN : string |
48392
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
21 |
val unlearnN : string |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
22 |
val learn_isarN : string |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
23 |
val learn_atpN : string |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
24 |
val relearn_isarN : string |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
25 |
val relearn_atpN : string |
48314
ee33ba3c0e05
added option to control which fact filter is used
blanchet
parents:
48313
diff
changeset
|
26 |
val fact_filters : string list |
48303
f1d135d0ea69
improved MaSh string escaping and make more operations string-based
blanchet
parents:
48302
diff
changeset
|
27 |
val escape_meta : string -> string |
f1d135d0ea69
improved MaSh string escaping and make more operations string-based
blanchet
parents:
48302
diff
changeset
|
28 |
val escape_metas : string list -> string |
48308 | 29 |
val unescape_meta : string -> string |
30 |
val unescape_metas : string -> string list |
|
48406 | 31 |
val extract_query : string -> string * (string * real) list |
48378 | 32 |
val nickname_of : thm -> string |
48406 | 33 |
val suggested_facts : |
34 |
(string * 'a) list -> ('b * thm) list -> (('b * thm) * 'a) list |
|
48321 | 35 |
val mesh_facts : |
48406 | 36 |
int -> ((('a * thm) * real) list * ('a * thm) list) list -> ('a * thm) list |
48251
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
37 |
val theory_ord : theory * theory -> order |
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
38 |
val thm_ord : thm * thm -> order |
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
39 |
val goal_of_thm : theory -> thm -> thm |
48321 | 40 |
val run_prover_for_mash : |
48318 | 41 |
Proof.context -> params -> string -> fact list -> thm -> prover_result |
48392
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
42 |
val features_of : |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
43 |
Proof.context -> string -> theory -> stature -> term list -> string list |
48404 | 44 |
val isar_dependencies_of : unit Symtab.table -> thm -> string list option |
48392
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
45 |
val atp_dependencies_of : |
48404 | 46 |
Proof.context -> params -> string -> int -> fact list -> unit Symtab.table |
47 |
-> thm -> string list option |
|
48332
271a4a6af734
optimize parent computation in MaSh + remove temporary files
blanchet
parents:
48330
diff
changeset
|
48 |
val mash_CLEAR : Proof.context -> unit |
48308 | 49 |
val mash_ADD : |
48316
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents:
48315
diff
changeset
|
50 |
Proof.context -> bool |
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents:
48315
diff
changeset
|
51 |
-> (string * string list * string list * string list) list -> unit |
48404 | 52 |
val mash_REPROVE : |
53 |
Proof.context -> bool -> (string * string list) list -> unit |
|
48316
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents:
48315
diff
changeset
|
54 |
val mash_QUERY : |
48406 | 55 |
Proof.context -> bool -> int -> string list * string list |
56 |
-> (string * real) list |
|
48332
271a4a6af734
optimize parent computation in MaSh + remove temporary files
blanchet
parents:
48330
diff
changeset
|
57 |
val mash_unlearn : Proof.context -> unit |
48318 | 58 |
val mash_could_suggest_facts : unit -> bool |
48321 | 59 |
val mash_can_suggest_facts : Proof.context -> bool |
48406 | 60 |
val mash_suggested_facts : |
48321 | 61 |
Proof.context -> params -> string -> int -> term list -> term |
48406 | 62 |
-> ('a * thm) list -> (('a * thm) * real) list * ('a * thm) list |
48383 | 63 |
val mash_learn_proof : |
48384
83dc102041e6
learn on explicit "min" command but do the learning in a thread, since it may take a couple of seconds
blanchet
parents:
48383
diff
changeset
|
64 |
Proof.context -> params -> string -> term -> ('a * thm) list -> thm list |
83dc102041e6
learn on explicit "min" command but do the learning in a thread, since it may take a couple of seconds
blanchet
parents:
48383
diff
changeset
|
65 |
-> unit |
48395
85a7fb65507a
learning should honor the fact override and the chained facts
blanchet
parents:
48394
diff
changeset
|
66 |
val mash_learn : |
85a7fb65507a
learning should honor the fact override and the chained facts
blanchet
parents:
48394
diff
changeset
|
67 |
Proof.context -> params -> fact_override -> thm list -> bool -> unit |
48288
255c6e1fd505
rationalize relevance filter, slowing moving code from Iter to MaSh
blanchet
parents:
48251
diff
changeset
|
68 |
val relevant_facts : |
48292 | 69 |
Proof.context -> params -> string -> int -> fact_override -> term list |
48296
e7f01b7e244e
gracefully handle the case of empty theories when going up the accessibility chain
blanchet
parents:
48293
diff
changeset
|
70 |
-> term -> fact list -> fact list |
48319
340187063d84
use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents:
48318
diff
changeset
|
71 |
val kill_learners : unit -> unit |
340187063d84
use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents:
48318
diff
changeset
|
72 |
val running_learners : unit -> unit |
48248 | 73 |
end; |
74 |
||
48381 | 75 |
structure Sledgehammer_MaSh : SLEDGEHAMMER_MASH = |
48248 | 76 |
struct |
48249 | 77 |
|
48251
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
78 |
open ATP_Util |
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
79 |
open ATP_Problem_Generate |
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
80 |
open Sledgehammer_Util |
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
81 |
open Sledgehammer_Fact |
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
82 |
open Sledgehammer_Provers |
48318 | 83 |
open Sledgehammer_Minimize |
48381 | 84 |
open Sledgehammer_MePo |
48251
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
85 |
|
48308 | 86 |
val trace = |
48380 | 87 |
Attrib.setup_config_bool @{binding sledgehammer_mash_trace} (K false) |
48308 | 88 |
fun trace_msg ctxt msg = if Config.get ctxt trace then tracing (msg ()) else () |
89 |
||
48319
340187063d84
use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents:
48318
diff
changeset
|
90 |
val MaShN = "MaSh" |
340187063d84
use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents:
48318
diff
changeset
|
91 |
|
48379
2b5ad61e2ccc
renamed "iter" fact filter to "MePo" (Meng--Paulson)
blanchet
parents:
48378
diff
changeset
|
92 |
val mepoN = "mepo" |
48314
ee33ba3c0e05
added option to control which fact filter is used
blanchet
parents:
48313
diff
changeset
|
93 |
val mashN = "mash" |
48379
2b5ad61e2ccc
renamed "iter" fact filter to "MePo" (Meng--Paulson)
blanchet
parents:
48378
diff
changeset
|
94 |
val meshN = "mesh" |
48314
ee33ba3c0e05
added option to control which fact filter is used
blanchet
parents:
48313
diff
changeset
|
95 |
|
48379
2b5ad61e2ccc
renamed "iter" fact filter to "MePo" (Meng--Paulson)
blanchet
parents:
48378
diff
changeset
|
96 |
val fact_filters = [meshN, mepoN, mashN] |
48314
ee33ba3c0e05
added option to control which fact filter is used
blanchet
parents:
48313
diff
changeset
|
97 |
|
48392
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
98 |
val unlearnN = "unlearn" |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
99 |
val learn_isarN = "learn_isar" |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
100 |
val learn_atpN = "learn_atp" |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
101 |
val relearn_isarN = "relearn_isar" |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
102 |
val relearn_atpN = "relearn_atp" |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
103 |
|
48314
ee33ba3c0e05
added option to control which fact filter is used
blanchet
parents:
48313
diff
changeset
|
104 |
fun mash_home () = getenv "MASH_HOME" |
48394
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
105 |
fun mash_model_dir () = |
48309 | 106 |
getenv "ISABELLE_HOME_USER" ^ "/mash" |
48316
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents:
48315
diff
changeset
|
107 |
|> tap (Isabelle_System.mkdir o Path.explode) |
48394
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
108 |
val mash_state_dir = mash_model_dir |
48314
ee33ba3c0e05
added option to control which fact filter is used
blanchet
parents:
48313
diff
changeset
|
109 |
fun mash_state_path () = mash_state_dir () ^ "/state" |> Path.explode |
48251
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
110 |
|
48330 | 111 |
|
48251
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
112 |
(*** Isabelle helpers ***) |
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
113 |
|
48308 | 114 |
fun meta_char c = |
48251
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
115 |
if Char.isAlphaNum c orelse c = #"_" orelse c = #"." orelse c = #"(" orelse |
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
116 |
c = #")" orelse c = #"," then |
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
117 |
String.str c |
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
118 |
else |
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
119 |
(* fixed width, in case more digits follow *) |
48395
85a7fb65507a
learning should honor the fact override and the chained facts
blanchet
parents:
48394
diff
changeset
|
120 |
"%" ^ stringN_of_int 3 (Char.ord c) |
48251
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
121 |
|
48308 | 122 |
fun unmeta_chars accum [] = String.implode (rev accum) |
48395
85a7fb65507a
learning should honor the fact override and the chained facts
blanchet
parents:
48394
diff
changeset
|
123 |
| unmeta_chars accum (#"%" :: d1 :: d2 :: d3 :: cs) = |
48308 | 124 |
(case Int.fromString (String.implode [d1, d2, d3]) of |
125 |
SOME n => unmeta_chars (Char.chr n :: accum) cs |
|
126 |
| NONE => "" (* error *)) |
|
48395
85a7fb65507a
learning should honor the fact override and the chained facts
blanchet
parents:
48394
diff
changeset
|
127 |
| unmeta_chars _ (#"%" :: _) = "" (* error *) |
48308 | 128 |
| unmeta_chars accum (c :: cs) = unmeta_chars (c :: accum) cs |
129 |
||
130 |
val escape_meta = String.translate meta_char |
|
48303
f1d135d0ea69
improved MaSh string escaping and make more operations string-based
blanchet
parents:
48302
diff
changeset
|
131 |
val escape_metas = map escape_meta #> space_implode " " |
48315
82d6e46c673f
fixed order of accessibles + other tweaks to MaSh
blanchet
parents:
48314
diff
changeset
|
132 |
val unescape_meta = String.explode #> unmeta_chars [] |
82d6e46c673f
fixed order of accessibles + other tweaks to MaSh
blanchet
parents:
48314
diff
changeset
|
133 |
val unescape_metas = |
82d6e46c673f
fixed order of accessibles + other tweaks to MaSh
blanchet
parents:
48314
diff
changeset
|
134 |
space_explode " " #> filter_out (curry (op =) "") #> map unescape_meta |
48251
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
135 |
|
48406 | 136 |
fun extract_node line = |
137 |
case space_explode ":" line of |
|
138 |
[name, parents] => (unescape_meta name, unescape_metas parents) |
|
139 |
| _ => ("", []) |
|
140 |
||
141 |
fun extract_suggestion sugg = |
|
142 |
case space_explode "=" sugg of |
|
143 |
[name, weight] => |
|
144 |
SOME (unescape_meta name, Real.fromString weight |> the_default 0.0) |
|
145 |
| _ => NONE |
|
146 |
||
48311 | 147 |
fun extract_query line = |
148 |
case space_explode ":" line of |
|
48406 | 149 |
[goal, suggs] => |
150 |
(unescape_meta goal, |
|
151 |
map_filter extract_suggestion (space_explode " " suggs)) |
|
48312 | 152 |
| _ => ("", []) |
48311 | 153 |
|
48378 | 154 |
fun parent_of_local_thm th = |
155 |
let |
|
156 |
val thy = th |> Thm.theory_of_thm |
|
157 |
val facts = thy |> Global_Theory.facts_of |
|
158 |
val space = facts |> Facts.space_of |
|
159 |
fun id_of s = #id (Name_Space.the_entry space s) |
|
160 |
fun max_id (s', _) (s, id) = |
|
161 |
let val id' = id_of s' in if id > id' then (s, id) else (s', id') end |
|
162 |
in ("", ~1) |> Facts.fold_static max_id facts |> fst end |
|
163 |
||
164 |
val local_prefix = "local" ^ Long_Name.separator |
|
165 |
||
166 |
fun nickname_of th = |
|
48394
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
167 |
if Thm.has_name_hint th then |
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
168 |
let val hint = Thm.get_name_hint th in |
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
169 |
(* FIXME: There must be a better way to detect local facts. *) |
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
170 |
case try (unprefix local_prefix) hint of |
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
171 |
SOME suf => |
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
172 |
parent_of_local_thm th ^ Long_Name.separator ^ Long_Name.separator ^ suf |
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
173 |
| NONE => hint |
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
174 |
end |
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
175 |
else |
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
176 |
backquote_thm th |
48378 | 177 |
|
48330 | 178 |
fun suggested_facts suggs facts = |
179 |
let |
|
48378 | 180 |
fun add_fact (fact as (_, th)) = Symtab.default (nickname_of th, fact) |
48330 | 181 |
val tab = Symtab.empty |> fold add_fact facts |
48406 | 182 |
fun find_sugg (name, weight) = |
183 |
Symtab.lookup tab name |> Option.map (rpair weight) |
|
184 |
in map_filter find_sugg suggs end |
|
48311 | 185 |
|
48406 | 186 |
fun sum_avg [] = 0 |
187 |
| sum_avg xs = Real.ceil (100000.0 * fold (curry (op +)) xs 0.0) div length xs |
|
48328
ca0b7d19dd62
attempt at meshing according to more meaningful factors
blanchet
parents:
48327
diff
changeset
|
188 |
|
48406 | 189 |
fun normalize_scores [] = [] |
190 |
| normalize_scores ((fact, score) :: tail) = |
|
191 |
(fact, 1.0) :: map (apsnd (curry Real.* (1.0 / score))) tail |
|
48313
0faafdffa662
mesh facts by taking into consideration whether a fact is known to MeSh
blanchet
parents:
48312
diff
changeset
|
192 |
|
48406 | 193 |
fun mesh_facts max_facts [(sels, unks)] = |
194 |
map fst (take max_facts sels) @ take (max_facts - length sels) unks |
|
48314
ee33ba3c0e05
added option to control which fact filter is used
blanchet
parents:
48313
diff
changeset
|
195 |
| mesh_facts max_facts mess = |
ee33ba3c0e05
added option to control which fact filter is used
blanchet
parents:
48313
diff
changeset
|
196 |
let |
48406 | 197 |
val mess = mess |> map (apfst (normalize_scores #> `length)) |
48314
ee33ba3c0e05
added option to control which fact filter is used
blanchet
parents:
48313
diff
changeset
|
198 |
val fact_eq = Thm.eq_thm o pairself snd |
48406 | 199 |
fun score_at sels = try (nth sels) #> Option.map snd |
48320
891a24a48155
improved meshing of MaSh and Meng--Paulson if some MaSh suggestions are cut-off (the common case)
blanchet
parents:
48319
diff
changeset
|
200 |
fun score_in fact ((sel_len, sels), unks) = |
48406 | 201 |
case find_index (curry fact_eq fact o fst) sels of |
48320
891a24a48155
improved meshing of MaSh and Meng--Paulson if some MaSh suggestions are cut-off (the common case)
blanchet
parents:
48319
diff
changeset
|
202 |
~1 => (case find_index (curry fact_eq fact) unks of |
48406 | 203 |
~1 => score_at sels sel_len |
48320
891a24a48155
improved meshing of MaSh and Meng--Paulson if some MaSh suggestions are cut-off (the common case)
blanchet
parents:
48319
diff
changeset
|
204 |
| _ => NONE) |
48406 | 205 |
| rank => score_at sels rank |
206 |
fun weight_of fact = mess |> map_filter (score_in fact) |> sum_avg |
|
207 |
val facts = |
|
208 |
fold (union fact_eq o map fst o take max_facts o snd o fst) mess [] |
|
48314
ee33ba3c0e05
added option to control which fact filter is used
blanchet
parents:
48313
diff
changeset
|
209 |
in |
48406 | 210 |
facts |> map (`weight_of) |> sort (int_ord o swap o pairself fst) |
48328
ca0b7d19dd62
attempt at meshing according to more meaningful factors
blanchet
parents:
48327
diff
changeset
|
211 |
|> map snd |> take max_facts |
48314
ee33ba3c0e05
added option to control which fact filter is used
blanchet
parents:
48313
diff
changeset
|
212 |
end |
48312 | 213 |
|
48395
85a7fb65507a
learning should honor the fact override and the chained facts
blanchet
parents:
48394
diff
changeset
|
214 |
val thy_feature_name_of = prefix "y" |
85a7fb65507a
learning should honor the fact override and the chained facts
blanchet
parents:
48394
diff
changeset
|
215 |
val const_name_of = prefix "c" |
85a7fb65507a
learning should honor the fact override and the chained facts
blanchet
parents:
48394
diff
changeset
|
216 |
val type_name_of = prefix "t" |
85a7fb65507a
learning should honor the fact override and the chained facts
blanchet
parents:
48394
diff
changeset
|
217 |
val class_name_of = prefix "s" |
48251
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
218 |
|
48324 | 219 |
fun theory_ord p = |
220 |
if Theory.eq_thy p then |
|
221 |
EQUAL |
|
222 |
else if Theory.subthy p then |
|
223 |
LESS |
|
224 |
else if Theory.subthy (swap p) then |
|
225 |
GREATER |
|
226 |
else case int_ord (pairself (length o Theory.ancestors_of) p) of |
|
227 |
EQUAL => string_ord (pairself Context.theory_name p) |
|
228 |
| order => order |
|
229 |
||
230 |
val thm_ord = theory_ord o pairself theory_of_thm |
|
231 |
||
48392
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
232 |
val freezeT = Type.legacy_freeze_type |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
233 |
|
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
234 |
fun freeze (t $ u) = freeze t $ freeze u |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
235 |
| freeze (Abs (s, T, t)) = Abs (s, freezeT T, freeze t) |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
236 |
| freeze (Var ((s, _), T)) = Free (s, freezeT T) |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
237 |
| freeze (Const (s, T)) = Const (s, freezeT T) |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
238 |
| freeze (Free (s, T)) = Free (s, freezeT T) |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
239 |
| freeze t = t |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
240 |
|
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
241 |
fun goal_of_thm thy = prop_of #> freeze #> cterm_of thy #> Goal.init |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
242 |
|
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
243 |
fun run_prover_for_mash ctxt params prover facts goal = |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
244 |
let |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
245 |
val problem = |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
246 |
{state = Proof.init ctxt, goal = goal, subgoal = 1, subgoal_count = 1, |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
247 |
facts = facts |> map (apfst (apfst (fn name => name ()))) |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
248 |
|> map Untranslated_Fact} |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
249 |
in |
48399
4bacc8983b3d
learn from SMT proofs when they can be minimized by Metis
blanchet
parents:
48398
diff
changeset
|
250 |
get_minimizing_prover ctxt MaSh (K (K ())) prover params (K (K (K ""))) |
48392
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
251 |
problem |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
252 |
end |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
253 |
|
48326 | 254 |
val bad_types = [@{type_name prop}, @{type_name bool}, @{type_name fun}] |
255 |
||
48398 | 256 |
val logical_consts = |
257 |
[@{const_name prop}, @{const_name Pure.conjunction}] @ atp_logical_consts |
|
258 |
||
48318 | 259 |
fun interesting_terms_types_and_classes ctxt prover term_max_depth |
260 |
type_max_depth ts = |
|
48251
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
261 |
let |
48318 | 262 |
fun is_bad_const (x as (s, _)) args = |
48398 | 263 |
member (op =) logical_consts s orelse |
48318 | 264 |
fst (is_built_in_const_for_prover ctxt prover x args) |
48304 | 265 |
fun add_classes @{sort type} = I |
266 |
| add_classes S = union (op =) (map class_name_of S) |
|
48251
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
267 |
fun do_add_type (Type (s, Ts)) = |
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
268 |
(not (member (op =) bad_types s) ? insert (op =) (type_name_of s)) |
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
269 |
#> fold do_add_type Ts |
48304 | 270 |
| do_add_type (TFree (_, S)) = add_classes S |
271 |
| do_add_type (TVar (_, S)) = add_classes S |
|
48251
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
272 |
fun add_type T = type_max_depth >= 0 ? do_add_type T |
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
273 |
fun mk_app s args = |
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
274 |
if member (op <>) args "" then s ^ "(" ^ space_implode "," args ^ ")" |
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
275 |
else s |
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
276 |
fun patternify ~1 _ = "" |
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
277 |
| patternify depth t = |
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
278 |
case strip_comb t of |
48398 | 279 |
(Const (x as (s, _)), args) => |
280 |
if is_bad_const x args then "" |
|
281 |
else mk_app (const_name_of s) (map (patternify (depth - 1)) args) |
|
48251
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
282 |
| _ => "" |
48406 | 283 |
fun add_pattern depth t = |
284 |
case patternify depth t of "" => I | s => insert (op =) s |
|
48251
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
285 |
fun add_term_patterns ~1 _ = I |
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
286 |
| add_term_patterns depth t = |
48406 | 287 |
add_pattern depth t #> add_term_patterns (depth - 1) t |
48251
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
288 |
val add_term = add_term_patterns term_max_depth |
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
289 |
fun add_patterns t = |
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
290 |
let val (head, args) = strip_comb t in |
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
291 |
(case head of |
48398 | 292 |
Const (_, T) => add_term t #> add_type T |
48251
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
293 |
| Free (_, T) => add_type T |
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
294 |
| Var (_, T) => add_type T |
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
295 |
| Abs (_, T, body) => add_type T #> add_patterns body |
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
296 |
| _ => I) |
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
297 |
#> fold add_patterns args |
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
298 |
end |
48326 | 299 |
in [] |> fold add_patterns ts end |
48251
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
300 |
|
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
301 |
fun is_exists (s, _) = (s = @{const_name Ex} orelse s = @{const_name Ex1}) |
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
302 |
|
48297 | 303 |
val term_max_depth = 1 |
304 |
val type_max_depth = 1 |
|
48251
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
305 |
|
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
306 |
(* TODO: Generate type classes for types? *) |
48385 | 307 |
fun features_of ctxt prover thy (scope, status) ts = |
48303
f1d135d0ea69
improved MaSh string escaping and make more operations string-based
blanchet
parents:
48302
diff
changeset
|
308 |
thy_feature_name_of (Context.theory_name thy) :: |
48318 | 309 |
interesting_terms_types_and_classes ctxt prover term_max_depth type_max_depth |
310 |
ts |
|
48332
271a4a6af734
optimize parent computation in MaSh + remove temporary files
blanchet
parents:
48330
diff
changeset
|
311 |
|> forall is_lambda_free ts ? cons "no_lams" |
271a4a6af734
optimize parent computation in MaSh + remove temporary files
blanchet
parents:
48330
diff
changeset
|
312 |
|> forall (not o exists_Const is_exists) ts ? cons "no_skos" |
48385 | 313 |
|> scope <> Global ? cons "local" |
48302 | 314 |
|> (case status of |
315 |
General => I |
|
316 |
| Induction => cons "induction" |
|
317 |
| Intro => cons "intro" |
|
318 |
| Inductive => cons "inductive" |
|
319 |
| Elim => cons "elim" |
|
320 |
| Simp => cons "simp" |
|
321 |
| Def => cons "def") |
|
48251
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
322 |
|
48404 | 323 |
(* Too many dependencies is a sign that a decision procedure is at work. There |
324 |
isn't much too learn from such proofs. *) |
|
325 |
val max_dependencies = 10 |
|
326 |
val atp_dependency_default_max_fact = 50 |
|
48251
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
327 |
|
48404 | 328 |
fun trim_dependencies deps = |
329 |
if length deps <= max_dependencies then SOME deps else NONE |
|
48251
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
330 |
|
48406 | 331 |
fun isar_dependencies_of all_names = |
332 |
thms_in_proof (SOME all_names) #> trim_dependencies |
|
48404 | 333 |
|
334 |
fun atp_dependencies_of ctxt (params as {verbose, max_facts, ...}) prover |
|
335 |
auto_level facts all_names th = |
|
48392
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
336 |
case isar_dependencies_of all_names th of |
48404 | 337 |
SOME [] => NONE |
48392
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
338 |
| isar_deps => |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
339 |
let |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
340 |
val thy = Proof_Context.theory_of ctxt |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
341 |
val goal = goal_of_thm thy th |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
342 |
val (_, hyp_ts, concl_t) = ATP_Util.strip_subgoal ctxt goal 1 |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
343 |
val facts = facts |> filter (fn (_, th') => thm_ord (th', th) = LESS) |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
344 |
fun fix_name ((_, stature), th) = ((fn () => nickname_of th, stature), th) |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
345 |
fun is_dep dep (_, th) = nickname_of th = dep |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
346 |
fun add_isar_dep facts dep accum = |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
347 |
if exists (is_dep dep) accum then |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
348 |
accum |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
349 |
else case find_first (is_dep dep) facts of |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
350 |
SOME ((name, status), th) => accum @ [((name, status), th)] |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
351 |
| NONE => accum (* shouldn't happen *) |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
352 |
val facts = |
48406 | 353 |
facts |> mepo_suggested_facts ctxt params prover |
48404 | 354 |
(max_facts |> the_default atp_dependency_default_max_fact) |
355 |
NONE hyp_ts concl_t |
|
356 |
|> fold (add_isar_dep facts) (these isar_deps) |
|
48392
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
357 |
|> map fix_name |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
358 |
in |
48404 | 359 |
if verbose andalso auto_level = 0 then |
48392
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
360 |
let val num_facts = length facts in |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
361 |
"MaSh: " ^ quote prover ^ " on " ^ quote (nickname_of th) ^ |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
362 |
" with " ^ string_of_int num_facts ^ " fact" ^ plural_s num_facts ^ |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
363 |
"." |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
364 |
|> Output.urgent_message |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
365 |
end |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
366 |
else |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
367 |
(); |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
368 |
case run_prover_for_mash ctxt params prover facts goal of |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
369 |
{outcome = NONE, used_facts, ...} => |
48404 | 370 |
(if verbose andalso auto_level = 0 then |
48392
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
371 |
let val num_facts = length used_facts in |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
372 |
"Found proof with " ^ string_of_int num_facts ^ " fact" ^ |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
373 |
plural_s num_facts ^ "." |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
374 |
|> Output.urgent_message |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
375 |
end |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
376 |
else |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
377 |
(); |
48404 | 378 |
used_facts |> map fst |> trim_dependencies) |
379 |
| _ => NONE |
|
48392
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
380 |
end |
48251
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
381 |
|
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
382 |
|
48302 | 383 |
(*** Low-level communication with MaSh ***) |
384 |
||
48394
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
385 |
(* more friendly than "try o File.rm" for those who keep the files open in their |
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
386 |
text editor *) |
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
387 |
fun wipe_out file = File.write file "" |
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
388 |
|
48323 | 389 |
fun write_file (xs, f) file = |
48318 | 390 |
let val path = Path.explode file in |
48394
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
391 |
wipe_out path; |
48323 | 392 |
xs |> chunk_list 500 |
393 |
|> List.app (File.append path o space_implode "" o map f) |
|
48318 | 394 |
end |
48316
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents:
48315
diff
changeset
|
395 |
|
48394
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
396 |
fun run_mash_tool ctxt overlord save max_suggs write_cmds read_suggs = |
48311 | 397 |
let |
48394
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
398 |
val (temp_dir, serial) = |
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
399 |
if overlord then (getenv "ISABELLE_HOME_USER", "") |
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
400 |
else (getenv "ISABELLE_TMP", serial_string ()) |
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
401 |
val log_file = if overlord then temp_dir ^ "/mash_log" else "/dev/null" |
48316
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents:
48315
diff
changeset
|
402 |
val err_file = temp_dir ^ "/mash_err" ^ serial |
48318 | 403 |
val sugg_file = temp_dir ^ "/mash_suggs" ^ serial |
48316
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents:
48315
diff
changeset
|
404 |
val cmd_file = temp_dir ^ "/mash_commands" ^ serial |
48394
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
405 |
val core = |
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
406 |
"--inputFile " ^ cmd_file ^ " --predictions " ^ sugg_file ^ |
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
407 |
" --numberOfPredictions " ^ string_of_int max_suggs ^ |
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
408 |
(if save then " --saveModel" else "") |
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
409 |
val command = |
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
410 |
mash_home () ^ "/mash --quiet --outputDir " ^ mash_model_dir () ^ |
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
411 |
" --log " ^ log_file ^ " " ^ core ^ " >& " ^ err_file |
48316
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents:
48315
diff
changeset
|
412 |
in |
48323 | 413 |
write_file ([], K "") sugg_file; |
48316
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents:
48315
diff
changeset
|
414 |
write_file write_cmds cmd_file; |
48394
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
415 |
trace_msg ctxt (fn () => "Running " ^ command); |
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
416 |
Isabelle_System.bash command; |
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
417 |
read_suggs (fn () => try File.read_lines (Path.explode sugg_file) |> these) |
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
418 |
|> tap (fn _ => trace_msg ctxt (fn () => |
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
419 |
case try File.read (Path.explode err_file) of |
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
420 |
NONE => "Done" |
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
421 |
| SOME "" => "Done" |
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
422 |
| SOME s => "Error: " ^ elide_string 1000 s)) |
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
423 |
|> not overlord |
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
424 |
? tap (fn _ => List.app (wipe_out o Path.explode) |
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
425 |
[err_file, sugg_file, cmd_file]) |
48316
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents:
48315
diff
changeset
|
426 |
end |
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents:
48315
diff
changeset
|
427 |
|
48404 | 428 |
fun str_of_add (name, parents, feats, deps) = |
48316
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents:
48315
diff
changeset
|
429 |
"! " ^ escape_meta name ^ ": " ^ escape_metas parents ^ "; " ^ |
48311 | 430 |
escape_metas feats ^ "; " ^ escape_metas deps ^ "\n" |
431 |
||
48404 | 432 |
fun str_of_reprove (name, deps) = |
433 |
"p " ^ escape_meta name ^ ": " ^ escape_metas deps ^ "\n" |
|
434 |
||
48316
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents:
48315
diff
changeset
|
435 |
fun str_of_query (parents, feats) = |
48406 | 436 |
"? " ^ escape_metas parents ^ "; " ^ escape_metas feats ^ "\n" |
48316
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents:
48315
diff
changeset
|
437 |
|
48332
271a4a6af734
optimize parent computation in MaSh + remove temporary files
blanchet
parents:
48330
diff
changeset
|
438 |
fun mash_CLEAR ctxt = |
48394
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
439 |
let val path = mash_model_dir () |> Path.explode in |
48332
271a4a6af734
optimize parent computation in MaSh + remove temporary files
blanchet
parents:
48330
diff
changeset
|
440 |
trace_msg ctxt (K "MaSh CLEAR"); |
48394
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
441 |
File.fold_dir (fn file => fn _ => |
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
442 |
try File.rm (Path.append path (Path.basic file))) |
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
443 |
path NONE; |
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
444 |
() |
48309 | 445 |
end |
48302 | 446 |
|
48316
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents:
48315
diff
changeset
|
447 |
fun mash_ADD _ _ [] = () |
48404 | 448 |
| mash_ADD ctxt overlord adds = |
48316
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents:
48315
diff
changeset
|
449 |
(trace_msg ctxt (fn () => "MaSh ADD " ^ |
48404 | 450 |
elide_string 1000 (space_implode " " (map #1 adds))); |
451 |
run_mash_tool ctxt overlord true 0 (adds, str_of_add) (K ())) |
|
452 |
||
453 |
fun mash_REPROVE _ _ [] = () |
|
454 |
| mash_REPROVE ctxt overlord reps = |
|
455 |
(trace_msg ctxt (fn () => "MaSh REPROVE " ^ |
|
456 |
elide_string 1000 (space_implode " " (map #1 reps))); |
|
457 |
run_mash_tool ctxt overlord true 0 (reps, str_of_reprove) (K ())) |
|
48302 | 458 |
|
48318 | 459 |
fun mash_QUERY ctxt overlord max_suggs (query as (_, feats)) = |
48314
ee33ba3c0e05
added option to control which fact filter is used
blanchet
parents:
48313
diff
changeset
|
460 |
(trace_msg ctxt (fn () => "MaSh QUERY " ^ space_implode " " feats); |
48394
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
461 |
run_mash_tool ctxt overlord false max_suggs |
48323 | 462 |
([query], str_of_query) |
48394
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
463 |
(fn suggs => |
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
464 |
case suggs () of |
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
465 |
[] => [] |
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
466 |
| suggs => snd (extract_query (List.last suggs))) |
48311 | 467 |
handle List.Empty => []) |
48302 | 468 |
|
469 |
||
48251
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
470 |
(*** High-level communication with MaSh ***) |
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48249
diff
changeset
|
471 |
|
48321 | 472 |
fun try_graph ctxt when def f = |
473 |
f () |
|
474 |
handle Graph.CYCLES (cycle :: _) => |
|
475 |
(trace_msg ctxt (fn () => |
|
476 |
"Cycle involving " ^ commas cycle ^ " when " ^ when); def) |
|
48392
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
477 |
| Graph.DUP name => |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
478 |
(trace_msg ctxt (fn () => |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
479 |
"Duplicate fact " ^ quote name ^ " when " ^ when); def) |
48321 | 480 |
| Graph.UNDEF name => |
481 |
(trace_msg ctxt (fn () => |
|
482 |
"Unknown fact " ^ quote name ^ " when " ^ when); def) |
|
48392
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
483 |
| exn => |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
484 |
if Exn.is_interrupt exn then |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
485 |
reraise exn |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
486 |
else |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
487 |
(trace_msg ctxt (fn () => |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
488 |
"Internal error when " ^ when ^ ":\n" ^ |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
489 |
ML_Compiler.exn_message exn); def) |
48321 | 490 |
|
48406 | 491 |
fun graph_info G = |
492 |
string_of_int (length (Graph.keys G)) ^ " node(s), " ^ |
|
493 |
string_of_int (fold (Integer.add o length o snd) (Graph.dest G) 0) ^ |
|
494 |
" edge(s), " ^ |
|
495 |
string_of_int (length (Graph.minimals G)) ^ " minimal, " ^ |
|
496 |
string_of_int (length (Graph.maximals G)) ^ " maximal" |
|
497 |
||
48400 | 498 |
type mash_state = {fact_G : unit Graph.T} |
48301 | 499 |
|
48400 | 500 |
val empty_state = {fact_G = Graph.empty} |
48301 | 501 |
|
502 |
local |
|
503 |
||
48390
4147f2bc4442
add versioning to MaSh state + cleanup dead code
blanchet
parents:
48389
diff
changeset
|
504 |
val version = "*** MaSh 0.0 ***" |
4147f2bc4442
add versioning to MaSh state + cleanup dead code
blanchet
parents:
48389
diff
changeset
|
505 |
|
4147f2bc4442
add versioning to MaSh state + cleanup dead code
blanchet
parents:
48389
diff
changeset
|
506 |
fun load _ (state as (true, _)) = state |
4147f2bc4442
add versioning to MaSh state + cleanup dead code
blanchet
parents:
48389
diff
changeset
|
507 |
| load ctxt _ = |
48309 | 508 |
let val path = mash_state_path () in |
48302 | 509 |
(true, |
510 |
case try File.read_lines path of |
|
48406 | 511 |
SOME (version' :: node_lines) => |
48302 | 512 |
let |
48322
8a8d71e34297
fixed MaSh state load code so it works even if the facts are read in disorder
blanchet
parents:
48321
diff
changeset
|
513 |
fun add_edge_to name parent = |
48406 | 514 |
Graph.default_node (parent, ()) #> Graph.add_edge (parent, name) |
515 |
fun add_node line = |
|
516 |
case extract_node line of |
|
48316
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents:
48315
diff
changeset
|
517 |
("", _) => I (* shouldn't happen *) |
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents:
48315
diff
changeset
|
518 |
| (name, parents) => |
48406 | 519 |
Graph.default_node (name, ()) #> fold (add_edge_to name) parents |
48400 | 520 |
val fact_G = |
48322
8a8d71e34297
fixed MaSh state load code so it works even if the facts are read in disorder
blanchet
parents:
48321
diff
changeset
|
521 |
try_graph ctxt "loading state" Graph.empty (fn () => |
48406 | 522 |
Graph.empty |> version' = version ? fold add_node node_lines) |
523 |
in |
|
524 |
trace_msg ctxt (fn () => |
|
525 |
"Loaded fact graph (" ^ graph_info fact_G ^ ")"); |
|
526 |
{fact_G = fact_G} |
|
527 |
end |
|
48304 | 528 |
| _ => empty_state) |
48302 | 529 |
end |
48249 | 530 |
|
48406 | 531 |
fun save ctxt {fact_G} = |
48301 | 532 |
let |
48309 | 533 |
val path = mash_state_path () |
48318 | 534 |
fun fact_line_for name parents = |
535 |
escape_meta name ^ ": " ^ escape_metas parents |
|
48316
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents:
48315
diff
changeset
|
536 |
val append_fact = File.append path o suffix "\n" oo fact_line_for |
48400 | 537 |
fun append_entry (name, ((), (parents, _))) () = |
538 |
append_fact name (Graph.Keys.dest parents) |
|
48301 | 539 |
in |
48390
4147f2bc4442
add versioning to MaSh state + cleanup dead code
blanchet
parents:
48389
diff
changeset
|
540 |
File.write path (version ^ "\n"); |
48406 | 541 |
Graph.fold append_entry fact_G (); |
542 |
trace_msg ctxt (fn () => "Saved fact graph (" ^ graph_info fact_G ^ ")") |
|
48301 | 543 |
end |
544 |
||
48302 | 545 |
val global_state = |
48381 | 546 |
Synchronized.var "Sledgehammer_MaSh.global_state" (false, empty_state) |
48301 | 547 |
|
548 |
in |
|
549 |
||
48321 | 550 |
fun mash_map ctxt f = |
48406 | 551 |
Synchronized.change global_state (load ctxt ##> (f #> tap (save ctxt))) |
48302 | 552 |
|
48321 | 553 |
fun mash_get ctxt = |
48390
4147f2bc4442
add versioning to MaSh state + cleanup dead code
blanchet
parents:
48389
diff
changeset
|
554 |
Synchronized.change_result global_state (load ctxt #> `snd) |
48302 | 555 |
|
48332
271a4a6af734
optimize parent computation in MaSh + remove temporary files
blanchet
parents:
48330
diff
changeset
|
556 |
fun mash_unlearn ctxt = |
48302 | 557 |
Synchronized.change global_state (fn _ => |
48394
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
558 |
(mash_CLEAR ctxt; wipe_out (mash_state_path ()); (true, empty_state))) |
48301 | 559 |
|
560 |
end |
|
561 |
||
48318 | 562 |
fun mash_could_suggest_facts () = mash_home () <> "" |
48400 | 563 |
fun mash_can_suggest_facts ctxt = not (Graph.is_empty (#fact_G (mash_get ctxt))) |
48249 | 564 |
|
48400 | 565 |
fun queue_of xs = Queue.empty |> fold Queue.enqueue xs |
566 |
||
567 |
fun max_facts_in_graph fact_G facts = |
|
48316
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents:
48315
diff
changeset
|
568 |
let |
48378 | 569 |
val facts = [] |> fold (cons o nickname_of o snd) facts |
48330 | 570 |
val tab = Symtab.empty |> fold (fn name => Symtab.update (name, ())) facts |
48400 | 571 |
fun enqueue_new seen name = |
572 |
not (member (op =) seen name) ? Queue.enqueue name |
|
573 |
fun find_maxes seen maxs names = |
|
48401 | 574 |
case try Queue.dequeue names of |
575 |
NONE => map snd maxs |
|
576 |
| SOME (name, names) => |
|
577 |
if Symtab.defined tab name then |
|
578 |
let |
|
579 |
val new = (Graph.all_preds fact_G [name], name) |
|
48406 | 580 |
fun is_ancestor (_, x) (yp, _) = member (op =) yp x |
581 |
val maxs = maxs |> filter (fn max => not (is_ancestor max new)) |
|
582 |
val maxs = |
|
583 |
if exists (is_ancestor new) maxs then maxs |
|
584 |
else new :: filter_out (fn max => is_ancestor max new) maxs |
|
48401 | 585 |
in find_maxes (name :: seen) maxs names end |
586 |
else |
|
587 |
find_maxes (name :: seen) maxs |
|
588 |
(Graph.Keys.fold (enqueue_new seen) |
|
589 |
(Graph.imm_preds fact_G name) names) |
|
48400 | 590 |
in find_maxes [] [] (queue_of (Graph.maximals fact_G)) end |
48316
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents:
48315
diff
changeset
|
591 |
|
48318 | 592 |
(* Generate more suggestions than requested, because some might be thrown out |
593 |
later for various reasons and "meshing" gives better results with some |
|
594 |
slack. *) |
|
595 |
fun max_suggs_of max_facts = max_facts + Int.min (200, max_facts) |
|
596 |
||
48400 | 597 |
fun is_fact_in_graph fact_G (_, th) = |
598 |
can (Graph.get_node fact_G) (nickname_of th) |
|
48320
891a24a48155
improved meshing of MaSh and Meng--Paulson if some MaSh suggestions are cut-off (the common case)
blanchet
parents:
48319
diff
changeset
|
599 |
|
48406 | 600 |
fun mash_suggested_facts ctxt ({overlord, ...} : params) prover max_facts hyp_ts |
601 |
concl_t facts = |
|
48301 | 602 |
let |
48302 | 603 |
val thy = Proof_Context.theory_of ctxt |
48400 | 604 |
val fact_G = #fact_G (mash_get ctxt) |
605 |
val parents = max_facts_in_graph fact_G facts |
|
48385 | 606 |
val feats = features_of ctxt prover thy (Local, General) (concl_t :: hyp_ts) |
48318 | 607 |
val suggs = |
48400 | 608 |
if Graph.is_empty fact_G then [] |
48320
891a24a48155
improved meshing of MaSh and Meng--Paulson if some MaSh suggestions are cut-off (the common case)
blanchet
parents:
48319
diff
changeset
|
609 |
else mash_QUERY ctxt overlord (max_suggs_of max_facts) (parents, feats) |
891a24a48155
improved meshing of MaSh and Meng--Paulson if some MaSh suggestions are cut-off (the common case)
blanchet
parents:
48319
diff
changeset
|
610 |
val selected = facts |> suggested_facts suggs |
48400 | 611 |
val unknown = facts |> filter_out (is_fact_in_graph fact_G) |
48320
891a24a48155
improved meshing of MaSh and Meng--Paulson if some MaSh suggestions are cut-off (the common case)
blanchet
parents:
48319
diff
changeset
|
612 |
in (selected, unknown) end |
48249 | 613 |
|
48404 | 614 |
fun add_to_fact_graph ctxt (name, parents, feats, deps) (adds, graph) = |
48316
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents:
48315
diff
changeset
|
615 |
let |
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents:
48315
diff
changeset
|
616 |
fun maybe_add_from from (accum as (parents, graph)) = |
48321 | 617 |
try_graph ctxt "updating graph" accum (fn () => |
618 |
(from :: parents, Graph.add_edge_acyclic (from, name) graph)) |
|
619 |
val graph = graph |> Graph.default_node (name, ()) |
|
48316
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents:
48315
diff
changeset
|
620 |
val (parents, graph) = ([], graph) |> fold maybe_add_from parents |
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents:
48315
diff
changeset
|
621 |
val (deps, graph) = ([], graph) |> fold maybe_add_from deps |
48404 | 622 |
in ((name, parents, feats, deps) :: adds, graph) end |
48306 | 623 |
|
48384
83dc102041e6
learn on explicit "min" command but do the learning in a thread, since it may take a couple of seconds
blanchet
parents:
48383
diff
changeset
|
624 |
val learn_timeout_slack = 2.0 |
48318 | 625 |
|
48384
83dc102041e6
learn on explicit "min" command but do the learning in a thread, since it may take a couple of seconds
blanchet
parents:
48383
diff
changeset
|
626 |
fun launch_thread timeout task = |
48383 | 627 |
let |
48384
83dc102041e6
learn on explicit "min" command but do the learning in a thread, since it may take a couple of seconds
blanchet
parents:
48383
diff
changeset
|
628 |
val hard_timeout = time_mult learn_timeout_slack timeout |
83dc102041e6
learn on explicit "min" command but do the learning in a thread, since it may take a couple of seconds
blanchet
parents:
48383
diff
changeset
|
629 |
val birth_time = Time.now () |
83dc102041e6
learn on explicit "min" command but do the learning in a thread, since it may take a couple of seconds
blanchet
parents:
48383
diff
changeset
|
630 |
val death_time = Time.+ (birth_time, hard_timeout) |
83dc102041e6
learn on explicit "min" command but do the learning in a thread, since it may take a couple of seconds
blanchet
parents:
48383
diff
changeset
|
631 |
val desc = ("machine learner for Sledgehammer", "") |
83dc102041e6
learn on explicit "min" command but do the learning in a thread, since it may take a couple of seconds
blanchet
parents:
48383
diff
changeset
|
632 |
in Async_Manager.launch MaShN birth_time death_time desc task end |
83dc102041e6
learn on explicit "min" command but do the learning in a thread, since it may take a couple of seconds
blanchet
parents:
48383
diff
changeset
|
633 |
|
48400 | 634 |
fun freshish_name () = |
635 |
Date.fmt ".%Y_%m_%d_%H_%M_%S__" (Date.fromTimeLocal (Time.now ())) ^ |
|
636 |
serial_string () |
|
637 |
||
48384
83dc102041e6
learn on explicit "min" command but do the learning in a thread, since it may take a couple of seconds
blanchet
parents:
48383
diff
changeset
|
638 |
fun mash_learn_proof ctxt ({overlord, timeout, ...} : params) prover t facts |
83dc102041e6
learn on explicit "min" command but do the learning in a thread, since it may take a couple of seconds
blanchet
parents:
48383
diff
changeset
|
639 |
used_ths = |
83dc102041e6
learn on explicit "min" command but do the learning in a thread, since it may take a couple of seconds
blanchet
parents:
48383
diff
changeset
|
640 |
if is_smt_prover ctxt prover then |
83dc102041e6
learn on explicit "min" command but do the learning in a thread, since it may take a couple of seconds
blanchet
parents:
48383
diff
changeset
|
641 |
() |
83dc102041e6
learn on explicit "min" command but do the learning in a thread, since it may take a couple of seconds
blanchet
parents:
48383
diff
changeset
|
642 |
else |
48403
1f214c653c80
don't store fresh names in fact graph, since these cannot be the parents of any other facts
blanchet
parents:
48401
diff
changeset
|
643 |
launch_thread timeout (fn () => |
1f214c653c80
don't store fresh names in fact graph, since these cannot be the parents of any other facts
blanchet
parents:
48401
diff
changeset
|
644 |
let |
1f214c653c80
don't store fresh names in fact graph, since these cannot be the parents of any other facts
blanchet
parents:
48401
diff
changeset
|
645 |
val thy = Proof_Context.theory_of ctxt |
1f214c653c80
don't store fresh names in fact graph, since these cannot be the parents of any other facts
blanchet
parents:
48401
diff
changeset
|
646 |
val name = freshish_name () |
1f214c653c80
don't store fresh names in fact graph, since these cannot be the parents of any other facts
blanchet
parents:
48401
diff
changeset
|
647 |
val feats = features_of ctxt prover thy (Local, General) [t] |
1f214c653c80
don't store fresh names in fact graph, since these cannot be the parents of any other facts
blanchet
parents:
48401
diff
changeset
|
648 |
val deps = used_ths |> map nickname_of |
1f214c653c80
don't store fresh names in fact graph, since these cannot be the parents of any other facts
blanchet
parents:
48401
diff
changeset
|
649 |
val {fact_G} = mash_get ctxt |
1f214c653c80
don't store fresh names in fact graph, since these cannot be the parents of any other facts
blanchet
parents:
48401
diff
changeset
|
650 |
val parents = max_facts_in_graph fact_G facts |
1f214c653c80
don't store fresh names in fact graph, since these cannot be the parents of any other facts
blanchet
parents:
48401
diff
changeset
|
651 |
in |
1f214c653c80
don't store fresh names in fact graph, since these cannot be the parents of any other facts
blanchet
parents:
48401
diff
changeset
|
652 |
mash_ADD ctxt overlord [(name, parents, feats, deps)]; (true, "") |
1f214c653c80
don't store fresh names in fact graph, since these cannot be the parents of any other facts
blanchet
parents:
48401
diff
changeset
|
653 |
end) |
48383 | 654 |
|
48392
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
655 |
fun sendback sub = |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
656 |
Markup.markup Isabelle_Markup.sendback (sledgehammerN ^ " " ^ sub) |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
657 |
|
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
658 |
val commit_timeout = seconds 30.0 |
48332
271a4a6af734
optimize parent computation in MaSh + remove temporary files
blanchet
parents:
48330
diff
changeset
|
659 |
|
48318 | 660 |
(* The timeout is understood in a very slack fashion. *) |
48404 | 661 |
fun mash_learn_facts ctxt (params as {debug, verbose, overlord, ...}) prover |
662 |
auto_level atp learn_timeout facts = |
|
48304 | 663 |
let |
48318 | 664 |
val timer = Timer.startRealTimer () |
48392
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
665 |
fun next_commit_time () = |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
666 |
Time.+ (Timer.checkRealTimer timer, commit_timeout) |
48400 | 667 |
val {fact_G} = mash_get ctxt |
668 |
val (old_facts, new_facts) = |
|
669 |
facts |> List.partition (is_fact_in_graph fact_G) |
|
670 |
||> sort (thm_ord o pairself snd) |
|
48308 | 671 |
in |
48404 | 672 |
if null new_facts andalso (not atp orelse null old_facts) then |
673 |
if auto_level < 2 then |
|
674 |
"No new " ^ (if atp then "ATP" else "Isar") ^ " proofs to learn." ^ |
|
675 |
(if auto_level = 0 andalso not atp then |
|
676 |
"\n\nHint: Try " ^ sendback learn_atpN ^ " to learn from ATP proofs." |
|
677 |
else |
|
678 |
"") |
|
48392
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
679 |
else |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
680 |
"" |
48308 | 681 |
else |
48304 | 682 |
let |
48315
82d6e46c673f
fixed order of accessibles + other tweaks to MaSh
blanchet
parents:
48314
diff
changeset
|
683 |
val all_names = |
48400 | 684 |
facts |> map snd |
685 |
|> filter_out is_likely_tautology_or_too_meta |
|
686 |
|> map (rpair () o nickname_of) |
|
687 |
|> Symtab.make |
|
48404 | 688 |
val deps_of = |
689 |
if atp then |
|
690 |
atp_dependencies_of ctxt params prover auto_level facts all_names |
|
691 |
else |
|
692 |
isar_dependencies_of all_names |
|
693 |
fun do_commit [] [] state = state |
|
694 |
| do_commit adds reps {fact_G} = |
|
48392
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
695 |
let |
48404 | 696 |
val (adds, fact_G) = |
697 |
([], fact_G) |> fold (add_to_fact_graph ctxt) adds |
|
698 |
in |
|
699 |
mash_ADD ctxt overlord (rev adds); |
|
700 |
mash_REPROVE ctxt overlord reps; |
|
701 |
{fact_G = fact_G} |
|
702 |
end |
|
703 |
fun commit last adds reps = |
|
704 |
(if debug andalso auto_level = 0 then |
|
705 |
Output.urgent_message "Committing..." |
|
706 |
else |
|
707 |
(); |
|
708 |
mash_map ctxt (do_commit (rev adds) reps); |
|
709 |
if not last andalso auto_level = 0 then |
|
710 |
let val num_proofs = length adds + length reps in |
|
711 |
"Learned " ^ string_of_int num_proofs ^ " " ^ |
|
712 |
(if atp then "ATP" else "Isar") ^ " proof" ^ |
|
713 |
plural_s num_proofs ^ " in the last " ^ |
|
48392
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
714 |
string_from_time commit_timeout ^ "." |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
715 |
|> Output.urgent_message |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
716 |
end |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
717 |
else |
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
718 |
()) |
48404 | 719 |
fun learn_new_fact _ (accum as (_, (_, _, _, true))) = accum |
720 |
| learn_new_fact ((_, stature), th) |
|
721 |
(adds, (parents, n, next_commit, _)) = |
|
48318 | 722 |
let |
48378 | 723 |
val name = nickname_of th |
48332
271a4a6af734
optimize parent computation in MaSh + remove temporary files
blanchet
parents:
48330
diff
changeset
|
724 |
val feats = |
48385 | 725 |
features_of ctxt prover (theory_of_thm th) stature [prop_of th] |
48404 | 726 |
val deps = deps_of th |> these |
48394
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
blanchet
parents:
48392
diff
changeset
|
727 |
val n = n |> not (null deps) ? Integer.add 1 |
48404 | 728 |
val adds = (name, parents, feats, deps) :: adds |
729 |
val (adds, next_commit) = |
|
48392
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
730 |
if Time.> (Timer.checkRealTimer timer, next_commit) then |
48404 | 731 |
(commit false adds []; ([], next_commit_time ())) |
48392
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
732 |
else |
48404 | 733 |
(adds, next_commit) |
734 |
val timed_out = Time.> (Timer.checkRealTimer timer, learn_timeout) |
|
735 |
in (adds, ([name], n, next_commit, timed_out)) end |
|
736 |
val n = |
|
737 |
if null new_facts then |
|
738 |
0 |
|
739 |
else |
|
740 |
let |
|
741 |
val last_th = new_facts |> List.last |> snd |
|
742 |
(* crude approximation *) |
|
743 |
val ancestors = |
|
744 |
old_facts |
|
745 |
|> filter (fn (_, th) => thm_ord (th, last_th) <> GREATER) |
|
746 |
val parents = max_facts_in_graph fact_G ancestors |
|
747 |
val (adds, (_, n, _, _)) = |
|
748 |
([], (parents, 0, next_commit_time (), false)) |
|
749 |
|> fold learn_new_fact new_facts |
|
750 |
in commit true adds []; n end |
|
751 |
fun relearn_old_fact _ (accum as (_, (_, _, true))) = accum |
|
752 |
| relearn_old_fact (_, th) (reps, (n, next_commit, _)) = |
|
753 |
let |
|
754 |
val name = nickname_of th |
|
755 |
val (n, reps) = |
|
756 |
case deps_of th of |
|
757 |
SOME deps => (n + 1, (name, deps) :: reps) |
|
758 |
| NONE => (n, reps) |
|
759 |
val (reps, next_commit) = |
|
760 |
if Time.> (Timer.checkRealTimer timer, next_commit) then |
|
761 |
(commit false [] reps; ([], next_commit_time ())) |
|
762 |
else |
|
763 |
(reps, next_commit) |
|
764 |
val timed_out = Time.> (Timer.checkRealTimer timer, learn_timeout) |
|
765 |
in (reps, (n, next_commit, timed_out)) end |
|
766 |
val n = |
|
767 |
if null old_facts then |
|
768 |
n |
|
769 |
else |
|
770 |
let |
|
48406 | 771 |
fun priority_of (_, th) = |
48404 | 772 |
random_range 0 (1000 * max_dependencies) |
773 |
- 500 * (th |> isar_dependencies_of all_names |
|
774 |
|> Option.map length |
|
775 |
|> the_default max_dependencies) |
|
776 |
val old_facts = |
|
48406 | 777 |
old_facts |> map (`priority_of) |
48404 | 778 |
|> sort (int_ord o pairself fst) |
779 |
|> map snd |
|
780 |
val (reps, (n, _, _)) = |
|
781 |
([], (n, next_commit_time (), false)) |
|
782 |
|> fold relearn_old_fact old_facts |
|
783 |
in commit true [] reps; n end |
|
48318 | 784 |
in |
48404 | 785 |
if verbose orelse auto_level < 2 then |
786 |
"Learned " ^ string_of_int n ^ " nontrivial " ^ |
|
787 |
(if atp then "ATP" else "Isar") ^ " proof" ^ plural_s n ^ |
|
48319
340187063d84
use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents:
48318
diff
changeset
|
788 |
(if verbose then |
340187063d84
use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents:
48318
diff
changeset
|
789 |
" in " ^ string_from_time (Timer.checkRealTimer timer) |
340187063d84
use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents:
48318
diff
changeset
|
790 |
else |
340187063d84
use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents:
48318
diff
changeset
|
791 |
"") ^ "." |
340187063d84
use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents:
48318
diff
changeset
|
792 |
else |
340187063d84
use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents:
48318
diff
changeset
|
793 |
"" |
48318 | 794 |
end |
48308 | 795 |
end |
48304 | 796 |
|
48404 | 797 |
fun mash_learn ctxt (params as {provers, timeout, ...}) fact_override chained |
798 |
atp = |
|
48316
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents:
48315
diff
changeset
|
799 |
let |
48396 | 800 |
val css = Sledgehammer_Fact.clasimpset_rule_table_of ctxt |
48395
85a7fb65507a
learning should honor the fact override and the chained facts
blanchet
parents:
48394
diff
changeset
|
801 |
val ctxt = ctxt |> Config.put instantiate_inducts false |
85a7fb65507a
learning should honor the fact override and the chained facts
blanchet
parents:
48394
diff
changeset
|
802 |
val facts = |
48396 | 803 |
nearly_all_facts ctxt false fact_override Symtab.empty css chained [] |
804 |
@{prop True} |
|
48404 | 805 |
val num_facts = length facts |
806 |
val prover = hd provers |
|
807 |
fun learn auto_level atp = |
|
808 |
mash_learn_facts ctxt params prover auto_level atp infinite_timeout facts |
|
809 |
|> Output.urgent_message |
|
48316
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents:
48315
diff
changeset
|
810 |
in |
48404 | 811 |
(if atp then |
812 |
("MaShing through " ^ string_of_int num_facts ^ " fact" ^ |
|
813 |
plural_s num_facts ^ " for ATP proofs (" ^ quote prover ^ " timeout: " ^ |
|
814 |
string_from_time timeout ^ ").\n\nCollecting Isar proofs first..." |
|
815 |
|> Output.urgent_message; |
|
816 |
learn 1 false; |
|
817 |
"Now collecting ATP proofs. This may take several hours. You can \ |
|
818 |
\safely stop the learning process at any point." |
|
819 |
|> Output.urgent_message; |
|
820 |
learn 0 true) |
|
821 |
else |
|
822 |
("MaShing through " ^ string_of_int num_facts ^ " fact" ^ |
|
823 |
plural_s num_facts ^ " for Isar proofs..." |
|
824 |
|> Output.urgent_message; |
|
825 |
learn 0 false)) |
|
48316
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents:
48315
diff
changeset
|
826 |
end |
48249 | 827 |
|
48318 | 828 |
(* The threshold should be large enough so that MaSh doesn't kick in for Auto |
829 |
Sledgehammer and Try. *) |
|
830 |
val min_secs_for_learning = 15 |
|
831 |
||
48321 | 832 |
fun relevant_facts ctxt (params as {learn, fact_filter, timeout, ...}) prover |
833 |
max_facts ({add, only, ...} : fact_override) hyp_ts concl_t facts = |
|
48314
ee33ba3c0e05
added option to control which fact filter is used
blanchet
parents:
48313
diff
changeset
|
834 |
if not (subset (op =) (the_list fact_filter, fact_filters)) then |
ee33ba3c0e05
added option to control which fact filter is used
blanchet
parents:
48313
diff
changeset
|
835 |
error ("Unknown fact filter: " ^ quote (the fact_filter) ^ ".") |
ee33ba3c0e05
added option to control which fact filter is used
blanchet
parents:
48313
diff
changeset
|
836 |
else if only then |
48289 | 837 |
facts |
48321 | 838 |
else if max_facts <= 0 orelse null facts then |
48288
255c6e1fd505
rationalize relevance filter, slowing moving code from Iter to MaSh
blanchet
parents:
48251
diff
changeset
|
839 |
[] |
255c6e1fd505
rationalize relevance filter, slowing moving code from Iter to MaSh
blanchet
parents:
48251
diff
changeset
|
840 |
else |
255c6e1fd505
rationalize relevance filter, slowing moving code from Iter to MaSh
blanchet
parents:
48251
diff
changeset
|
841 |
let |
48327
568b3193e53e
don't include hidden facts in relevance filter + tweak MaSh learning
blanchet
parents:
48326
diff
changeset
|
842 |
fun maybe_learn () = |
48384
83dc102041e6
learn on explicit "min" command but do the learning in a thread, since it may take a couple of seconds
blanchet
parents:
48383
diff
changeset
|
843 |
if learn andalso not (Async_Manager.has_running_threads MaShN) andalso |
83dc102041e6
learn on explicit "min" command but do the learning in a thread, since it may take a couple of seconds
blanchet
parents:
48383
diff
changeset
|
844 |
Time.toSeconds timeout >= min_secs_for_learning then |
83dc102041e6
learn on explicit "min" command but do the learning in a thread, since it may take a couple of seconds
blanchet
parents:
48383
diff
changeset
|
845 |
let val timeout = time_mult learn_timeout_slack timeout in |
83dc102041e6
learn on explicit "min" command but do the learning in a thread, since it may take a couple of seconds
blanchet
parents:
48383
diff
changeset
|
846 |
launch_thread timeout |
48404 | 847 |
(fn () => (true, mash_learn_facts ctxt params prover 2 false |
48392
ca998fa08cd9
added "learn_from_atp" command to MaSh, for patient users
blanchet
parents:
48390
diff
changeset
|
848 |
timeout facts)) |
48319
340187063d84
use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents:
48318
diff
changeset
|
849 |
end |
48318 | 850 |
else |
851 |
() |
|
48314
ee33ba3c0e05
added option to control which fact filter is used
blanchet
parents:
48313
diff
changeset
|
852 |
val fact_filter = |
ee33ba3c0e05
added option to control which fact filter is used
blanchet
parents:
48313
diff
changeset
|
853 |
case fact_filter of |
48379
2b5ad61e2ccc
renamed "iter" fact filter to "MePo" (Meng--Paulson)
blanchet
parents:
48378
diff
changeset
|
854 |
SOME ff => (() |> ff <> mepoN ? maybe_learn; ff) |
48318 | 855 |
| NONE => |
48386
b903ea11b3bc
use good old MePo filter for SMT solvers by default, since arithmetic is built-in for them
blanchet
parents:
48385
diff
changeset
|
856 |
if is_smt_prover ctxt prover then mepoN |
b903ea11b3bc
use good old MePo filter for SMT solvers by default, since arithmetic is built-in for them
blanchet
parents:
48385
diff
changeset
|
857 |
else if mash_can_suggest_facts ctxt then (maybe_learn (); meshN) |
48379
2b5ad61e2ccc
renamed "iter" fact filter to "MePo" (Meng--Paulson)
blanchet
parents:
48378
diff
changeset
|
858 |
else if mash_could_suggest_facts () then (maybe_learn (); mepoN) |
2b5ad61e2ccc
renamed "iter" fact filter to "MePo" (Meng--Paulson)
blanchet
parents:
48378
diff
changeset
|
859 |
else mepoN |
48288
255c6e1fd505
rationalize relevance filter, slowing moving code from Iter to MaSh
blanchet
parents:
48251
diff
changeset
|
860 |
val add_ths = Attrib.eval_thms ctxt add |
48292 | 861 |
fun prepend_facts ths accepts = |
48288
255c6e1fd505
rationalize relevance filter, slowing moving code from Iter to MaSh
blanchet
parents:
48251
diff
changeset
|
862 |
((facts |> filter (member Thm.eq_thm_prop ths o snd)) @ |
48292 | 863 |
(accepts |> filter_out (member Thm.eq_thm_prop ths o snd))) |
48293 | 864 |
|> take max_facts |
48406 | 865 |
fun mepo () = |
866 |
facts |> mepo_suggested_facts ctxt params prover max_facts NONE hyp_ts |
|
867 |
concl_t |
|
868 |
|> weight_mepo_facts |
|
48314
ee33ba3c0e05
added option to control which fact filter is used
blanchet
parents:
48313
diff
changeset
|
869 |
fun mash () = |
48406 | 870 |
mash_suggested_facts ctxt params prover max_facts hyp_ts concl_t facts |
48314
ee33ba3c0e05
added option to control which fact filter is used
blanchet
parents:
48313
diff
changeset
|
871 |
val mess = |
48406 | 872 |
[] |> (if fact_filter <> mashN then cons (mepo (), []) else I) |
48379
2b5ad61e2ccc
renamed "iter" fact filter to "MePo" (Meng--Paulson)
blanchet
parents:
48378
diff
changeset
|
873 |
|> (if fact_filter <> mepoN then cons (mash ()) else I) |
48288
255c6e1fd505
rationalize relevance filter, slowing moving code from Iter to MaSh
blanchet
parents:
48251
diff
changeset
|
874 |
in |
48313
0faafdffa662
mesh facts by taking into consideration whether a fact is known to MeSh
blanchet
parents:
48312
diff
changeset
|
875 |
mesh_facts max_facts mess |
48288
255c6e1fd505
rationalize relevance filter, slowing moving code from Iter to MaSh
blanchet
parents:
48251
diff
changeset
|
876 |
|> not (null add_ths) ? prepend_facts add_ths |
255c6e1fd505
rationalize relevance filter, slowing moving code from Iter to MaSh
blanchet
parents:
48251
diff
changeset
|
877 |
end |
255c6e1fd505
rationalize relevance filter, slowing moving code from Iter to MaSh
blanchet
parents:
48251
diff
changeset
|
878 |
|
48319
340187063d84
use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents:
48318
diff
changeset
|
879 |
fun kill_learners () = Async_Manager.kill_threads MaShN "learner" |
340187063d84
use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents:
48318
diff
changeset
|
880 |
fun running_learners () = Async_Manager.running_threads MaShN "learner" |
340187063d84
use async manager to manage MaSh learners to make sure they get killed cleanly
blanchet
parents:
48318
diff
changeset
|
881 |
|
48248 | 882 |
end; |