author | blanchet |
Wed, 12 Dec 2012 00:24:06 +0100 | |
changeset 50484 | 8ec31bdb9d36 |
parent 50442 | 4f6a4d32522c |
child 50485 | 3c6ac2da2f45 |
permissions | -rw-r--r-- |
48234 | 1 |
(* Title: HOL/TPTP/mash_export.ML |
2 |
Author: Jasmin Blanchette, TU Muenchen |
|
3 |
Copyright 2012 |
|
4 |
||
5 |
Export Isabelle theory information for MaSh (Machine-learning for Sledgehammer). |
|
6 |
*) |
|
7 |
||
8 |
signature MASH_EXPORT = |
|
9 |
sig |
|
48251
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
blanchet
parents:
48250
diff
changeset
|
10 |
type params = Sledgehammer_Provers.params |
48235 | 11 |
|
50349 | 12 |
val generate_accessibility : |
13 |
Proof.context -> theory list -> bool -> string -> unit |
|
48318 | 14 |
val generate_features : |
50349 | 15 |
Proof.context -> string -> theory list -> bool -> string -> unit |
48333 | 16 |
val generate_isar_dependencies : |
50349 | 17 |
Proof.context -> theory list -> bool -> string -> unit |
50484
8ec31bdb9d36
adopt the neutral "prover" terminology for MaSh rather than the ambiguous/wrong ATP terminology (which sometimes excludes SMT solvers)
blanchet
parents:
50442
diff
changeset
|
18 |
val generate_prover_dependencies : |
50349 | 19 |
Proof.context -> params -> theory list -> bool -> string -> unit |
50411 | 20 |
val generate_isar_commands : |
21 |
Proof.context -> string -> theory list -> string -> unit |
|
50484
8ec31bdb9d36
adopt the neutral "prover" terminology for MaSh rather than the ambiguous/wrong ATP terminology (which sometimes excludes SMT solvers)
blanchet
parents:
50442
diff
changeset
|
22 |
val generate_prover_commands : |
50349 | 23 |
Proof.context -> params -> theory list -> string -> unit |
48379
2b5ad61e2ccc
renamed "iter" fact filter to "MePo" (Meng--Paulson)
blanchet
parents:
48378
diff
changeset
|
24 |
val generate_mepo_suggestions : |
50349 | 25 |
Proof.context -> params -> theory list -> int -> string -> unit |
48234 | 26 |
end; |
27 |
||
28 |
structure MaSh_Export : MASH_EXPORT = |
|
29 |
struct |
|
30 |
||
48381 | 31 |
open Sledgehammer_MePo |
32 |
open Sledgehammer_MaSh |
|
48245 | 33 |
|
48316
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents:
48315
diff
changeset
|
34 |
fun thy_map_from_facts ths = |
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents:
48315
diff
changeset
|
35 |
ths |> sort (thm_ord o swap o pairself snd) |
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents:
48315
diff
changeset
|
36 |
|> map (snd #> `(theory_of_thm #> Context.theory_name)) |
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents:
48315
diff
changeset
|
37 |
|> AList.coalesce (op =) |
48378 | 38 |
|> map (apsnd (map nickname_of)) |
48316
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents:
48315
diff
changeset
|
39 |
|
50349 | 40 |
fun has_thm_thy th thy = |
48316
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents:
48315
diff
changeset
|
41 |
Context.theory_name thy = Context.theory_name (theory_of_thm th) |
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents:
48315
diff
changeset
|
42 |
|
50349 | 43 |
fun has_thys thys th = exists (has_thm_thy th) thys |
44 |
||
45 |
fun all_facts ctxt = |
|
48531 | 46 |
let val css = Sledgehammer_Fact.clasimpset_rule_table_of ctxt in |
50442
4f6a4d32522c
don't blacklist "case" theorems -- this causes problems in MaSh later
blanchet
parents:
50434
diff
changeset
|
47 |
Sledgehammer_Fact.all_facts ctxt true false Symtab.empty [] [] css |
48531 | 48 |
end |
49 |
||
50349 | 50 |
fun add_thy_parent_facts thy_map thy = |
48316
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents:
48315
diff
changeset
|
51 |
let |
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents:
48315
diff
changeset
|
52 |
fun add_last thy = |
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents:
48315
diff
changeset
|
53 |
case AList.lookup (op =) thy_map (Context.theory_name thy) of |
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents:
48315
diff
changeset
|
54 |
SOME (last_fact :: _) => insert (op =) last_fact |
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents:
48315
diff
changeset
|
55 |
| _ => add_parent thy |
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents:
48315
diff
changeset
|
56 |
and add_parent thy = fold add_last (Theory.parents_of thy) |
50349 | 57 |
in add_parent thy end |
48316
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents:
48315
diff
changeset
|
58 |
|
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents:
48315
diff
changeset
|
59 |
val thy_name_of_fact = hd o Long_Name.explode |
50349 | 60 |
fun thy_of_fact thy = Context.get_theory thy o thy_name_of_fact |
48304 | 61 |
|
48438
3e45c98fe127
distinguish between recursive and nonrecursive definitions + clean up typedef dependencies in MaSh
blanchet
parents:
48406
diff
changeset
|
62 |
val all_names = map (rpair () o nickname_of) #> Symtab.make |
48316
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
blanchet
parents:
48315
diff
changeset
|
63 |
|
50349 | 64 |
fun generate_accessibility ctxt thys include_thys file_name = |
48304 | 65 |
let |
66 |
val path = file_name |> Path.explode |
|
67 |
val _ = File.write path "" |
|
68 |
fun do_fact fact prevs = |
|
69 |
let |
|
70 |
val s = escape_meta fact ^ ": " ^ escape_metas prevs ^ "\n" |
|
71 |
val _ = File.append path s |
|
72 |
in [fact] end |
|
48315
82d6e46c673f
fixed order of accessibles + other tweaks to MaSh
blanchet
parents:
48304
diff
changeset
|
73 |
val thy_map = |
50349 | 74 |
all_facts ctxt |
75 |
|> not include_thys ? filter_out (has_thys thys o snd) |
|
48315
82d6e46c673f
fixed order of accessibles + other tweaks to MaSh
blanchet
parents:
48304
diff
changeset
|
76 |
|> thy_map_from_facts |
48304 | 77 |
fun do_thy facts = |
78 |
let |
|
50349 | 79 |
val thy = thy_of_fact (Proof_Context.theory_of ctxt) (hd facts) |
80 |
val parents = add_thy_parent_facts thy_map thy [] |
|
48530
d443166f9520
repaired accessibility chains generated by MaSh exporter + tuned one function out
blanchet
parents:
48529
diff
changeset
|
81 |
in fold_rev do_fact facts parents; () end |
48333 | 82 |
in fold_rev (fn (_, facts) => fn () => do_thy facts) thy_map () end |
48304 | 83 |
|
50349 | 84 |
fun generate_features ctxt prover thys include_thys file_name = |
48304 | 85 |
let |
86 |
val path = file_name |> Path.explode |
|
87 |
val _ = File.write path "" |
|
88 |
val facts = |
|
50349 | 89 |
all_facts ctxt |
90 |
|> not include_thys ? filter_out (has_thys thys o snd) |
|
48385 | 91 |
fun do_fact ((_, stature), th) = |
48304 | 92 |
let |
48378 | 93 |
val name = nickname_of th |
48318 | 94 |
val feats = |
48385 | 95 |
features_of ctxt prover (theory_of_thm th) stature [prop_of th] |
50356 | 96 |
val s = escape_meta name ^ ": " ^ encode_features feats ^ "\n" |
48304 | 97 |
in File.append path s end |
98 |
in List.app do_fact facts end |
|
99 |
||
50484
8ec31bdb9d36
adopt the neutral "prover" terminology for MaSh rather than the ambiguous/wrong ATP terminology (which sometimes excludes SMT solvers)
blanchet
parents:
50442
diff
changeset
|
100 |
fun isar_or_prover_dependencies_of ctxt params_opt facts all_names th = |
50411 | 101 |
(case params_opt of |
102 |
SOME (params as {provers = prover :: _, ...}) => |
|
50484
8ec31bdb9d36
adopt the neutral "prover" terminology for MaSh rather than the ambiguous/wrong ATP terminology (which sometimes excludes SMT solvers)
blanchet
parents:
50442
diff
changeset
|
103 |
prover_dependencies_of ctxt params prover 0 facts all_names th |> snd |
50411 | 104 |
| NONE => isar_dependencies_of all_names th) |
105 |
|> these |
|
106 |
||
50484
8ec31bdb9d36
adopt the neutral "prover" terminology for MaSh rather than the ambiguous/wrong ATP terminology (which sometimes excludes SMT solvers)
blanchet
parents:
50442
diff
changeset
|
107 |
fun generate_isar_or_prover_dependencies ctxt params_opt thys include_thys |
8ec31bdb9d36
adopt the neutral "prover" terminology for MaSh rather than the ambiguous/wrong ATP terminology (which sometimes excludes SMT solvers)
blanchet
parents:
50442
diff
changeset
|
108 |
file_name = |
48304 | 109 |
let |
110 |
val path = file_name |> Path.explode |
|
111 |
val _ = File.write path "" |
|
112 |
val facts = |
|
50349 | 113 |
all_facts ctxt |
114 |
|> not include_thys ? filter_out (has_thys thys o snd) |
|
48304 | 115 |
val ths = facts |> map snd |
48324 | 116 |
val all_names = all_names ths |
48304 | 117 |
fun do_thm th = |
118 |
let |
|
48378 | 119 |
val name = nickname_of th |
48665 | 120 |
val deps = |
50484
8ec31bdb9d36
adopt the neutral "prover" terminology for MaSh rather than the ambiguous/wrong ATP terminology (which sometimes excludes SMT solvers)
blanchet
parents:
50442
diff
changeset
|
121 |
isar_or_prover_dependencies_of ctxt params_opt facts all_names th |
48304 | 122 |
val s = escape_meta name ^ ": " ^ escape_metas deps ^ "\n" |
123 |
in File.append path s end |
|
124 |
in List.app do_thm ths end |
|
125 |
||
50411 | 126 |
fun generate_isar_dependencies ctxt = |
50484
8ec31bdb9d36
adopt the neutral "prover" terminology for MaSh rather than the ambiguous/wrong ATP terminology (which sometimes excludes SMT solvers)
blanchet
parents:
50442
diff
changeset
|
127 |
generate_isar_or_prover_dependencies ctxt NONE |
50411 | 128 |
|
50484
8ec31bdb9d36
adopt the neutral "prover" terminology for MaSh rather than the ambiguous/wrong ATP terminology (which sometimes excludes SMT solvers)
blanchet
parents:
50442
diff
changeset
|
129 |
fun generate_prover_dependencies ctxt params = |
8ec31bdb9d36
adopt the neutral "prover" terminology for MaSh rather than the ambiguous/wrong ATP terminology (which sometimes excludes SMT solvers)
blanchet
parents:
50442
diff
changeset
|
130 |
generate_isar_or_prover_dependencies ctxt (SOME params) |
50411 | 131 |
|
50484
8ec31bdb9d36
adopt the neutral "prover" terminology for MaSh rather than the ambiguous/wrong ATP terminology (which sometimes excludes SMT solvers)
blanchet
parents:
50442
diff
changeset
|
132 |
fun generate_isar_or_prover_commands ctxt prover params_opt thys file_name = |
48234 | 133 |
let |
134 |
val path = file_name |> Path.explode |
|
135 |
val _ = File.write path "" |
|
50349 | 136 |
val facts = all_facts ctxt |
48234 | 137 |
val (new_facts, old_facts) = |
50349 | 138 |
facts |> List.partition (has_thys thys o snd) |
48234 | 139 |
|>> sort (thm_ord o pairself snd) |
48665 | 140 |
val all_names = all_names (map snd facts) |
48385 | 141 |
fun do_fact ((_, stature), th) prevs = |
48234 | 142 |
let |
48378 | 143 |
val name = nickname_of th |
50349 | 144 |
val feats = |
145 |
features_of ctxt prover (theory_of_thm th) stature [prop_of th] |
|
48665 | 146 |
val deps = |
50484
8ec31bdb9d36
adopt the neutral "prover" terminology for MaSh rather than the ambiguous/wrong ATP terminology (which sometimes excludes SMT solvers)
blanchet
parents:
50442
diff
changeset
|
147 |
isar_or_prover_dependencies_of ctxt params_opt facts all_names th |
48234 | 148 |
val kind = Thm.legacy_get_kind th |
48529
716ec3458b1d
generate fact name in queries again + use ATP dependencies when possible
blanchet
parents:
48438
diff
changeset
|
149 |
val core = |
716ec3458b1d
generate fact name in queries again + use ATP dependencies when possible
blanchet
parents:
48438
diff
changeset
|
150 |
escape_meta name ^ ": " ^ escape_metas prevs ^ "; " ^ |
50356 | 151 |
encode_features feats |
48666 | 152 |
val query = |
153 |
if kind = "" orelse null deps then "" else "? " ^ core ^ "\n" |
|
48529
716ec3458b1d
generate fact name in queries again + use ATP dependencies when possible
blanchet
parents:
48438
diff
changeset
|
154 |
val update = "! " ^ core ^ "; " ^ escape_metas deps ^ "\n" |
48234 | 155 |
val _ = File.append path (query ^ update) |
156 |
in [name] end |
|
48315
82d6e46c673f
fixed order of accessibles + other tweaks to MaSh
blanchet
parents:
48304
diff
changeset
|
157 |
val thy_map = old_facts |> thy_map_from_facts |
50349 | 158 |
val parents = fold (add_thy_parent_facts thy_map) thys [] |
48239
0016290f904c
generate Meng--Paulson facts for evaluation purposes
blanchet
parents:
48235
diff
changeset
|
159 |
in fold do_fact new_facts parents; () end |
0016290f904c
generate Meng--Paulson facts for evaluation purposes
blanchet
parents:
48235
diff
changeset
|
160 |
|
50411 | 161 |
fun generate_isar_commands ctxt prover = |
50484
8ec31bdb9d36
adopt the neutral "prover" terminology for MaSh rather than the ambiguous/wrong ATP terminology (which sometimes excludes SMT solvers)
blanchet
parents:
50442
diff
changeset
|
162 |
generate_isar_or_prover_commands ctxt prover NONE |
50411 | 163 |
|
50484
8ec31bdb9d36
adopt the neutral "prover" terminology for MaSh rather than the ambiguous/wrong ATP terminology (which sometimes excludes SMT solvers)
blanchet
parents:
50442
diff
changeset
|
164 |
fun generate_prover_commands ctxt (params as {provers = prover :: _, ...}) = |
8ec31bdb9d36
adopt the neutral "prover" terminology for MaSh rather than the ambiguous/wrong ATP terminology (which sometimes excludes SMT solvers)
blanchet
parents:
50442
diff
changeset
|
165 |
generate_isar_or_prover_commands ctxt prover (SOME params) |
50411 | 166 |
|
50349 | 167 |
fun generate_mepo_suggestions ctxt (params as {provers, ...}) thys max_relevant |
48292 | 168 |
file_name = |
48239
0016290f904c
generate Meng--Paulson facts for evaluation purposes
blanchet
parents:
48235
diff
changeset
|
169 |
let |
0016290f904c
generate Meng--Paulson facts for evaluation purposes
blanchet
parents:
48235
diff
changeset
|
170 |
val path = file_name |> Path.explode |
0016290f904c
generate Meng--Paulson facts for evaluation purposes
blanchet
parents:
48235
diff
changeset
|
171 |
val _ = File.write path "" |
48318 | 172 |
val prover = hd provers |
50349 | 173 |
val facts = all_facts ctxt |
48239
0016290f904c
generate Meng--Paulson facts for evaluation purposes
blanchet
parents:
48235
diff
changeset
|
174 |
val (new_facts, old_facts) = |
50349 | 175 |
facts |> List.partition (has_thys thys o snd) |
48239
0016290f904c
generate Meng--Paulson facts for evaluation purposes
blanchet
parents:
48235
diff
changeset
|
176 |
|>> sort (thm_ord o pairself snd) |
0016290f904c
generate Meng--Paulson facts for evaluation purposes
blanchet
parents:
48235
diff
changeset
|
177 |
fun do_fact (fact as (_, th)) old_facts = |
0016290f904c
generate Meng--Paulson facts for evaluation purposes
blanchet
parents:
48235
diff
changeset
|
178 |
let |
48378 | 179 |
val name = nickname_of th |
50349 | 180 |
val goal = goal_of_thm (Proof_Context.theory_of ctxt) th |
48292 | 181 |
val (_, hyp_ts, concl_t) = ATP_Util.strip_subgoal ctxt goal 1 |
48239
0016290f904c
generate Meng--Paulson facts for evaluation purposes
blanchet
parents:
48235
diff
changeset
|
182 |
val kind = Thm.legacy_get_kind th |
0016290f904c
generate Meng--Paulson facts for evaluation purposes
blanchet
parents:
48235
diff
changeset
|
183 |
val _ = |
0016290f904c
generate Meng--Paulson facts for evaluation purposes
blanchet
parents:
48235
diff
changeset
|
184 |
if kind <> "" then |
0016290f904c
generate Meng--Paulson facts for evaluation purposes
blanchet
parents:
48235
diff
changeset
|
185 |
let |
0016290f904c
generate Meng--Paulson facts for evaluation purposes
blanchet
parents:
48235
diff
changeset
|
186 |
val suggs = |
48292 | 187 |
old_facts |
48406 | 188 |
|> Sledgehammer_MePo.mepo_suggested_facts ctxt params prover |
48381 | 189 |
max_relevant NONE hyp_ts concl_t |
50402 | 190 |
|> map (nickname_of o snd) |
48303
f1d135d0ea69
improved MaSh string escaping and make more operations string-based
blanchet
parents:
48302
diff
changeset
|
191 |
val s = escape_meta name ^ ": " ^ escape_metas suggs ^ "\n" |
48239
0016290f904c
generate Meng--Paulson facts for evaluation purposes
blanchet
parents:
48235
diff
changeset
|
192 |
in File.append path s end |
0016290f904c
generate Meng--Paulson facts for evaluation purposes
blanchet
parents:
48235
diff
changeset
|
193 |
else |
0016290f904c
generate Meng--Paulson facts for evaluation purposes
blanchet
parents:
48235
diff
changeset
|
194 |
() |
0016290f904c
generate Meng--Paulson facts for evaluation purposes
blanchet
parents:
48235
diff
changeset
|
195 |
in fact :: old_facts end |
0016290f904c
generate Meng--Paulson facts for evaluation purposes
blanchet
parents:
48235
diff
changeset
|
196 |
in fold do_fact new_facts old_facts; () end |
48234 | 197 |
|
198 |
end; |