| author | blanchet | 
| Fri, 05 Sep 2014 00:41:01 +0200 | |
| changeset 58187 | d2ddd401d74d | 
| parent 58061 | 3d060f43accb | 
| child 58205 | 369513534627 | 
| permissions | -rw-r--r-- | 
| 48285 | 1 | (* Title: HOL/TPTP/mash_eval.ML | 
| 48234 | 2 | Author: Jasmin Blanchette, TU Muenchen | 
| 3 | Copyright 2012 | |
| 4 | ||
| 48285 | 5 | Evaluate proof suggestions from MaSh (Machine-learning for Sledgehammer). | 
| 48234 | 6 | *) | 
| 7 | ||
| 48285 | 8 | signature MASH_EVAL = | 
| 48234 | 9 | sig | 
| 55201 | 10 | type params = Sledgehammer_Prover.params | 
| 48251 
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
 blanchet parents: 
48250diff
changeset | 11 | |
| 57456 | 12 | val evaluate_mash_suggestions : Proof.context -> params -> int * int option -> string option -> | 
| 13 | string list -> string -> unit | |
| 48234 | 14 | end; | 
| 15 | ||
| 48285 | 16 | structure MaSh_Eval : MASH_EVAL = | 
| 48234 | 17 | struct | 
| 48235 | 18 | |
| 50557 | 19 | open Sledgehammer_Util | 
| 48315 
82d6e46c673f
fixed order of accessibles + other tweaks to MaSh
 blanchet parents: 
48313diff
changeset | 20 | open Sledgehammer_Fact | 
| 50557 | 21 | open Sledgehammer_MePo | 
| 48381 | 22 | open Sledgehammer_MaSh | 
| 55201 | 23 | open Sledgehammer_Prover | 
| 55212 | 24 | open Sledgehammer_Prover_ATP | 
| 55198 | 25 | open Sledgehammer_Commands | 
| 57431 
02c408aed5ee
killed Python version of MaSh, now that the SML version works adequately
 blanchet parents: 
57406diff
changeset | 26 | open MaSh_Export | 
| 48240 | 27 | |
| 53980 
7e6a82c593f4
made SML/NJ happy (NB: toplevel ML environment is unmanaged);
 wenzelm parents: 
53139diff
changeset | 28 | val prefix = Library.prefix | 
| 
7e6a82c593f4
made SML/NJ happy (NB: toplevel ML environment is unmanaged);
 wenzelm parents: 
53139diff
changeset | 29 | |
| 57456 | 30 | fun evaluate_mash_suggestions ctxt params range prob_dir_name file_names report_file_name = | 
| 48235 | 31 | let | 
| 55205 | 32 | val thy = Proof_Context.theory_of ctxt | 
| 51028 | 33 | val zeros = [0, 0, 0, 0, 0, 0] | 
| 50448 
0a740d127187
have MaSh evaluator keep all raw problem/solution files in a directory
 blanchet parents: 
50442diff
changeset | 34 | val report_path = report_file_name |> Path.explode | 
| 
0a740d127187
have MaSh evaluator keep all raw problem/solution files in a directory
 blanchet parents: 
50442diff
changeset | 35 | val _ = File.write report_path "" | 
| 57432 | 36 | |
| 50589 | 37 | fun print s = File.append report_path (s ^ "\n") | 
| 57432 | 38 | |
| 55205 | 39 |     val {provers, max_facts, slice, type_enc, lam_trans, timeout, ...} = default_params thy []
 | 
| 48318 | 40 | val prover = hd provers | 
| 57108 
dc0b4f50e288
more generous max number of suggestions, for more safety
 blanchet parents: 
55212diff
changeset | 41 | val max_suggs = generous_max_suggestions (the max_facts) | 
| 57456 | 42 | |
| 43 | val method_of_file_name = | |
| 44 | perhaps (try (unsuffix "_suggestions")) o List.last o space_explode "/" | |
| 45 | ||
| 46 | val methods = "isar" :: map method_of_file_name file_names | |
| 50964 
2a990baa09af
use precomputed MaSh/MePo data whenever available
 blanchet parents: 
50953diff
changeset | 47 | val lines_of = Path.explode #> try File.read_lines #> these | 
| 57456 | 48 | val liness0 = map lines_of file_names | 
| 49 | val num_lines = fold (Integer.max o length) liness0 0 | |
| 57432 | 50 | |
| 50964 
2a990baa09af
use precomputed MaSh/MePo data whenever available
 blanchet parents: 
50953diff
changeset | 51 | fun pad lines = lines @ replicate (num_lines - length lines) "" | 
| 57432 | 52 | |
| 57456 | 53 | val liness = map pad liness0 | 
| 54 | ||
| 50557 | 55 | val css = clasimpset_rule_table_of ctxt | 
| 50442 
4f6a4d32522c
don't blacklist "case" theorems -- this causes problems in MaSh later
 blanchet parents: 
50440diff
changeset | 56 | val facts = all_facts ctxt true false Symtab.empty [] [] css | 
| 50735 
6b232d76cbc9
refined class handling, to prevent cycles in fact graph
 blanchet parents: 
50633diff
changeset | 57 | val name_tabs = build_name_tables nickname_of_thm facts | 
| 57432 | 58 | |
| 48289 | 59 | fun with_index facts s = (find_index (curry (op =) s) facts + 1, s) | 
| 50952 | 60 | fun index_str (j, s) = s ^ "@" ^ string_of_int j | 
| 50953 | 61 | val str_of_method = enclose " " ": " | 
| 57432 | 62 | |
| 63 |     fun str_of_result method facts ({outcome, run_time, used_facts, ...} : prover_result) =
 | |
| 51004 
5f2788c38127
distinguish raw and non-raw facts, using raw for 10 000s of facts and non-raw after selection of some hundreds
 blanchet parents: 
50967diff
changeset | 64 | let val facts = facts |> map (fst o fst) in | 
| 50953 | 65 | str_of_method method ^ | 
| 48289 | 66 | (if is_none outcome then | 
| 52031 
9a9238342963
tuning -- renamed '_from_' to '_of_' in Sledgehammer
 blanchet parents: 
51199diff
changeset | 67 |            "Success (" ^ ATP_Util.string_of_time run_time ^ "): " ^
 | 
| 48289 | 68 | (used_facts |> map (with_index facts o fst) | 
| 69 | |> sort (int_ord o pairself fst) | |
| 50952 | 70 | |> map index_str | 
| 48289 | 71 | |> space_implode " ") ^ | 
| 48293 | 72 | (if length facts < the max_facts then | 
| 48289 | 73 | " (of " ^ string_of_int (length facts) ^ ")" | 
| 74 | else | |
| 75 | "") | |
| 76 | else | |
| 77 | "Failure: " ^ | |
| 48293 | 78 | (facts |> take (the max_facts) |> tag_list 1 | 
| 50952 | 79 | |> map index_str | 
| 48289 | 80 | |> space_implode " ")) | 
| 81 | end | |
| 57432 | 82 | |
| 57456 | 83 | fun solve_goal (j, lines) = | 
| 50559 
89c0d2f13cca
MaSh exporter can now export subsets of the facts, as consecutive ranges
 blanchet parents: 
50557diff
changeset | 84 | if in_range range j then | 
| 
89c0d2f13cca
MaSh exporter can now export subsets of the facts, as consecutive ranges
 blanchet parents: 
50557diff
changeset | 85 | let | 
| 57125 
2f620ef839ee
added another way of invoking Python code, for experiments
 blanchet parents: 
57108diff
changeset | 86 | val get_suggs = extract_suggestions ##> (take max_suggs #> map fst) | 
| 57456 | 87 | val (names, suggss0) = split_list (map get_suggs lines) | 
| 88 | val [name] = names |> filter (curry (op <>) "") |> distinct (op =) | |
| 50964 
2a990baa09af
use precomputed MaSh/MePo data whenever available
 blanchet parents: 
50953diff
changeset | 89 | handle General.Match => error "Input files out of sync." | 
| 50559 
89c0d2f13cca
MaSh exporter can now export subsets of the facts, as consecutive ranges
 blanchet parents: 
50557diff
changeset | 90 | val th = | 
| 50624 
4d0997abce79
improved thm order hack, in case the default names are overridden
 blanchet parents: 
50620diff
changeset | 91 | case find_first (fn (_, th) => nickname_of_thm th = name) facts of | 
| 50559 
89c0d2f13cca
MaSh exporter can now export subsets of the facts, as consecutive ranges
 blanchet parents: 
50557diff
changeset | 92 | SOME (_, th) => th | 
| 
89c0d2f13cca
MaSh exporter can now export subsets of the facts, as consecutive ranges
 blanchet parents: 
50557diff
changeset | 93 |             | NONE => error ("No fact called \"" ^ name ^ "\".")
 | 
| 
89c0d2f13cca
MaSh exporter can now export subsets of the facts, as consecutive ranges
 blanchet parents: 
50557diff
changeset | 94 | val goal = goal_of_thm (Proof_Context.theory_of ctxt) th | 
| 52196 
2281f33e8da6
redid rac7830871177 to avoid duplicate fixed variable (e.g. lemma "P (a::nat)" proof - have "!!a::int. Q a" sledgehammer [e])
 blanchet parents: 
52125diff
changeset | 95 | val (_, hyp_ts, concl_t) = ATP_Util.strip_subgoal goal 1 ctxt | 
| 57306 
ff10067b2248
optimized traversal of proof terms by skipping bad apples (e.g. full_exhaustive_int'.pinduct)
 blanchet parents: 
57150diff
changeset | 96 | val isar_deps = these (isar_dependencies_of name_tabs th) | 
| 57456 | 97 | val suggss = isar_deps :: suggss0 | 
| 57406 | 98 | val facts = facts |> filter (fn (_, th') => thm_less (th', th)) | 
| 57432 | 99 | |
| 50559 
89c0d2f13cca
MaSh exporter can now export subsets of the facts, as consecutive ranges
 blanchet parents: 
50557diff
changeset | 100 | (* adapted from "mirabelle_sledgehammer.ML" *) | 
| 50953 | 101 | fun set_file_name method (SOME dir) = | 
| 50559 
89c0d2f13cca
MaSh exporter can now export subsets of the facts, as consecutive ranges
 blanchet parents: 
50557diff
changeset | 102 | let | 
| 57432 | 103 | val prob_prefix = "goal_" ^ string_of_int j ^ "__" ^ encode_str name ^ "__" ^ method | 
| 50559 
89c0d2f13cca
MaSh exporter can now export subsets of the facts, as consecutive ranges
 blanchet parents: 
50557diff
changeset | 104 | in | 
| 55212 | 105 | Config.put atp_dest_dir dir | 
| 106 | #> Config.put atp_problem_prefix (prob_prefix ^ "__") | |
| 58061 | 107 | #> Config.put SMT_Config.debug_files (dir ^ "/" ^ prob_prefix) | 
| 50559 
89c0d2f13cca
MaSh exporter can now export subsets of the facts, as consecutive ranges
 blanchet parents: 
50557diff
changeset | 108 | end | 
| 
89c0d2f13cca
MaSh exporter can now export subsets of the facts, as consecutive ranges
 blanchet parents: 
50557diff
changeset | 109 | | set_file_name _ NONE = I | 
| 57432 | 110 | |
| 53139 | 111 | fun prove method suggs = | 
| 57456 | 112 | if null facts then | 
| 50953 | 113 | (str_of_method method ^ "Skipped", 0) | 
| 50952 | 114 | else | 
| 115 | let | |
| 116 | fun nickify ((_, stature), th) = | |
| 117 | ((K (encode_str (nickname_of_thm th)), stature), th) | |
| 57432 | 118 | |
| 50952 | 119 | val facts = | 
| 53139 | 120 | suggs | 
| 121 | |> find_suggested_facts ctxt facts | |
| 122 | |> map (fact_of_raw_fact #> nickify) | |
| 50952 | 123 | |> maybe_instantiate_inducts ctxt hyp_ts concl_t | 
| 124 | |> take (the max_facts) | |
| 51004 
5f2788c38127
distinguish raw and non-raw facts, using raw for 10 000s of facts and non-raw after selection of some hundreds
 blanchet parents: 
50967diff
changeset | 125 | |> map fact_of_raw_fact | 
| 50953 | 126 | val ctxt = ctxt |> set_file_name method prob_dir_name | 
| 57434 | 127 |                 val res as {outcome, ...} = run_prover_for_mash ctxt params prover name facts goal
 | 
| 50952 | 128 | val ok = if is_none outcome then 1 else 0 | 
| 57432 | 129 | in | 
| 130 | (str_of_result method facts res, ok) | |
| 131 | end | |
| 132 | ||
| 57456 | 133 | val ress = map2 prove methods suggss | 
| 50559 
89c0d2f13cca
MaSh exporter can now export subsets of the facts, as consecutive ranges
 blanchet parents: 
50557diff
changeset | 134 | in | 
| 50591 | 135 | "Goal " ^ string_of_int j ^ ": " ^ name :: map fst ress | 
| 50587 
bd6582be1562
synchronize access to shared reference and print proper total
 blanchet parents: 
50563diff
changeset | 136 | |> cat_lines |> print; | 
| 50591 | 137 | map snd ress | 
| 50559 
89c0d2f13cca
MaSh exporter can now export subsets of the facts, as consecutive ranges
 blanchet parents: 
50557diff
changeset | 138 | end | 
| 
89c0d2f13cca
MaSh exporter can now export subsets of the facts, as consecutive ranges
 blanchet parents: 
50557diff
changeset | 139 | else | 
| 51028 | 140 | zeros | 
| 57432 | 141 | |
| 50557 | 142 | val inst_inducts = Config.get ctxt instantiate_inducts | 
| 48245 | 143 | val options = | 
| 50767 | 144 | ["prover = " ^ prover, | 
| 145 | "max_facts = " ^ string_of_int (the max_facts), | |
| 146 | "slice" |> not slice ? prefix "dont_", | |
| 147 | "type_enc = " ^ the_default "smart" type_enc, | |
| 148 | "lam_trans = " ^ the_default "smart" lam_trans, | |
| 54816 
10d48c2a3e32
made timeouts in Sledgehammer not be 'option's -- simplified lots of code
 blanchet parents: 
54141diff
changeset | 149 | "timeout = " ^ ATP_Util.string_of_time timeout, | 
| 48241 | 150 | "instantiate_inducts" |> not inst_inducts ? prefix "dont_"] | 
| 50587 
bd6582be1562
synchronize access to shared reference and print proper total
 blanchet parents: 
50563diff
changeset | 151 | val _ = print " * * *"; | 
| 
bd6582be1562
synchronize access to shared reference and print proper total
 blanchet parents: 
50563diff
changeset | 152 |     val _ = print ("Options: " ^ commas options);
 | 
| 57456 | 153 | val oks = Par_List.map solve_goal (tag_list 1 liness) | 
| 50620 | 154 | val n = length oks | 
| 57456 | 155 | |
| 156 | fun total_of method ok = | |
| 157 |       str_of_method method ^ string_of_int ok ^ " (" ^ Real.fmt (StringCvt.FIX (SOME 1))
 | |
| 158 | (100.0 * Real.fromInt ok / Real.fromInt (Int.max (1, n))) ^ "%)" | |
| 159 | ||
| 160 | val oks' = if n = 0 then zeros else map Integer.sum (map_transpose I oks) | |
| 48241 | 161 | in | 
| 57456 | 162 | "Successes (of " ^ string_of_int n ^ " goals)" :: | 
| 163 | map2 total_of methods oks' | |
| 50437 | 164 | |> cat_lines |> print | 
| 48241 | 165 | end | 
| 48235 | 166 | |
| 48234 | 167 | end; |