author | blanchet |
Fri, 01 Jul 2011 15:53:38 +0200 | |
changeset 43626 | a867ebb12209 |
parent 43572 | ae612a423dad |
child 43989 | eb763b3ff9ed |
permissions | -rw-r--r-- |
36375
2482446a604c
move the minimizer to the Sledgehammer directory
blanchet
parents:
36373
diff
changeset
|
1 |
(* Title: HOL/Tools/Sledgehammer/sledgehammer_isar.ML |
35866
513074557e06
move the Sledgehammer Isar commands together into one file;
blanchet
parents:
diff
changeset
|
2 |
Author: Jasmin Blanchette, TU Muenchen |
513074557e06
move the Sledgehammer Isar commands together into one file;
blanchet
parents:
diff
changeset
|
3 |
|
513074557e06
move the Sledgehammer Isar commands together into one file;
blanchet
parents:
diff
changeset
|
4 |
Adds "sledgehammer" and related commands to Isabelle/Isar's outer syntax. |
513074557e06
move the Sledgehammer Isar commands together into one file;
blanchet
parents:
diff
changeset
|
5 |
*) |
513074557e06
move the Sledgehammer Isar commands together into one file;
blanchet
parents:
diff
changeset
|
6 |
|
35963 | 7 |
signature SLEDGEHAMMER_ISAR = |
8 |
sig |
|
41087
d7b5fd465198
split "Sledgehammer" module into two parts, to resolve forthcoming dependency problems
blanchet
parents:
40941
diff
changeset
|
9 |
type params = Sledgehammer_Provers.params |
35963 | 10 |
|
43020
abb5d1f907e4
added "try" command, to launch Solve Direct, Quickcheck, Nitpick, Sledgehammer, and Try Methods
blanchet
parents:
43018
diff
changeset
|
11 |
val sledgehammerN : string |
39318 | 12 |
val auto : bool Unsynchronized.ref |
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39335
diff
changeset
|
13 |
val provers : string Unsynchronized.ref |
39318 | 14 |
val timeout : int Unsynchronized.ref |
40069 | 15 |
val default_params : Proof.context -> (string * string) list -> params |
39318 | 16 |
val setup : theory -> theory |
35963 | 17 |
end; |
18 |
||
35971 | 19 |
structure Sledgehammer_Isar : SLEDGEHAMMER_ISAR = |
35866
513074557e06
move the Sledgehammer Isar commands together into one file;
blanchet
parents:
diff
changeset
|
20 |
struct |
513074557e06
move the Sledgehammer Isar commands together into one file;
blanchet
parents:
diff
changeset
|
21 |
|
38028 | 22 |
open ATP_Systems |
43085
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
blanchet
parents:
43064
diff
changeset
|
23 |
open ATP_Translate |
35971 | 24 |
open Sledgehammer_Util |
41087
d7b5fd465198
split "Sledgehammer" module into two parts, to resolve forthcoming dependency problems
blanchet
parents:
40941
diff
changeset
|
25 |
open Sledgehammer_Provers |
38988 | 26 |
open Sledgehammer_Minimize |
41087
d7b5fd465198
split "Sledgehammer" module into two parts, to resolve forthcoming dependency problems
blanchet
parents:
40941
diff
changeset
|
27 |
open Sledgehammer_Run |
35866
513074557e06
move the Sledgehammer Isar commands together into one file;
blanchet
parents:
diff
changeset
|
28 |
|
43020
abb5d1f907e4
added "try" command, to launch Solve Direct, Quickcheck, Nitpick, Sledgehammer, and Try Methods
blanchet
parents:
43018
diff
changeset
|
29 |
val sledgehammerN = "sledgehammer" |
abb5d1f907e4
added "try" command, to launch Solve Direct, Quickcheck, Nitpick, Sledgehammer, and Try Methods
blanchet
parents:
43018
diff
changeset
|
30 |
val sledgehammer_paramsN = "sledgehammer_params" |
abb5d1f907e4
added "try" command, to launch Solve Direct, Quickcheck, Nitpick, Sledgehammer, and Try Methods
blanchet
parents:
43018
diff
changeset
|
31 |
|
abb5d1f907e4
added "try" command, to launch Solve Direct, Quickcheck, Nitpick, Sledgehammer, and Try Methods
blanchet
parents:
43018
diff
changeset
|
32 |
val runN = "run" |
abb5d1f907e4
added "try" command, to launch Solve Direct, Quickcheck, Nitpick, Sledgehammer, and Try Methods
blanchet
parents:
43018
diff
changeset
|
33 |
val minN = "min" |
abb5d1f907e4
added "try" command, to launch Solve Direct, Quickcheck, Nitpick, Sledgehammer, and Try Methods
blanchet
parents:
43018
diff
changeset
|
34 |
val messagesN = "messages" |
abb5d1f907e4
added "try" command, to launch Solve Direct, Quickcheck, Nitpick, Sledgehammer, and Try Methods
blanchet
parents:
43018
diff
changeset
|
35 |
val supported_proversN = "supported_provers" |
abb5d1f907e4
added "try" command, to launch Solve Direct, Quickcheck, Nitpick, Sledgehammer, and Try Methods
blanchet
parents:
43018
diff
changeset
|
36 |
val running_proversN = "running_provers" |
abb5d1f907e4
added "try" command, to launch Solve Direct, Quickcheck, Nitpick, Sledgehammer, and Try Methods
blanchet
parents:
43018
diff
changeset
|
37 |
val kill_proversN = "kill_provers" |
abb5d1f907e4
added "try" command, to launch Solve Direct, Quickcheck, Nitpick, Sledgehammer, and Try Methods
blanchet
parents:
43018
diff
changeset
|
38 |
val refresh_tptpN = "refresh_tptp" |
abb5d1f907e4
added "try" command, to launch Solve Direct, Quickcheck, Nitpick, Sledgehammer, and Try Methods
blanchet
parents:
43018
diff
changeset
|
39 |
|
39318 | 40 |
val auto = Unsynchronized.ref false |
41 |
||
42 |
val _ = |
|
43 |
ProofGeneralPgip.add_preference Preferences.category_tracing |
|
44 |
(Preferences.bool_pref auto "auto-sledgehammer" |
|
39327 | 45 |
"Run Sledgehammer automatically.") |
39318 | 46 |
|
36394
1a48d18449d8
move "neg_clausify" method and "clausify" attribute to "sledgehammer_isar.ML"
blanchet
parents:
36378
diff
changeset
|
47 |
(** Sledgehammer commands **) |
1a48d18449d8
move "neg_clausify" method and "clausify" attribute to "sledgehammer_isar.ML"
blanchet
parents:
36378
diff
changeset
|
48 |
|
39318 | 49 |
val no_relevance_override = {add = [], del = [], only = false} |
50 |
fun add_relevance_override ns : relevance_override = |
|
35966
f8c738abaed8
honor the newly introduced Sledgehammer parameters and fixed the parsing;
blanchet
parents:
35965
diff
changeset
|
51 |
{add = ns, del = [], only = false} |
39318 | 52 |
fun del_relevance_override ns : relevance_override = |
35966
f8c738abaed8
honor the newly introduced Sledgehammer parameters and fixed the parsing;
blanchet
parents:
35965
diff
changeset
|
53 |
{add = [], del = ns, only = false} |
f8c738abaed8
honor the newly introduced Sledgehammer parameters and fixed the parsing;
blanchet
parents:
35965
diff
changeset
|
54 |
fun only_relevance_override ns : relevance_override = |
f8c738abaed8
honor the newly introduced Sledgehammer parameters and fixed the parsing;
blanchet
parents:
35965
diff
changeset
|
55 |
{add = ns, del = [], only = true} |
36003 | 56 |
fun merge_relevance_override_pairwise (r1 : relevance_override) |
57 |
(r2 : relevance_override) = |
|
35966
f8c738abaed8
honor the newly introduced Sledgehammer parameters and fixed the parsing;
blanchet
parents:
35965
diff
changeset
|
58 |
{add = #add r1 @ #add r2, del = #del r1 @ #del r2, |
36183
f723348b2231
Sledgehammer: the empty set of fact () should mean nothing, not unchanged
blanchet
parents:
36143
diff
changeset
|
59 |
only = #only r1 andalso #only r2} |
36188 | 60 |
fun merge_relevance_overrides rs = |
61 |
fold merge_relevance_override_pairwise rs (only_relevance_override []) |
|
35965
0fce6db7babd
added a syntax for specifying facts to Sledgehammer;
blanchet
parents:
35963
diff
changeset
|
62 |
|
36371
8c83ea1a7740
move the Sledgehammer menu options to "sledgehammer_isar.ML"
blanchet
parents:
36290
diff
changeset
|
63 |
(*** parameters ***) |
8c83ea1a7740
move the Sledgehammer menu options to "sledgehammer_isar.ML"
blanchet
parents:
36290
diff
changeset
|
64 |
|
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39335
diff
changeset
|
65 |
val provers = Unsynchronized.ref "" |
39335
87a9ff4d5817
use 30 s instead of 60 s as the default Sledgehammer timeout;
blanchet
parents:
39327
diff
changeset
|
66 |
val timeout = Unsynchronized.ref 30 |
36371
8c83ea1a7740
move the Sledgehammer menu options to "sledgehammer_isar.ML"
blanchet
parents:
36290
diff
changeset
|
67 |
|
8c83ea1a7740
move the Sledgehammer menu options to "sledgehammer_isar.ML"
blanchet
parents:
36290
diff
changeset
|
68 |
val _ = |
8c83ea1a7740
move the Sledgehammer menu options to "sledgehammer_isar.ML"
blanchet
parents:
36290
diff
changeset
|
69 |
ProofGeneralPgip.add_preference Preferences.category_proof |
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39335
diff
changeset
|
70 |
(Preferences.string_pref provers |
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39335
diff
changeset
|
71 |
"Sledgehammer: Provers" |
36371
8c83ea1a7740
move the Sledgehammer menu options to "sledgehammer_isar.ML"
blanchet
parents:
36290
diff
changeset
|
72 |
"Default automatic provers (separated by whitespace)") |
8c83ea1a7740
move the Sledgehammer menu options to "sledgehammer_isar.ML"
blanchet
parents:
36290
diff
changeset
|
73 |
|
8c83ea1a7740
move the Sledgehammer menu options to "sledgehammer_isar.ML"
blanchet
parents:
36290
diff
changeset
|
74 |
val _ = |
8c83ea1a7740
move the Sledgehammer menu options to "sledgehammer_isar.ML"
blanchet
parents:
36290
diff
changeset
|
75 |
ProofGeneralPgip.add_preference Preferences.category_proof |
8c83ea1a7740
move the Sledgehammer menu options to "sledgehammer_isar.ML"
blanchet
parents:
36290
diff
changeset
|
76 |
(Preferences.int_pref timeout |
36373
66af0a49de39
move some sledgehammer stuff out of "atp_manager.ML"
blanchet
parents:
36371
diff
changeset
|
77 |
"Sledgehammer: Time Limit" |
36371
8c83ea1a7740
move the Sledgehammer menu options to "sledgehammer_isar.ML"
blanchet
parents:
36290
diff
changeset
|
78 |
"ATPs will be interrupted after this time (in seconds)") |
8c83ea1a7740
move the Sledgehammer menu options to "sledgehammer_isar.ML"
blanchet
parents:
36290
diff
changeset
|
79 |
|
35963 | 80 |
type raw_param = string * string list |
81 |
||
82 |
val default_default_params = |
|
41208
1b28c43a7074
make "debug" imply "blocking", since in blocking mode the exceptions flow through and are more instructive
blanchet
parents:
41153
diff
changeset
|
83 |
[("debug", "false"), |
35963 | 84 |
("verbose", "false"), |
36143
6490319b1703
added "overlord" option (to get easy access to output files for debugging) + systematically use "raw_goal" rather than an inconsistent mixture
blanchet
parents:
36142
diff
changeset
|
85 |
("overlord", "false"), |
41208
1b28c43a7074
make "debug" imply "blocking", since in blocking mode the exceptions flow through and are more instructive
blanchet
parents:
41153
diff
changeset
|
86 |
("blocking", "false"), |
43626
a867ebb12209
renamed "type_sys" to "type_enc", which is more accurate
blanchet
parents:
43572
diff
changeset
|
87 |
("type_enc", "smart"), |
43572
ae612a423dad
added "sound" option to force Sledgehammer to be pedantically sound
blanchet
parents:
43569
diff
changeset
|
88 |
("sound", "false"), |
42180
a6c141925a8a
added monomorphization option to Sledgehammer ATPs -- this looks promising but is still off by default
blanchet
parents:
41727
diff
changeset
|
89 |
("relevance_thresholds", "0.45 0.85"), |
a6c141925a8a
added monomorphization option to Sledgehammer ATPs -- this looks promising but is still off by default
blanchet
parents:
41727
diff
changeset
|
90 |
("max_relevant", "smart"), |
42783
226962b6a6d1
reduce the number of mono iterations to prevent the mono code from going berserk
blanchet
parents:
42776
diff
changeset
|
91 |
("max_mono_iters", "3"), |
43352
597f31069e18
fewer monomorphic instances are necessary, thanks to Sascha's new monomorphizer -- backed up by Judgment Day
blanchet
parents:
43259
diff
changeset
|
92 |
("max_new_mono_instances", "200"), |
35963 | 93 |
("isar_proof", "false"), |
42443
724e612ba248
implemented general slicing for ATPs, especially E 1.2w and above
blanchet
parents:
42361
diff
changeset
|
94 |
("isar_shrink_factor", "1"), |
43011
5f8d74d3b297
added syntax for specifying Metis timeout (currently used only by SMT solvers)
blanchet
parents:
43009
diff
changeset
|
95 |
("slicing", "true"), |
43034
18259246abb5
try both "metis" and (on failure) "metisFT" in replay
blanchet
parents:
43024
diff
changeset
|
96 |
("preplay_timeout", "4")] |
35963 | 97 |
|
36140
08b2a7ecb6c3
fixed handling of "sledgehammer_params" that get a default value from Isabelle menu;
blanchet
parents:
36064
diff
changeset
|
98 |
val alias_params = |
43353
6c008d3efb0a
removed "atp" and "atps" aliases, which users should have forgotten by now if they ever used them
blanchet
parents:
43352
diff
changeset
|
99 |
[("prover", "provers")] |
36140
08b2a7ecb6c3
fixed handling of "sledgehammer_params" that get a default value from Isabelle menu;
blanchet
parents:
36064
diff
changeset
|
100 |
val negated_alias_params = |
41208
1b28c43a7074
make "debug" imply "blocking", since in blocking mode the exceptions flow through and are more instructive
blanchet
parents:
41153
diff
changeset
|
101 |
[("no_debug", "debug"), |
35963 | 102 |
("quiet", "verbose"), |
36143
6490319b1703
added "overlord" option (to get easy access to output files for debugging) + systematically use "raw_goal" rather than an inconsistent mixture
blanchet
parents:
36142
diff
changeset
|
103 |
("no_overlord", "overlord"), |
41208
1b28c43a7074
make "debug" imply "blocking", since in blocking mode the exceptions flow through and are more instructive
blanchet
parents:
41153
diff
changeset
|
104 |
("non_blocking", "blocking"), |
43572
ae612a423dad
added "sound" option to force Sledgehammer to be pedantically sound
blanchet
parents:
43569
diff
changeset
|
105 |
("unsound", "sound"), |
42443
724e612ba248
implemented general slicing for ATPs, especially E 1.2w and above
blanchet
parents:
42361
diff
changeset
|
106 |
("no_isar_proof", "isar_proof"), |
724e612ba248
implemented general slicing for ATPs, especially E 1.2w and above
blanchet
parents:
42361
diff
changeset
|
107 |
("no_slicing", "slicing")] |
35963 | 108 |
|
36281
dbbf4d5d584d
pass relevant options from "sledgehammer" to "sledgehammer minimize";
blanchet
parents:
36235
diff
changeset
|
109 |
val params_for_minimize = |
43626
a867ebb12209
renamed "type_sys" to "type_enc", which is more accurate
blanchet
parents:
43572
diff
changeset
|
110 |
["debug", "verbose", "overlord", "type_enc", "sound", "max_mono_iters", |
43259
30c141dc22d6
killed "explicit_apply" option in Sledgehammer -- the "smart" default is about as lightweight as "false" and just as complete as "true"
blanchet
parents:
43100
diff
changeset
|
111 |
"max_new_mono_instances", "isar_proof", "isar_shrink_factor", "timeout", |
30c141dc22d6
killed "explicit_apply" option in Sledgehammer -- the "smart" default is about as lightweight as "false" and just as complete as "true"
blanchet
parents:
43100
diff
changeset
|
112 |
"preplay_timeout"] |
36281
dbbf4d5d584d
pass relevant options from "sledgehammer" to "sledgehammer minimize";
blanchet
parents:
36235
diff
changeset
|
113 |
|
43569
b342cd125533
removed "full_types" option from Sledgehammer, now that virtually sound encodings are used as the default anyway
blanchet
parents:
43353
diff
changeset
|
114 |
val property_dependent_params = ["provers", "timeout"] |
35866
513074557e06
move the Sledgehammer Isar commands together into one file;
blanchet
parents:
diff
changeset
|
115 |
|
35963 | 116 |
fun is_known_raw_param s = |
117 |
AList.defined (op =) default_default_params s orelse |
|
36140
08b2a7ecb6c3
fixed handling of "sledgehammer_params" that get a default value from Isabelle menu;
blanchet
parents:
36064
diff
changeset
|
118 |
AList.defined (op =) alias_params s orelse |
08b2a7ecb6c3
fixed handling of "sledgehammer_params" that get a default value from Isabelle menu;
blanchet
parents:
36064
diff
changeset
|
119 |
AList.defined (op =) negated_alias_params s orelse |
38985
162bbbea4e4d
added "expect" feature of Nitpick to Sledgehammer, for regression testing
blanchet
parents:
38982
diff
changeset
|
120 |
member (op =) property_dependent_params s orelse s = "expect" |
35963 | 121 |
|
41258
73401632a80c
convenient syntax for setting provers -- useful for debugging, not for general consumption and hence not documented
blanchet
parents:
41208
diff
changeset
|
122 |
fun is_prover_list ctxt s = |
73401632a80c
convenient syntax for setting provers -- useful for debugging, not for general consumption and hence not documented
blanchet
parents:
41208
diff
changeset
|
123 |
case space_explode " " s of |
41727
ab3f6d76fb23
available_provers ~> supported_provers (for clarity)
blanchet
parents:
41472
diff
changeset
|
124 |
ss as _ :: _ => forall (is_prover_supported ctxt) ss |
41258
73401632a80c
convenient syntax for setting provers -- useful for debugging, not for general consumption and hence not documented
blanchet
parents:
41208
diff
changeset
|
125 |
| _ => false |
73401632a80c
convenient syntax for setting provers -- useful for debugging, not for general consumption and hence not documented
blanchet
parents:
41208
diff
changeset
|
126 |
|
43626
a867ebb12209
renamed "type_sys" to "type_enc", which is more accurate
blanchet
parents:
43572
diff
changeset
|
127 |
(* "provers =" and "type_enc =" can be left out. The latter is a secret |
43572
ae612a423dad
added "sound" option to force Sledgehammer to be pedantically sound
blanchet
parents:
43569
diff
changeset
|
128 |
feature. *) |
41258
73401632a80c
convenient syntax for setting provers -- useful for debugging, not for general consumption and hence not documented
blanchet
parents:
41208
diff
changeset
|
129 |
fun check_and_repair_raw_param ctxt (name, value) = |
42776 | 130 |
if is_known_raw_param name then |
131 |
(name, value) |
|
132 |
else if is_prover_list ctxt name andalso null value then |
|
133 |
("provers", [name]) |
|
43626
a867ebb12209
renamed "type_sys" to "type_enc", which is more accurate
blanchet
parents:
43572
diff
changeset
|
134 |
else if can type_enc_from_string name andalso null value then |
a867ebb12209
renamed "type_sys" to "type_enc", which is more accurate
blanchet
parents:
43572
diff
changeset
|
135 |
("type_enc", [name]) |
42776 | 136 |
else |
137 |
error ("Unknown parameter: " ^ quote name ^ ".") |
|
35866
513074557e06
move the Sledgehammer Isar commands together into one file;
blanchet
parents:
diff
changeset
|
138 |
|
36140
08b2a7ecb6c3
fixed handling of "sledgehammer_params" that get a default value from Isabelle menu;
blanchet
parents:
36064
diff
changeset
|
139 |
fun unalias_raw_param (name, value) = |
08b2a7ecb6c3
fixed handling of "sledgehammer_params" that get a default value from Isabelle menu;
blanchet
parents:
36064
diff
changeset
|
140 |
case AList.lookup (op =) alias_params name of |
08b2a7ecb6c3
fixed handling of "sledgehammer_params" that get a default value from Isabelle menu;
blanchet
parents:
36064
diff
changeset
|
141 |
SOME name' => (name', value) |
08b2a7ecb6c3
fixed handling of "sledgehammer_params" that get a default value from Isabelle menu;
blanchet
parents:
36064
diff
changeset
|
142 |
| NONE => |
08b2a7ecb6c3
fixed handling of "sledgehammer_params" that get a default value from Isabelle menu;
blanchet
parents:
36064
diff
changeset
|
143 |
case AList.lookup (op =) negated_alias_params name of |
08b2a7ecb6c3
fixed handling of "sledgehammer_params" that get a default value from Isabelle menu;
blanchet
parents:
36064
diff
changeset
|
144 |
SOME name' => (name', case value of |
08b2a7ecb6c3
fixed handling of "sledgehammer_params" that get a default value from Isabelle menu;
blanchet
parents:
36064
diff
changeset
|
145 |
["false"] => ["true"] |
08b2a7ecb6c3
fixed handling of "sledgehammer_params" that get a default value from Isabelle menu;
blanchet
parents:
36064
diff
changeset
|
146 |
| ["true"] => ["false"] |
08b2a7ecb6c3
fixed handling of "sledgehammer_params" that get a default value from Isabelle menu;
blanchet
parents:
36064
diff
changeset
|
147 |
| [] => ["false"] |
08b2a7ecb6c3
fixed handling of "sledgehammer_params" that get a default value from Isabelle menu;
blanchet
parents:
36064
diff
changeset
|
148 |
| _ => value) |
08b2a7ecb6c3
fixed handling of "sledgehammer_params" that get a default value from Isabelle menu;
blanchet
parents:
36064
diff
changeset
|
149 |
| NONE => (name, value) |
35963 | 150 |
|
43009
f58bab6be6a9
reintroduced Waldmeister but limit the number of remote threads created
blanchet
parents:
43008
diff
changeset
|
151 |
(* Ensure that type systems such as "simple!" and "mangled_preds?" are handled |
f58bab6be6a9
reintroduced Waldmeister but limit the number of remote threads created
blanchet
parents:
43008
diff
changeset
|
152 |
correctly. *) |
f58bab6be6a9
reintroduced Waldmeister but limit the number of remote threads created
blanchet
parents:
43008
diff
changeset
|
153 |
fun implode_param [s, "?"] = s ^ "?" |
f58bab6be6a9
reintroduced Waldmeister but limit the number of remote threads created
blanchet
parents:
43008
diff
changeset
|
154 |
| implode_param [s, "!"] = s ^ "!" |
f58bab6be6a9
reintroduced Waldmeister but limit the number of remote threads created
blanchet
parents:
43008
diff
changeset
|
155 |
| implode_param ss = space_implode " " ss |
f58bab6be6a9
reintroduced Waldmeister but limit the number of remote threads created
blanchet
parents:
43008
diff
changeset
|
156 |
|
41472
f6ab14e61604
misc tuning and comments based on review of Theory_Data, Proof_Data, Generic_Data usage;
wenzelm
parents:
41258
diff
changeset
|
157 |
structure Data = Theory_Data |
f6ab14e61604
misc tuning and comments based on review of Theory_Data, Proof_Data, Generic_Data usage;
wenzelm
parents:
41258
diff
changeset
|
158 |
( |
35963 | 159 |
type T = raw_param list |
160 |
val empty = default_default_params |> map (apsnd single) |
|
161 |
val extend = I |
|
41472
f6ab14e61604
misc tuning and comments based on review of Theory_Data, Proof_Data, Generic_Data usage;
wenzelm
parents:
41258
diff
changeset
|
162 |
fun merge data : T = AList.merge (op =) (K true) data |
f6ab14e61604
misc tuning and comments based on review of Theory_Data, Proof_Data, Generic_Data usage;
wenzelm
parents:
41258
diff
changeset
|
163 |
) |
35866
513074557e06
move the Sledgehammer Isar commands together into one file;
blanchet
parents:
diff
changeset
|
164 |
|
41727
ab3f6d76fb23
available_provers ~> supported_provers (for clarity)
blanchet
parents:
41472
diff
changeset
|
165 |
fun remotify_prover_if_supported_and_not_already_remote ctxt name = |
40072
27f2a45b0aab
more robust handling of "remote_" vs. non-"remote_" provers
blanchet
parents:
40069
diff
changeset
|
166 |
if String.isPrefix remote_prefix name then |
27f2a45b0aab
more robust handling of "remote_" vs. non-"remote_" provers
blanchet
parents:
40069
diff
changeset
|
167 |
SOME name |
27f2a45b0aab
more robust handling of "remote_" vs. non-"remote_" provers
blanchet
parents:
40069
diff
changeset
|
168 |
else |
27f2a45b0aab
more robust handling of "remote_" vs. non-"remote_" provers
blanchet
parents:
40069
diff
changeset
|
169 |
let val remote_name = remote_prefix ^ name in |
41727
ab3f6d76fb23
available_provers ~> supported_provers (for clarity)
blanchet
parents:
41472
diff
changeset
|
170 |
if is_prover_supported ctxt remote_name then SOME remote_name else NONE |
40072
27f2a45b0aab
more robust handling of "remote_" vs. non-"remote_" provers
blanchet
parents:
40069
diff
changeset
|
171 |
end |
27f2a45b0aab
more robust handling of "remote_" vs. non-"remote_" provers
blanchet
parents:
40069
diff
changeset
|
172 |
|
27f2a45b0aab
more robust handling of "remote_" vs. non-"remote_" provers
blanchet
parents:
40069
diff
changeset
|
173 |
fun remotify_prover_if_not_installed ctxt name = |
41727
ab3f6d76fb23
available_provers ~> supported_provers (for clarity)
blanchet
parents:
41472
diff
changeset
|
174 |
if is_prover_supported ctxt name andalso is_prover_installed ctxt name then |
40941
a3e6f8634a11
replace "smt" prover with specific SMT solvers, e.g. "z3" -- whatever the SMT module gives us
blanchet
parents:
40931
diff
changeset
|
175 |
SOME name |
a3e6f8634a11
replace "smt" prover with specific SMT solvers, e.g. "z3" -- whatever the SMT module gives us
blanchet
parents:
40931
diff
changeset
|
176 |
else |
41727
ab3f6d76fb23
available_provers ~> supported_provers (for clarity)
blanchet
parents:
41472
diff
changeset
|
177 |
remotify_prover_if_supported_and_not_already_remote ctxt name |
40072
27f2a45b0aab
more robust handling of "remote_" vs. non-"remote_" provers
blanchet
parents:
40069
diff
changeset
|
178 |
|
43009
f58bab6be6a9
reintroduced Waldmeister but limit the number of remote threads created
blanchet
parents:
43008
diff
changeset
|
179 |
fun avoid_too_many_threads _ _ [] = [] |
f58bab6be6a9
reintroduced Waldmeister but limit the number of remote threads created
blanchet
parents:
43008
diff
changeset
|
180 |
| avoid_too_many_threads _ (0, 0) _ = [] |
f58bab6be6a9
reintroduced Waldmeister but limit the number of remote threads created
blanchet
parents:
43008
diff
changeset
|
181 |
| avoid_too_many_threads ctxt (0, max_remote) provers = |
f58bab6be6a9
reintroduced Waldmeister but limit the number of remote threads created
blanchet
parents:
43008
diff
changeset
|
182 |
provers |
f58bab6be6a9
reintroduced Waldmeister but limit the number of remote threads created
blanchet
parents:
43008
diff
changeset
|
183 |
|> map_filter (remotify_prover_if_supported_and_not_already_remote ctxt) |
f58bab6be6a9
reintroduced Waldmeister but limit the number of remote threads created
blanchet
parents:
43008
diff
changeset
|
184 |
|> take max_remote |
f58bab6be6a9
reintroduced Waldmeister but limit the number of remote threads created
blanchet
parents:
43008
diff
changeset
|
185 |
| avoid_too_many_threads _ (max_local, 0) provers = |
f58bab6be6a9
reintroduced Waldmeister but limit the number of remote threads created
blanchet
parents:
43008
diff
changeset
|
186 |
provers |
f58bab6be6a9
reintroduced Waldmeister but limit the number of remote threads created
blanchet
parents:
43008
diff
changeset
|
187 |
|> filter_out (String.isPrefix remote_prefix) |
f58bab6be6a9
reintroduced Waldmeister but limit the number of remote threads created
blanchet
parents:
43008
diff
changeset
|
188 |
|> take max_local |
f58bab6be6a9
reintroduced Waldmeister but limit the number of remote threads created
blanchet
parents:
43008
diff
changeset
|
189 |
| avoid_too_many_threads ctxt max_local_and_remote (prover :: provers) = |
f58bab6be6a9
reintroduced Waldmeister but limit the number of remote threads created
blanchet
parents:
43008
diff
changeset
|
190 |
let |
f58bab6be6a9
reintroduced Waldmeister but limit the number of remote threads created
blanchet
parents:
43008
diff
changeset
|
191 |
val max_local_and_remote = |
f58bab6be6a9
reintroduced Waldmeister but limit the number of remote threads created
blanchet
parents:
43008
diff
changeset
|
192 |
max_local_and_remote |
f58bab6be6a9
reintroduced Waldmeister but limit the number of remote threads created
blanchet
parents:
43008
diff
changeset
|
193 |
|> (if String.isPrefix remote_prefix prover then apsnd else apfst) |
f58bab6be6a9
reintroduced Waldmeister but limit the number of remote threads created
blanchet
parents:
43008
diff
changeset
|
194 |
(Integer.add ~1) |
f58bab6be6a9
reintroduced Waldmeister but limit the number of remote threads created
blanchet
parents:
43008
diff
changeset
|
195 |
in prover :: avoid_too_many_threads ctxt max_local_and_remote provers end |
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39335
diff
changeset
|
196 |
|
43009
f58bab6be6a9
reintroduced Waldmeister but limit the number of remote threads created
blanchet
parents:
43008
diff
changeset
|
197 |
val max_default_remote_threads = 4 |
42688
097a61baeca9
smoother handling of ! and ? in type system names
blanchet
parents:
42613
diff
changeset
|
198 |
|
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39335
diff
changeset
|
199 |
(* The first ATP of the list is used by Auto Sledgehammer. Because of the low |
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39335
diff
changeset
|
200 |
timeout, it makes sense to put SPASS first. *) |
40069 | 201 |
fun default_provers_param_value ctxt = |
43009
f58bab6be6a9
reintroduced Waldmeister but limit the number of remote threads created
blanchet
parents:
43008
diff
changeset
|
202 |
[spassN, eN, vampireN, SMT_Solver.solver_name_of ctxt, sine_eN, waldmeisterN] |
40941
a3e6f8634a11
replace "smt" prover with specific SMT solvers, e.g. "z3" -- whatever the SMT module gives us
blanchet
parents:
40931
diff
changeset
|
203 |
|> map_filter (remotify_prover_if_not_installed ctxt) |
43009
f58bab6be6a9
reintroduced Waldmeister but limit the number of remote threads created
blanchet
parents:
43008
diff
changeset
|
204 |
|> avoid_too_many_threads ctxt (Multithreading.max_threads_value (), |
f58bab6be6a9
reintroduced Waldmeister but limit the number of remote threads created
blanchet
parents:
43008
diff
changeset
|
205 |
max_default_remote_threads) |
42776 | 206 |
|> implode_param |
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39335
diff
changeset
|
207 |
|
36140
08b2a7ecb6c3
fixed handling of "sledgehammer_params" that get a default value from Isabelle menu;
blanchet
parents:
36064
diff
changeset
|
208 |
val set_default_raw_param = Data.map o AList.update (op =) o unalias_raw_param |
40069 | 209 |
fun default_raw_params ctxt = |
42361 | 210 |
let val thy = Proof_Context.theory_of ctxt in |
40069 | 211 |
Data.get thy |
212 |
|> fold (AList.default (op =)) |
|
213 |
[("provers", [case !provers of |
|
214 |
"" => default_provers_param_value ctxt |
|
215 |
| s => s]), |
|
216 |
("timeout", let val timeout = !timeout in |
|
217 |
[if timeout <= 0 then "none" |
|
40341
03156257040f
standardize on seconds for Nitpick and Sledgehammer timeouts
blanchet
parents:
40181
diff
changeset
|
218 |
else string_of_int timeout] |
40069 | 219 |
end)] |
220 |
end |
|
35963 | 221 |
|
222 |
val infinity_time_in_secs = 60 * 60 * 24 * 365 |
|
223 |
val the_timeout = the_default (Time.fromSeconds infinity_time_in_secs) |
|
35866
513074557e06
move the Sledgehammer Isar commands together into one file;
blanchet
parents:
diff
changeset
|
224 |
|
43021 | 225 |
fun extract_params mode default_params override_params = |
35963 | 226 |
let |
36140
08b2a7ecb6c3
fixed handling of "sledgehammer_params" that get a default value from Isabelle menu;
blanchet
parents:
36064
diff
changeset
|
227 |
val override_params = map unalias_raw_param override_params |
35963 | 228 |
val raw_params = rev override_params @ rev default_params |
42776 | 229 |
val lookup = Option.map implode_param o AList.lookup (op =) raw_params |
35963 | 230 |
val lookup_string = the_default "" o lookup |
231 |
fun general_lookup_bool option default_value name = |
|
232 |
case lookup name of |
|
35970
3d41a2a490f0
revert debugging output that shouldn't have been submitted in the first place
blanchet
parents:
35966
diff
changeset
|
233 |
SOME s => parse_bool_option option name s |
35963 | 234 |
| NONE => default_value |
235 |
val lookup_bool = the o general_lookup_bool false (SOME false) |
|
236 |
fun lookup_time name = |
|
39318 | 237 |
case lookup name of |
238 |
SOME s => parse_time_option name s |
|
239 |
| NONE => NONE |
|
35966
f8c738abaed8
honor the newly introduced Sledgehammer parameters and fixed the parsing;
blanchet
parents:
35965
diff
changeset
|
240 |
fun lookup_int name = |
35963 | 241 |
case lookup name of |
35966
f8c738abaed8
honor the newly introduced Sledgehammer parameters and fixed the parsing;
blanchet
parents:
35965
diff
changeset
|
242 |
NONE => 0 |
f8c738abaed8
honor the newly introduced Sledgehammer parameters and fixed the parsing;
blanchet
parents:
35965
diff
changeset
|
243 |
| SOME s => case Int.fromString s of |
f8c738abaed8
honor the newly introduced Sledgehammer parameters and fixed the parsing;
blanchet
parents:
35965
diff
changeset
|
244 |
SOME n => n |
f8c738abaed8
honor the newly introduced Sledgehammer parameters and fixed the parsing;
blanchet
parents:
35965
diff
changeset
|
245 |
| NONE => error ("Parameter " ^ quote name ^ |
f8c738abaed8
honor the newly introduced Sledgehammer parameters and fixed the parsing;
blanchet
parents:
35965
diff
changeset
|
246 |
" must be assigned an integer value.") |
40343
4521d56aef63
use floating-point numbers for Sledgehammer's "thresholds" option rather than percentages;
blanchet
parents:
40341
diff
changeset
|
247 |
fun lookup_real_pair name = |
38745
ad577fd62ee4
reorganize options regarding to the relevance threshold and decay
blanchet
parents:
38744
diff
changeset
|
248 |
case lookup name of |
40343
4521d56aef63
use floating-point numbers for Sledgehammer's "thresholds" option rather than percentages;
blanchet
parents:
40341
diff
changeset
|
249 |
NONE => (0.0, 0.0) |
4521d56aef63
use floating-point numbers for Sledgehammer's "thresholds" option rather than percentages;
blanchet
parents:
40341
diff
changeset
|
250 |
| SOME s => case s |> space_explode " " |> map Real.fromString of |
4521d56aef63
use floating-point numbers for Sledgehammer's "thresholds" option rather than percentages;
blanchet
parents:
40341
diff
changeset
|
251 |
[SOME r1, SOME r2] => (r1, r2) |
38745
ad577fd62ee4
reorganize options regarding to the relevance threshold and decay
blanchet
parents:
38744
diff
changeset
|
252 |
| _ => error ("Parameter " ^ quote name ^ |
40343
4521d56aef63
use floating-point numbers for Sledgehammer's "thresholds" option rather than percentages;
blanchet
parents:
40341
diff
changeset
|
253 |
"must be assigned a pair of floating-point \ |
4521d56aef63
use floating-point numbers for Sledgehammer's "thresholds" option rather than percentages;
blanchet
parents:
40341
diff
changeset
|
254 |
\values (e.g., \"0.6 0.95\")") |
43064
b6e61d22fa61
made "explicit_apply" smarter -- no need to force explicit applications in minimizer on all constants, better do it more fine granularly
blanchet
parents:
43057
diff
changeset
|
255 |
fun lookup_option lookup' name = |
38589
b03f8fe043ec
added "max_relevant_per_iter" option to Sledgehammer
blanchet
parents:
38282
diff
changeset
|
256 |
case lookup name of |
b03f8fe043ec
added "max_relevant_per_iter" option to Sledgehammer
blanchet
parents:
38282
diff
changeset
|
257 |
SOME "smart" => NONE |
43064
b6e61d22fa61
made "explicit_apply" smarter -- no need to force explicit applications in minimizer on all constants, better do it more fine granularly
blanchet
parents:
43057
diff
changeset
|
258 |
| _ => SOME (lookup' name) |
43021 | 259 |
val debug = mode <> Auto_Try andalso lookup_bool "debug" |
260 |
val verbose = debug orelse (mode <> Auto_Try andalso lookup_bool "verbose") |
|
36143
6490319b1703
added "overlord" option (to get easy access to output files for debugging) + systematically use "raw_goal" rather than an inconsistent mixture
blanchet
parents:
36142
diff
changeset
|
261 |
val overlord = lookup_bool "overlord" |
42995
e23f61546cf0
always run Sledgehammer synchronously in the jEdit interface (until the multithreading support for Proof General is ported)
blanchet
parents:
42944
diff
changeset
|
262 |
val blocking = |
43021 | 263 |
Isabelle_Process.is_active () orelse mode <> Normal orelse debug orelse |
42995
e23f61546cf0
always run Sledgehammer synchronously in the jEdit interface (until the multithreading support for Proof General is ported)
blanchet
parents:
42944
diff
changeset
|
264 |
lookup_bool "blocking" |
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39335
diff
changeset
|
265 |
val provers = lookup_string "provers" |> space_explode " " |
43021 | 266 |
|> mode = Auto_Try ? single o hd |
43626
a867ebb12209
renamed "type_sys" to "type_enc", which is more accurate
blanchet
parents:
43572
diff
changeset
|
267 |
val type_enc = |
43021 | 268 |
if mode = Auto_Try then |
43569
b342cd125533
removed "full_types" option from Sledgehammer, now that virtually sound encodings are used as the default anyway
blanchet
parents:
43353
diff
changeset
|
269 |
NONE |
43626
a867ebb12209
renamed "type_sys" to "type_enc", which is more accurate
blanchet
parents:
43572
diff
changeset
|
270 |
else case lookup_string "type_enc" of |
43569
b342cd125533
removed "full_types" option from Sledgehammer, now that virtually sound encodings are used as the default anyway
blanchet
parents:
43353
diff
changeset
|
271 |
"smart" => NONE |
43626
a867ebb12209
renamed "type_sys" to "type_enc", which is more accurate
blanchet
parents:
43572
diff
changeset
|
272 |
| s => SOME (type_enc_from_string s) |
43572
ae612a423dad
added "sound" option to force Sledgehammer to be pedantically sound
blanchet
parents:
43569
diff
changeset
|
273 |
val sound = mode = Auto_Try orelse lookup_bool "sound" |
42180
a6c141925a8a
added monomorphization option to Sledgehammer ATPs -- this looks promising but is still off by default
blanchet
parents:
41727
diff
changeset
|
274 |
val relevance_thresholds = lookup_real_pair "relevance_thresholds" |
43064
b6e61d22fa61
made "explicit_apply" smarter -- no need to force explicit applications in minimizer on all constants, better do it more fine granularly
blanchet
parents:
43057
diff
changeset
|
275 |
val max_relevant = lookup_option lookup_int "max_relevant" |
42724
4d6bcf846759
added "max_mono_instances" option to Sledgehammer and renamed old "monomorphize_limit" option
blanchet
parents:
42688
diff
changeset
|
276 |
val max_mono_iters = lookup_int "max_mono_iters" |
42740
31334a7b109d
renamed "max_mono_instances" to "max_new_mono_instances" and changed its semantics accordingly
blanchet
parents:
42736
diff
changeset
|
277 |
val max_new_mono_instances = lookup_int "max_new_mono_instances" |
35963 | 278 |
val isar_proof = lookup_bool "isar_proof" |
36924 | 279 |
val isar_shrink_factor = Int.max (1, lookup_int "isar_shrink_factor") |
43021 | 280 |
val slicing = mode <> Auto_Try andalso lookup_bool "slicing" |
281 |
val timeout = |
|
282 |
(if mode = Auto_Try then NONE else lookup_time "timeout") |> the_timeout |
|
43015
21b6baec55b1
renamed "metis_timeout" to "preplay_timeout" and continued implementation
blanchet
parents:
43013
diff
changeset
|
283 |
val preplay_timeout = |
43021 | 284 |
if mode = Auto_Try then Time.zeroTime |
43015
21b6baec55b1
renamed "metis_timeout" to "preplay_timeout" and continued implementation
blanchet
parents:
43013
diff
changeset
|
285 |
else lookup_time "preplay_timeout" |> the_timeout |
38985
162bbbea4e4d
added "expect" feature of Nitpick to Sledgehammer, for regression testing
blanchet
parents:
38982
diff
changeset
|
286 |
val expect = lookup_string "expect" |
35963 | 287 |
in |
41208
1b28c43a7074
make "debug" imply "blocking", since in blocking mode the exceptions flow through and are more instructive
blanchet
parents:
41153
diff
changeset
|
288 |
{debug = debug, verbose = verbose, overlord = overlord, blocking = blocking, |
42180
a6c141925a8a
added monomorphization option to Sledgehammer ATPs -- this looks promising but is still off by default
blanchet
parents:
41727
diff
changeset
|
289 |
provers = provers, relevance_thresholds = relevance_thresholds, |
42724
4d6bcf846759
added "max_mono_instances" option to Sledgehammer and renamed old "monomorphize_limit" option
blanchet
parents:
42688
diff
changeset
|
290 |
max_relevant = max_relevant, max_mono_iters = max_mono_iters, |
43626
a867ebb12209
renamed "type_sys" to "type_enc", which is more accurate
blanchet
parents:
43572
diff
changeset
|
291 |
max_new_mono_instances = max_new_mono_instances, type_enc = type_enc, |
43572
ae612a423dad
added "sound" option to force Sledgehammer to be pedantically sound
blanchet
parents:
43569
diff
changeset
|
292 |
sound = sound, isar_proof = isar_proof, |
ae612a423dad
added "sound" option to force Sledgehammer to be pedantically sound
blanchet
parents:
43569
diff
changeset
|
293 |
isar_shrink_factor = isar_shrink_factor, slicing = slicing, |
ae612a423dad
added "sound" option to force Sledgehammer to be pedantically sound
blanchet
parents:
43569
diff
changeset
|
294 |
timeout = timeout, preplay_timeout = preplay_timeout, expect = expect} |
35963 | 295 |
end |
35866
513074557e06
move the Sledgehammer Isar commands together into one file;
blanchet
parents:
diff
changeset
|
296 |
|
43021 | 297 |
fun get_params mode ctxt = extract_params mode (default_raw_params ctxt) |
298 |
fun default_params thy = get_params Normal thy o map (apsnd single) |
|
35866
513074557e06
move the Sledgehammer Isar commands together into one file;
blanchet
parents:
diff
changeset
|
299 |
|
36373
66af0a49de39
move some sledgehammer stuff out of "atp_manager.ML"
blanchet
parents:
36371
diff
changeset
|
300 |
(* Sledgehammer the given subgoal *) |
66af0a49de39
move some sledgehammer stuff out of "atp_manager.ML"
blanchet
parents:
36371
diff
changeset
|
301 |
|
43051 | 302 |
val default_minimize_prover = Metis_Tactics.metisN |
303 |
||
36281
dbbf4d5d584d
pass relevant options from "sledgehammer" to "sledgehammer minimize";
blanchet
parents:
36235
diff
changeset
|
304 |
val is_raw_param_relevant_for_minimize = |
dbbf4d5d584d
pass relevant options from "sledgehammer" to "sledgehammer minimize";
blanchet
parents:
36235
diff
changeset
|
305 |
member (op =) params_for_minimize o fst o unalias_raw_param |
dbbf4d5d584d
pass relevant options from "sledgehammer" to "sledgehammer minimize";
blanchet
parents:
36235
diff
changeset
|
306 |
fun string_for_raw_param (key, values) = |
42776 | 307 |
key ^ (case implode_param values of "" => "" | value => " = " ^ value) |
36281
dbbf4d5d584d
pass relevant options from "sledgehammer" to "sledgehammer minimize";
blanchet
parents:
36235
diff
changeset
|
308 |
|
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39335
diff
changeset
|
309 |
fun minimize_command override_params i prover_name fact_names = |
43057 | 310 |
let |
311 |
val params = |
|
312 |
override_params |
|
313 |
|> filter is_raw_param_relevant_for_minimize |
|
314 |
|> map string_for_raw_param |
|
315 |
|> (if prover_name = default_minimize_prover then I else cons prover_name) |
|
316 |
|> space_implode ", " |
|
317 |
in |
|
318 |
sledgehammerN ^ " " ^ minN ^ |
|
319 |
(if params = "" then "" else enclose " [" "]" params) ^ |
|
320 |
" (" ^ space_implode " " fact_names ^ ")" ^ |
|
321 |
(if i = 1 then "" else " " ^ string_of_int i) |
|
322 |
end |
|
36281
dbbf4d5d584d
pass relevant options from "sledgehammer" to "sledgehammer minimize";
blanchet
parents:
36235
diff
changeset
|
323 |
|
35966
f8c738abaed8
honor the newly introduced Sledgehammer parameters and fixed the parsing;
blanchet
parents:
35965
diff
changeset
|
324 |
fun hammer_away override_params subcommand opt_i relevance_override state = |
35963 | 325 |
let |
40069 | 326 |
val ctxt = Proof.context_of state |
41258
73401632a80c
convenient syntax for setting provers -- useful for debugging, not for general consumption and hence not documented
blanchet
parents:
41208
diff
changeset
|
327 |
val override_params = |
73401632a80c
convenient syntax for setting provers -- useful for debugging, not for general consumption and hence not documented
blanchet
parents:
41208
diff
changeset
|
328 |
override_params |> map (check_and_repair_raw_param ctxt) |
35965
0fce6db7babd
added a syntax for specifying facts to Sledgehammer;
blanchet
parents:
35963
diff
changeset
|
329 |
in |
0fce6db7babd
added a syntax for specifying facts to Sledgehammer;
blanchet
parents:
35963
diff
changeset
|
330 |
if subcommand = runN then |
36281
dbbf4d5d584d
pass relevant options from "sledgehammer" to "sledgehammer minimize";
blanchet
parents:
36235
diff
changeset
|
331 |
let val i = the_default 1 opt_i in |
43021 | 332 |
run_sledgehammer (get_params Normal ctxt override_params) Normal i |
39318 | 333 |
relevance_override (minimize_command override_params i) |
334 |
state |
|
335 |
|> K () |
|
36281
dbbf4d5d584d
pass relevant options from "sledgehammer" to "sledgehammer minimize";
blanchet
parents:
36235
diff
changeset
|
336 |
end |
43008
bb212c2ad238
renamed "minimize" to "min" to make Sledgehammer output a little bit more concise
blanchet
parents:
42997
diff
changeset
|
337 |
else if subcommand = minN then |
43051 | 338 |
run_minimize (get_params Minimize ctxt |
339 |
(("provers", [default_minimize_prover]) :: |
|
340 |
override_params)) |
|
43021 | 341 |
(the_default 1 opt_i) (#add relevance_override) state |
35965
0fce6db7babd
added a syntax for specifying facts to Sledgehammer;
blanchet
parents:
35963
diff
changeset
|
342 |
else if subcommand = messagesN then |
0fce6db7babd
added a syntax for specifying facts to Sledgehammer;
blanchet
parents:
35963
diff
changeset
|
343 |
messages opt_i |
41727
ab3f6d76fb23
available_provers ~> supported_provers (for clarity)
blanchet
parents:
41472
diff
changeset
|
344 |
else if subcommand = supported_proversN then |
ab3f6d76fb23
available_provers ~> supported_provers (for clarity)
blanchet
parents:
41472
diff
changeset
|
345 |
supported_provers ctxt |
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39335
diff
changeset
|
346 |
else if subcommand = running_proversN then |
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39335
diff
changeset
|
347 |
running_provers () |
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39335
diff
changeset
|
348 |
else if subcommand = kill_proversN then |
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39335
diff
changeset
|
349 |
kill_provers () |
35965
0fce6db7babd
added a syntax for specifying facts to Sledgehammer;
blanchet
parents:
35963
diff
changeset
|
350 |
else if subcommand = refresh_tptpN then |
0fce6db7babd
added a syntax for specifying facts to Sledgehammer;
blanchet
parents:
35963
diff
changeset
|
351 |
refresh_systems_on_tptp () |
0fce6db7babd
added a syntax for specifying facts to Sledgehammer;
blanchet
parents:
35963
diff
changeset
|
352 |
else |
0fce6db7babd
added a syntax for specifying facts to Sledgehammer;
blanchet
parents:
35963
diff
changeset
|
353 |
error ("Unknown subcommand: " ^ quote subcommand ^ ".") |
0fce6db7babd
added a syntax for specifying facts to Sledgehammer;
blanchet
parents:
35963
diff
changeset
|
354 |
end |
35963 | 355 |
|
35966
f8c738abaed8
honor the newly introduced Sledgehammer parameters and fixed the parsing;
blanchet
parents:
35965
diff
changeset
|
356 |
fun sledgehammer_trans (((subcommand, params), relevance_override), opt_i) = |
f8c738abaed8
honor the newly introduced Sledgehammer parameters and fixed the parsing;
blanchet
parents:
35965
diff
changeset
|
357 |
Toplevel.keep (hammer_away params subcommand opt_i relevance_override |
f8c738abaed8
honor the newly introduced Sledgehammer parameters and fixed the parsing;
blanchet
parents:
35965
diff
changeset
|
358 |
o Toplevel.proof_of) |
35963 | 359 |
|
42776 | 360 |
fun string_for_raw_param (name, value) = name ^ " = " ^ implode_param value |
35963 | 361 |
|
35965
0fce6db7babd
added a syntax for specifying facts to Sledgehammer;
blanchet
parents:
35963
diff
changeset
|
362 |
fun sledgehammer_params_trans params = |
35963 | 363 |
Toplevel.theory |
35965
0fce6db7babd
added a syntax for specifying facts to Sledgehammer;
blanchet
parents:
35963
diff
changeset
|
364 |
(fold set_default_raw_param params |
39318 | 365 |
#> tap (fn thy => |
42361 | 366 |
let val ctxt = Proof_Context.init_global thy in |
40069 | 367 |
writeln ("Default parameters for Sledgehammer:\n" ^ |
368 |
(case default_raw_params ctxt |> rev of |
|
369 |
[] => "none" |
|
370 |
| params => |
|
41258
73401632a80c
convenient syntax for setting provers -- useful for debugging, not for general consumption and hence not documented
blanchet
parents:
41208
diff
changeset
|
371 |
params |> map (check_and_repair_raw_param ctxt) |
73401632a80c
convenient syntax for setting provers -- useful for debugging, not for general consumption and hence not documented
blanchet
parents:
41208
diff
changeset
|
372 |
|> map string_for_raw_param |
73401632a80c
convenient syntax for setting provers -- useful for debugging, not for general consumption and hence not documented
blanchet
parents:
41208
diff
changeset
|
373 |
|> sort_strings |> cat_lines)) |
40069 | 374 |
end)) |
35963 | 375 |
|
42776 | 376 |
val parse_key = |
377 |
Scan.repeat1 (Parse.typ_group || Parse.$$$ "?" || Parse.$$$ "!") |
|
43100 | 378 |
>> implode_param |
42581
398fff2c6b8f
use ! for mildly unsound and !! for very unsound encodings
blanchet
parents:
42579
diff
changeset
|
379 |
val parse_value = |
42589
9f7c48463645
restructured type systems some more -- the old naming schemes had "argshg diff |less" and "tagshg diff |less" as equivalent and didn't support a monomorphic version of "tags"
blanchet
parents:
42581
diff
changeset
|
380 |
Scan.repeat1 (Parse.xname || Parse.float_number || Parse.$$$ "?" |
42581
398fff2c6b8f
use ! for mildly unsound and !! for very unsound encodings
blanchet
parents:
42579
diff
changeset
|
381 |
|| Parse.$$$ "!") |
36960
01594f816e3a
prefer structure Keyword, Parse, Parse_Spec, Outer_Syntax;
wenzelm
parents:
36924
diff
changeset
|
382 |
val parse_param = parse_key -- Scan.optional (Parse.$$$ "=" |-- parse_value) [] |
01594f816e3a
prefer structure Keyword, Parse, Parse_Spec, Outer_Syntax;
wenzelm
parents:
36924
diff
changeset
|
383 |
val parse_params = Scan.optional (Args.bracks (Parse.list parse_param)) [] |
35965
0fce6db7babd
added a syntax for specifying facts to Sledgehammer;
blanchet
parents:
35963
diff
changeset
|
384 |
val parse_fact_refs = |
38996 | 385 |
Scan.repeat1 (Scan.unless (Parse.name -- Args.colon) Parse_Spec.xthm) |
35966
f8c738abaed8
honor the newly introduced Sledgehammer parameters and fixed the parsing;
blanchet
parents:
35965
diff
changeset
|
386 |
val parse_relevance_chunk = |
39318 | 387 |
(Args.add |-- Args.colon |-- parse_fact_refs >> add_relevance_override) |
388 |
|| (Args.del |-- Args.colon |-- parse_fact_refs >> del_relevance_override) |
|
36188 | 389 |
|| (parse_fact_refs >> only_relevance_override) |
35966
f8c738abaed8
honor the newly introduced Sledgehammer parameters and fixed the parsing;
blanchet
parents:
35965
diff
changeset
|
390 |
val parse_relevance_override = |
36188 | 391 |
Scan.optional (Args.parens (Scan.repeat parse_relevance_chunk |
392 |
>> merge_relevance_overrides)) |
|
39318 | 393 |
no_relevance_override |
35963 | 394 |
val parse_sledgehammer_command = |
37399
34f080a12063
proper polymorphic Skolemization of uncached facts + synchronization of caching and relevance filter
blanchet
parents:
37344
diff
changeset
|
395 |
(Scan.optional Parse.short_ident runN -- parse_params |
34f080a12063
proper polymorphic Skolemization of uncached facts + synchronization of caching and relevance filter
blanchet
parents:
37344
diff
changeset
|
396 |
-- parse_relevance_override -- Scan.option Parse.nat) #>> sledgehammer_trans |
35963 | 397 |
val parse_sledgehammer_params_command = |
398 |
parse_params #>> sledgehammer_params_trans |
|
399 |
||
400 |
val _ = |
|
36960
01594f816e3a
prefer structure Keyword, Parse, Parse_Spec, Outer_Syntax;
wenzelm
parents:
36924
diff
changeset
|
401 |
Outer_Syntax.improper_command sledgehammerN |
01594f816e3a
prefer structure Keyword, Parse, Parse_Spec, Outer_Syntax;
wenzelm
parents:
36924
diff
changeset
|
402 |
"search for first-order proof using automatic theorem provers" Keyword.diag |
36394
1a48d18449d8
move "neg_clausify" method and "clausify" attribute to "sledgehammer_isar.ML"
blanchet
parents:
36378
diff
changeset
|
403 |
parse_sledgehammer_command |
35963 | 404 |
val _ = |
36960
01594f816e3a
prefer structure Keyword, Parse, Parse_Spec, Outer_Syntax;
wenzelm
parents:
36924
diff
changeset
|
405 |
Outer_Syntax.command sledgehammer_paramsN |
01594f816e3a
prefer structure Keyword, Parse, Parse_Spec, Outer_Syntax;
wenzelm
parents:
36924
diff
changeset
|
406 |
"set and display the default parameters for Sledgehammer" Keyword.thy_decl |
36394
1a48d18449d8
move "neg_clausify" method and "clausify" attribute to "sledgehammer_isar.ML"
blanchet
parents:
36378
diff
changeset
|
407 |
parse_sledgehammer_params_command |
1a48d18449d8
move "neg_clausify" method and "clausify" attribute to "sledgehammer_isar.ML"
blanchet
parents:
36378
diff
changeset
|
408 |
|
43020
abb5d1f907e4
added "try" command, to launch Solve Direct, Quickcheck, Nitpick, Sledgehammer, and Try Methods
blanchet
parents:
43018
diff
changeset
|
409 |
fun try_sledgehammer auto state = |
abb5d1f907e4
added "try" command, to launch Solve Direct, Quickcheck, Nitpick, Sledgehammer, and Try Methods
blanchet
parents:
43018
diff
changeset
|
410 |
let |
abb5d1f907e4
added "try" command, to launch Solve Direct, Quickcheck, Nitpick, Sledgehammer, and Try Methods
blanchet
parents:
43018
diff
changeset
|
411 |
val ctxt = Proof.context_of state |
43021 | 412 |
val mode = if auto then Auto_Try else Try |
43020
abb5d1f907e4
added "try" command, to launch Solve Direct, Quickcheck, Nitpick, Sledgehammer, and Try Methods
blanchet
parents:
43018
diff
changeset
|
413 |
val i = 1 |
abb5d1f907e4
added "try" command, to launch Solve Direct, Quickcheck, Nitpick, Sledgehammer, and Try Methods
blanchet
parents:
43018
diff
changeset
|
414 |
in |
43021 | 415 |
run_sledgehammer (get_params mode ctxt []) mode i no_relevance_override |
43020
abb5d1f907e4
added "try" command, to launch Solve Direct, Quickcheck, Nitpick, Sledgehammer, and Try Methods
blanchet
parents:
43018
diff
changeset
|
416 |
(minimize_command [] i) state |
40931 | 417 |
end |
39318 | 418 |
|
43024
58150aa44941
prioritize try and auto try's tools, with fast ones first, with a slight preference for provers vs. counterexample generators
blanchet
parents:
43021
diff
changeset
|
419 |
val setup = Try.register_tool (sledgehammerN, (40, auto, try_sledgehammer)) |
39318 | 420 |
|
35866
513074557e06
move the Sledgehammer Isar commands together into one file;
blanchet
parents:
diff
changeset
|
421 |
end; |