src/HOL/Tools/Sledgehammer/sledgehammer.ML
author blanchet
Mon, 09 Aug 2010 14:08:30 +0200
changeset 38290 581a402a80f0
parent 38282 319c59682c51
child 38455 131f7c46cf2c
permissions -rw-r--r--
prevent ATP thread for staying around for 1 minute if an exception occurred earlier; this is a workaround for what could be a misfeature of "Async_Manager", which I'd rather not touch
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
38021
e024504943d1 rename "ATP_Manager" ML module to "Sledgehammer";
blanchet
parents: 38020
diff changeset
     1
(*  Title:      HOL/Tools/Sledgehammer/sledgehammer.ML
28477
9339d4dcec8b version of sledgehammer using threads instead of processes, misc cleanup;
wenzelm
parents:
diff changeset
     2
    Author:     Fabian Immler, TU Muenchen
32996
d2e48879e65a removed disjunctive group cancellation -- provers run independently;
wenzelm
parents: 32995
diff changeset
     3
    Author:     Makarius
35969
c9565298df9e added support for Sledgehammer parameters;
blanchet
parents: 35867
diff changeset
     4
    Author:     Jasmin Blanchette, TU Muenchen
28477
9339d4dcec8b version of sledgehammer using threads instead of processes, misc cleanup;
wenzelm
parents:
diff changeset
     5
38021
e024504943d1 rename "ATP_Manager" ML module to "Sledgehammer";
blanchet
parents: 38020
diff changeset
     6
Sledgehammer's heart.
28477
9339d4dcec8b version of sledgehammer using threads instead of processes, misc cleanup;
wenzelm
parents:
diff changeset
     7
*)
9339d4dcec8b version of sledgehammer using threads instead of processes, misc cleanup;
wenzelm
parents:
diff changeset
     8
38021
e024504943d1 rename "ATP_Manager" ML module to "Sledgehammer";
blanchet
parents: 38020
diff changeset
     9
signature SLEDGEHAMMER =
28477
9339d4dcec8b version of sledgehammer using threads instead of processes, misc cleanup;
wenzelm
parents:
diff changeset
    10
sig
38023
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
    11
  type failure = ATP_Systems.failure
35969
c9565298df9e added support for Sledgehammer parameters;
blanchet
parents: 35867
diff changeset
    12
  type relevance_override = Sledgehammer_Fact_Filter.relevance_override
36281
dbbf4d5d584d pass relevant options from "sledgehammer" to "sledgehammer minimize";
blanchet
parents: 36235
diff changeset
    13
  type minimize_command = Sledgehammer_Proof_Reconstruct.minimize_command
35969
c9565298df9e added support for Sledgehammer parameters;
blanchet
parents: 35867
diff changeset
    14
  type params =
c9565298df9e added support for Sledgehammer parameters;
blanchet
parents: 35867
diff changeset
    15
    {debug: bool,
c9565298df9e added support for Sledgehammer parameters;
blanchet
parents: 35867
diff changeset
    16
     verbose: bool,
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: 36064
diff changeset
    17
     overlord: bool,
35969
c9565298df9e added support for Sledgehammer parameters;
blanchet
parents: 35867
diff changeset
    18
     atps: string list,
c9565298df9e added support for Sledgehammer parameters;
blanchet
parents: 35867
diff changeset
    19
     full_types: bool,
36235
61159615a0c5 added "explicit_apply" option to Sledgehammer, to control whether an explicit apply function should be used as much or as little as possible (replaces a previous global variable)
blanchet
parents: 36231
diff changeset
    20
     explicit_apply: bool,
35969
c9565298df9e added support for Sledgehammer parameters;
blanchet
parents: 35867
diff changeset
    21
     relevance_threshold: real,
36922
12f87df9c1a5 renamed two Sledgehammer options
blanchet
parents: 36489
diff changeset
    22
     relevance_convergence: real,
36220
f3655a3ae1ab rename Sledgehammer "theory_const" option to "theory_relevant", now that I understand better what it does
blanchet
parents: 36184
diff changeset
    23
     theory_relevant: bool option,
36922
12f87df9c1a5 renamed two Sledgehammer options
blanchet
parents: 36489
diff changeset
    24
     defs_relevant: bool,
35969
c9565298df9e added support for Sledgehammer parameters;
blanchet
parents: 35867
diff changeset
    25
     isar_proof: bool,
36924
ff01d3ae9ad4 renamed options
blanchet
parents: 36922
diff changeset
    26
     isar_shrink_factor: int,
35969
c9565298df9e added support for Sledgehammer parameters;
blanchet
parents: 35867
diff changeset
    27
     timeout: Time.time,
c9565298df9e added support for Sledgehammer parameters;
blanchet
parents: 35867
diff changeset
    28
     minimize_timeout: Time.time}
35867
16279c4c7a33 move all ATP setup code into ATP_Wrapper
blanchet
parents: 35866
diff changeset
    29
  type problem =
35969
c9565298df9e added support for Sledgehammer parameters;
blanchet
parents: 35867
diff changeset
    30
    {subgoal: int,
c9565298df9e added support for Sledgehammer parameters;
blanchet
parents: 35867
diff changeset
    31
     goal: Proof.context * (thm list * thm),
c9565298df9e added support for Sledgehammer parameters;
blanchet
parents: 35867
diff changeset
    32
     relevance_override: relevance_override,
38084
e2aac207d13b "axiom_clauses" -> "axioms" (these are no longer clauses)
blanchet
parents: 38083
diff changeset
    33
     axioms: (string * thm) list option}
35867
16279c4c7a33 move all ATP setup code into ATP_Wrapper
blanchet
parents: 35866
diff changeset
    34
  type prover_result =
36370
a4f601daa175 centralized ATP-specific error handling in "atp_wrapper.ML"
blanchet
parents: 36369
diff changeset
    35
    {outcome: failure option,
35969
c9565298df9e added support for Sledgehammer parameters;
blanchet
parents: 35867
diff changeset
    36
     message: string,
37926
e6ff246c0cdb renamings + only need second component of name pool to reconstruct proofs
blanchet
parents: 37627
diff changeset
    37
     pool: string Symtab.table,
38015
b30c3c2e1030 implemented "sublinear" minimization algorithm
blanchet
parents: 38002
diff changeset
    38
     used_thm_names: string list,
35969
c9565298df9e added support for Sledgehammer parameters;
blanchet
parents: 35867
diff changeset
    39
     atp_run_time_in_msecs: int,
36369
d2cd0d04b8e6 handle ATP proof delimiters in a cleaner, more extensible fashion
blanchet
parents: 36289
diff changeset
    40
     output: string,
35969
c9565298df9e added support for Sledgehammer parameters;
blanchet
parents: 35867
diff changeset
    41
     proof: string,
38282
319c59682c51 move Sledgehammer's HOL -> FOL translation to separate file (sledgehammer_translate.ML)
blanchet
parents: 38277
diff changeset
    42
     axiom_names: string Vector.vector,
38083
c4b57f68ddb3 remove the "extra_clauses" business introduced in 19a5f1c8a844;
blanchet
parents: 38061
diff changeset
    43
     conjecture_shape: int list list}
38100
e458a0dd3dc1 use "explicit_apply" in the minimizer whenever it might make a difference to prevent freak failures;
blanchet
parents: 38098
diff changeset
    44
  type prover = params -> minimize_command -> problem -> prover_result
35867
16279c4c7a33 move all ATP setup code into ATP_Wrapper
blanchet
parents: 35866
diff changeset
    45
38023
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
    46
  val dest_dir : string Config.T
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
    47
  val problem_prefix : string Config.T
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
    48
  val measure_runtime : bool Config.T
35969
c9565298df9e added support for Sledgehammer parameters;
blanchet
parents: 35867
diff changeset
    49
  val kill_atps: unit -> unit
c9565298df9e added support for Sledgehammer parameters;
blanchet
parents: 35867
diff changeset
    50
  val running_atps: unit -> unit
29112
f2b45eea6dac added 'atp_messages' command, which displays recent messages synchronously;
wenzelm
parents: 28835
diff changeset
    51
  val messages: int option -> unit
38023
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
    52
  val get_prover_fun : theory -> string -> prover
38044
463177795c49 minor refactoring
blanchet
parents: 38040
diff changeset
    53
  val run_sledgehammer :
463177795c49 minor refactoring
blanchet
parents: 38040
diff changeset
    54
    params -> int -> relevance_override -> (string -> minimize_command)
463177795c49 minor refactoring
blanchet
parents: 38040
diff changeset
    55
    -> Proof.state -> unit
38023
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
    56
  val setup : theory -> theory
28477
9339d4dcec8b version of sledgehammer using threads instead of processes, misc cleanup;
wenzelm
parents:
diff changeset
    57
end;
9339d4dcec8b version of sledgehammer using threads instead of processes, misc cleanup;
wenzelm
parents:
diff changeset
    58
38021
e024504943d1 rename "ATP_Manager" ML module to "Sledgehammer";
blanchet
parents: 38020
diff changeset
    59
structure Sledgehammer : SLEDGEHAMMER =
28477
9339d4dcec8b version of sledgehammer using threads instead of processes, misc cleanup;
wenzelm
parents:
diff changeset
    60
struct
9339d4dcec8b version of sledgehammer using threads instead of processes, misc cleanup;
wenzelm
parents:
diff changeset
    61
38028
22dcaec5fa77 minor refactoring
blanchet
parents: 38023
diff changeset
    62
open ATP_Problem
22dcaec5fa77 minor refactoring
blanchet
parents: 38023
diff changeset
    63
open ATP_Systems
37578
9367cb36b1c4 renamed "Sledgehammer_FOL_Clauses" to "Metis_Clauses", so that Metis doesn't depend on Sledgehammer
blanchet
parents: 37577
diff changeset
    64
open Metis_Clauses
38023
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
    65
open Sledgehammer_Util
36063
cdc6855a6387 make Sledgehammer output "by" vs. "apply", "qed" vs. "next", and any necessary "prefer"
blanchet
parents: 36059
diff changeset
    66
open Sledgehammer_Fact_Filter
38282
319c59682c51 move Sledgehammer's HOL -> FOL translation to separate file (sledgehammer_translate.ML)
blanchet
parents: 38277
diff changeset
    67
open Sledgehammer_Translate
36063
cdc6855a6387 make Sledgehammer output "by" vs. "apply", "qed" vs. "next", and any necessary "prefer"
blanchet
parents: 36059
diff changeset
    68
open Sledgehammer_Proof_Reconstruct
37583
9ce2451647d5 factored non-ATP specific code from "ATP_Manager" out, so that it can be reused for the LEO-II integration
blanchet
parents: 37581
diff changeset
    69
38023
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
    70
37583
9ce2451647d5 factored non-ATP specific code from "ATP_Manager" out, so that it can be reused for the LEO-II integration
blanchet
parents: 37581
diff changeset
    71
(** The Sledgehammer **)
9ce2451647d5 factored non-ATP specific code from "ATP_Manager" out, so that it can be reused for the LEO-II integration
blanchet
parents: 37581
diff changeset
    72
38102
019a49759829 fix bug in the newly introduced "bound concealing" code
blanchet
parents: 38100
diff changeset
    73
(* Identifier to distinguish Sledgehammer from other tools using
019a49759829 fix bug in the newly introduced "bound concealing" code
blanchet
parents: 38100
diff changeset
    74
   "Async_Manager". *)
37585
c2ed8112ce57 multiplexing
blanchet
parents: 37584
diff changeset
    75
val das_Tool = "Sledgehammer"
c2ed8112ce57 multiplexing
blanchet
parents: 37584
diff changeset
    76
c2ed8112ce57 multiplexing
blanchet
parents: 37584
diff changeset
    77
fun kill_atps () = Async_Manager.kill_threads das_Tool "ATPs"
c2ed8112ce57 multiplexing
blanchet
parents: 37584
diff changeset
    78
fun running_atps () = Async_Manager.running_threads das_Tool "ATPs"
c2ed8112ce57 multiplexing
blanchet
parents: 37584
diff changeset
    79
val messages = Async_Manager.thread_messages das_Tool "ATP"
35969
c9565298df9e added support for Sledgehammer parameters;
blanchet
parents: 35867
diff changeset
    80
36281
dbbf4d5d584d pass relevant options from "sledgehammer" to "sledgehammer minimize";
blanchet
parents: 36235
diff changeset
    81
(** problems, results, provers, etc. **)
35969
c9565298df9e added support for Sledgehammer parameters;
blanchet
parents: 35867
diff changeset
    82
c9565298df9e added support for Sledgehammer parameters;
blanchet
parents: 35867
diff changeset
    83
type params =
c9565298df9e added support for Sledgehammer parameters;
blanchet
parents: 35867
diff changeset
    84
  {debug: bool,
c9565298df9e added support for Sledgehammer parameters;
blanchet
parents: 35867
diff changeset
    85
   verbose: bool,
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: 36064
diff changeset
    86
   overlord: bool,
35969
c9565298df9e added support for Sledgehammer parameters;
blanchet
parents: 35867
diff changeset
    87
   atps: string list,
c9565298df9e added support for Sledgehammer parameters;
blanchet
parents: 35867
diff changeset
    88
   full_types: bool,
36235
61159615a0c5 added "explicit_apply" option to Sledgehammer, to control whether an explicit apply function should be used as much or as little as possible (replaces a previous global variable)
blanchet
parents: 36231
diff changeset
    89
   explicit_apply: bool,
35969
c9565298df9e added support for Sledgehammer parameters;
blanchet
parents: 35867
diff changeset
    90
   relevance_threshold: real,
36922
12f87df9c1a5 renamed two Sledgehammer options
blanchet
parents: 36489
diff changeset
    91
   relevance_convergence: real,
36220
f3655a3ae1ab rename Sledgehammer "theory_const" option to "theory_relevant", now that I understand better what it does
blanchet
parents: 36184
diff changeset
    92
   theory_relevant: bool option,
36922
12f87df9c1a5 renamed two Sledgehammer options
blanchet
parents: 36489
diff changeset
    93
   defs_relevant: bool,
35969
c9565298df9e added support for Sledgehammer parameters;
blanchet
parents: 35867
diff changeset
    94
   isar_proof: bool,
36924
ff01d3ae9ad4 renamed options
blanchet
parents: 36922
diff changeset
    95
   isar_shrink_factor: int,
35969
c9565298df9e added support for Sledgehammer parameters;
blanchet
parents: 35867
diff changeset
    96
   timeout: Time.time,
c9565298df9e added support for Sledgehammer parameters;
blanchet
parents: 35867
diff changeset
    97
   minimize_timeout: Time.time}
35867
16279c4c7a33 move all ATP setup code into ATP_Wrapper
blanchet
parents: 35866
diff changeset
    98
16279c4c7a33 move all ATP setup code into ATP_Wrapper
blanchet
parents: 35866
diff changeset
    99
type problem =
35969
c9565298df9e added support for Sledgehammer parameters;
blanchet
parents: 35867
diff changeset
   100
  {subgoal: int,
c9565298df9e added support for Sledgehammer parameters;
blanchet
parents: 35867
diff changeset
   101
   goal: Proof.context * (thm list * thm),
c9565298df9e added support for Sledgehammer parameters;
blanchet
parents: 35867
diff changeset
   102
   relevance_override: relevance_override,
38084
e2aac207d13b "axiom_clauses" -> "axioms" (these are no longer clauses)
blanchet
parents: 38083
diff changeset
   103
   axioms: (string * thm) list option}
35867
16279c4c7a33 move all ATP setup code into ATP_Wrapper
blanchet
parents: 35866
diff changeset
   104
16279c4c7a33 move all ATP setup code into ATP_Wrapper
blanchet
parents: 35866
diff changeset
   105
type prover_result =
36370
a4f601daa175 centralized ATP-specific error handling in "atp_wrapper.ML"
blanchet
parents: 36369
diff changeset
   106
  {outcome: failure option,
35969
c9565298df9e added support for Sledgehammer parameters;
blanchet
parents: 35867
diff changeset
   107
   message: string,
37926
e6ff246c0cdb renamings + only need second component of name pool to reconstruct proofs
blanchet
parents: 37627
diff changeset
   108
   pool: string Symtab.table,
38015
b30c3c2e1030 implemented "sublinear" minimization algorithm
blanchet
parents: 38002
diff changeset
   109
   used_thm_names: string list,
35969
c9565298df9e added support for Sledgehammer parameters;
blanchet
parents: 35867
diff changeset
   110
   atp_run_time_in_msecs: int,
36369
d2cd0d04b8e6 handle ATP proof delimiters in a cleaner, more extensible fashion
blanchet
parents: 36289
diff changeset
   111
   output: string,
35969
c9565298df9e added support for Sledgehammer parameters;
blanchet
parents: 35867
diff changeset
   112
   proof: string,
38282
319c59682c51 move Sledgehammer's HOL -> FOL translation to separate file (sledgehammer_translate.ML)
blanchet
parents: 38277
diff changeset
   113
   axiom_names: string Vector.vector,
38083
c4b57f68ddb3 remove the "extra_clauses" business introduced in 19a5f1c8a844;
blanchet
parents: 38061
diff changeset
   114
   conjecture_shape: int list list}
35867
16279c4c7a33 move all ATP setup code into ATP_Wrapper
blanchet
parents: 35866
diff changeset
   115
38100
e458a0dd3dc1 use "explicit_apply" in the minimizer whenever it might make a difference to prevent freak failures;
blanchet
parents: 38098
diff changeset
   116
type prover = params -> minimize_command -> problem -> prover_result
35867
16279c4c7a33 move all ATP setup code into ATP_Wrapper
blanchet
parents: 35866
diff changeset
   117
38023
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   118
(* configuration attributes *)
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   119
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   120
val (dest_dir, dest_dir_setup) = Attrib.config_string "atp_dest_dir" (K "");
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   121
  (*Empty string means create files in Isabelle's temporary files directory.*)
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   122
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   123
val (problem_prefix, problem_prefix_setup) =
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   124
  Attrib.config_string "atp_problem_prefix" (K "prob");
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   125
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   126
val (measure_runtime, measure_runtime_setup) =
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   127
  Attrib.config_bool "atp_measure_runtime" (K false);
28484
4ed9239b09c1 misc simplifcation and tuning;
wenzelm
parents: 28478
diff changeset
   128
38023
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   129
fun with_path cleanup after f path =
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   130
  Exn.capture f path
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   131
  |> tap (fn _ => cleanup path)
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   132
  |> Exn.release
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   133
  |> tap (after path)
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   134
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   135
(* Splits by the first possible of a list of delimiters. *)
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   136
fun extract_proof delims output =
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   137
  case pairself (find_first (fn s => String.isSubstring s output))
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   138
                (ListPair.unzip delims) of
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   139
    (SOME begin_delim, SOME end_delim) =>
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   140
    (output |> first_field begin_delim |> the |> snd
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   141
            |> first_field end_delim |> the |> fst
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   142
            |> first_field "\n" |> the |> snd
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   143
     handle Option.Option => "")
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   144
  | _ => ""
28484
4ed9239b09c1 misc simplifcation and tuning;
wenzelm
parents: 28478
diff changeset
   145
38023
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   146
fun extract_proof_and_outcome complete res_code proof_delims known_failures
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   147
                              output =
38061
685d1f0f75b3 handle Perl and "libwww-perl" failures more gracefully, giving the user some clues about what goes on
blanchet
parents: 38044
diff changeset
   148
  case known_failure_in_output output known_failures of
685d1f0f75b3 handle Perl and "libwww-perl" failures more gracefully, giving the user some clues about what goes on
blanchet
parents: 38044
diff changeset
   149
    NONE => (case extract_proof proof_delims output of
685d1f0f75b3 handle Perl and "libwww-perl" failures more gracefully, giving the user some clues about what goes on
blanchet
parents: 38044
diff changeset
   150
             "" => ("", SOME MalformedOutput)
38023
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   151
           | proof => if res_code = 0 then (proof, NONE)
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   152
                      else ("", SOME UnknownError))
38061
685d1f0f75b3 handle Perl and "libwww-perl" failures more gracefully, giving the user some clues about what goes on
blanchet
parents: 38044
diff changeset
   153
  | SOME failure =>
38023
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   154
    ("", SOME (if failure = IncompleteUnprovable andalso complete then
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   155
                 Unprovable
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   156
               else
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   157
                 failure))
28582
c269a3045fdf info: back to plain printing;
wenzelm
parents: 28571
diff changeset
   158
38023
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   159
fun extract_clause_sequence output =
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   160
  let
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   161
    val tokens_of = String.tokens (not o Char.isAlphaNum)
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   162
    fun extract_num ("clause" :: (ss as _ :: _)) =
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   163
    Int.fromString (List.last ss)
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   164
      | extract_num _ = NONE
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   165
  in output |> split_lines |> map_filter (extract_num o tokens_of) end
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   166
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   167
val set_ClauseFormulaRelationN = "set_ClauseFormulaRelation"
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   168
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   169
val parse_clause_formula_pair =
38105
373351f5f834 don't choke on synonyms when parsing SPASS's Flotter output + renamings;
blanchet
parents: 38102
diff changeset
   170
  $$ "(" |-- scan_integer --| $$ "," -- Symbol.scan_id
373351f5f834 don't choke on synonyms when parsing SPASS's Flotter output + renamings;
blanchet
parents: 38102
diff changeset
   171
  --| Scan.repeat ($$ "," |-- Symbol.scan_id) --| $$ ")"
38023
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   172
  --| Scan.option ($$ ",")
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   173
val parse_clause_formula_relation =
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   174
  Scan.this_string set_ClauseFormulaRelationN |-- $$ "("
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   175
  |-- Scan.repeat parse_clause_formula_pair
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   176
val extract_clause_formula_relation =
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   177
  Substring.full
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   178
  #> Substring.position set_ClauseFormulaRelationN
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   179
  #> snd #> Substring.string #> strip_spaces #> explode
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   180
  #> parse_clause_formula_relation #> fst
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   181
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   182
fun repair_conjecture_shape_and_theorem_names output conjecture_shape
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   183
                                              thm_names =
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   184
  if String.isSubstring set_ClauseFormulaRelationN output then
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   185
    (* This is a hack required for keeping track of axioms after they have been
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   186
       clausified by SPASS's Flotter tool. The "SPASS_TPTP" script is also part
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   187
       of this hack. *)
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   188
    let
38040
174568533593 fix bug in the SPASS Flotter hack, when a conjecture FOF is translated to several CNF clauses
blanchet
parents: 38039
diff changeset
   189
      val j0 = hd (hd conjecture_shape)
38023
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   190
      val seq = extract_clause_sequence output
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   191
      val name_map = extract_clause_formula_relation output
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   192
      fun renumber_conjecture j =
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   193
        AList.find (op =) name_map (conjecture_prefix ^ Int.toString (j - j0))
38040
174568533593 fix bug in the SPASS Flotter hack, when a conjecture FOF is translated to several CNF clauses
blanchet
parents: 38039
diff changeset
   194
        |> map (fn s => find_index (curry (op =) s) seq + 1)
38023
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   195
    in
38040
174568533593 fix bug in the SPASS Flotter hack, when a conjecture FOF is translated to several CNF clauses
blanchet
parents: 38039
diff changeset
   196
      (conjecture_shape |> map (maps renumber_conjecture),
38105
373351f5f834 don't choke on synonyms when parsing SPASS's Flotter output + renamings;
blanchet
parents: 38102
diff changeset
   197
       seq |> map (fn j => case j |> AList.lookup (op =) name_map |> the
373351f5f834 don't choke on synonyms when parsing SPASS's Flotter output + renamings;
blanchet
parents: 38102
diff changeset
   198
                                  |> try (unprefix axiom_prefix) of
38023
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   199
                             SOME s' => undo_ascii_of s'
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   200
                           | NONE => "")
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   201
           |> Vector.fromList)
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   202
    end
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   203
  else
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   204
    (conjecture_shape, thm_names)
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   205
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   206
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   207
(* generic TPTP-based provers *)
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   208
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   209
fun prover_fun name
38092
81a003f7de0d speed up the minimizer by using the time taken for the first iteration as a timeout for the following iterations, and fix a subtle bug in "string_for_failure"
blanchet
parents: 38091
diff changeset
   210
        {exec, required_execs, arguments, proof_delims, known_failures,
81a003f7de0d speed up the minimizer by using the time taken for the first iteration as a timeout for the following iterations, and fix a subtle bug in "string_for_failure"
blanchet
parents: 38091
diff changeset
   211
         max_new_relevant_facts_per_iter, prefers_theory_relevant,
81a003f7de0d speed up the minimizer by using the time taken for the first iteration as a timeout for the following iterations, and fix a subtle bug in "string_for_failure"
blanchet
parents: 38091
diff changeset
   212
         explicit_forall}
38023
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   213
        ({debug, overlord, full_types, explicit_apply, relevance_threshold,
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   214
          relevance_convergence, theory_relevant, defs_relevant, isar_proof,
38100
e458a0dd3dc1 use "explicit_apply" in the minimizer whenever it might make a difference to prevent freak failures;
blanchet
parents: 38098
diff changeset
   215
          isar_shrink_factor, timeout, ...} : params)
e458a0dd3dc1 use "explicit_apply" in the minimizer whenever it might make a difference to prevent freak failures;
blanchet
parents: 38098
diff changeset
   216
        minimize_command
38084
e2aac207d13b "axiom_clauses" -> "axioms" (these are no longer clauses)
blanchet
parents: 38083
diff changeset
   217
        ({subgoal, goal, relevance_override, axioms} : problem) =
38023
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   218
  let
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   219
    val (ctxt, (_, th)) = goal;
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   220
    val thy = ProofContext.theory_of ctxt
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   221
    val (params, hyp_ts, concl_t) = strip_subgoal th subgoal
38084
e2aac207d13b "axiom_clauses" -> "axioms" (these are no longer clauses)
blanchet
parents: 38083
diff changeset
   222
    val the_axioms =
e2aac207d13b "axiom_clauses" -> "axioms" (these are no longer clauses)
blanchet
parents: 38083
diff changeset
   223
      case axioms of
38083
c4b57f68ddb3 remove the "extra_clauses" business introduced in 19a5f1c8a844;
blanchet
parents: 38061
diff changeset
   224
        SOME axioms => axioms
38023
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   225
      | NONE => relevant_facts full_types relevance_threshold
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   226
                    relevance_convergence defs_relevant
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   227
                    max_new_relevant_facts_per_iter
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   228
                    (the_default prefers_theory_relevant theory_relevant)
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   229
                    relevance_override goal hyp_ts concl_t
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   230
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   231
    (* path to unique problem file *)
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   232
    val the_dest_dir = if overlord then getenv "ISABELLE_HOME_USER"
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   233
                       else Config.get ctxt dest_dir;
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   234
    val the_problem_prefix = Config.get ctxt problem_prefix;
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   235
    fun prob_pathname nr =
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   236
      let
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   237
        val probfile =
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   238
          Path.basic ((if overlord then "prob_" ^ name
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   239
                       else the_problem_prefix ^ serial_string ())
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   240
                      ^ "_" ^ string_of_int nr)
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   241
      in
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   242
        if the_dest_dir = "" then File.tmp_path probfile
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   243
        else if File.exists (Path.explode the_dest_dir)
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   244
        then Path.append (Path.explode the_dest_dir) probfile
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   245
        else error ("No such directory: " ^ the_dest_dir ^ ".")
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   246
      end;
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   247
38092
81a003f7de0d speed up the minimizer by using the time taken for the first iteration as a timeout for the following iterations, and fix a subtle bug in "string_for_failure"
blanchet
parents: 38091
diff changeset
   248
    val command = Path.explode (getenv (fst exec) ^ "/" ^ snd exec)
38023
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   249
    (* write out problem file and call prover *)
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   250
    fun command_line complete probfile =
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   251
      let
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   252
        val core = File.shell_path command ^ " " ^ arguments complete timeout ^
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   253
                   " " ^ File.shell_path probfile
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   254
      in
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   255
        (if Config.get ctxt measure_runtime then
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   256
           "TIMEFORMAT='%3U'; { time " ^ core ^ " ; }"
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   257
         else
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   258
           "exec " ^ core) ^ " 2>&1"
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   259
      end
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   260
    fun split_time s =
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   261
      let
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   262
        val split = String.tokens (fn c => str c = "\n");
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   263
        val (output, t) = s |> split |> split_last |> apfst cat_lines;
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   264
        fun as_num f = f >> (fst o read_int);
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   265
        val num = as_num (Scan.many1 Symbol.is_ascii_digit);
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   266
        val digit = Scan.one Symbol.is_ascii_digit;
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   267
        val num3 = as_num (digit ::: digit ::: (digit >> single));
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   268
        val time = num --| Scan.$$ "." -- num3 >> (fn (a, b) => a * 1000 + b);
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   269
        val as_time = the_default 0 o Scan.read Symbol.stopper time o explode;
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   270
      in (output, as_time t) end;
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   271
    fun run_on probfile =
38092
81a003f7de0d speed up the minimizer by using the time taken for the first iteration as a timeout for the following iterations, and fix a subtle bug in "string_for_failure"
blanchet
parents: 38091
diff changeset
   272
      case filter (curry (op =) "" o getenv o fst) (exec :: required_execs) of
38032
54448f5d151f improve detection of installed SPASS
blanchet
parents: 38028
diff changeset
   273
        (home_var, _) :: _ =>
38023
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   274
        error ("The environment variable " ^ quote home_var ^ " is not set.")
38032
54448f5d151f improve detection of installed SPASS
blanchet
parents: 38028
diff changeset
   275
      | [] =>
54448f5d151f improve detection of installed SPASS
blanchet
parents: 38028
diff changeset
   276
        if File.exists command then
54448f5d151f improve detection of installed SPASS
blanchet
parents: 38028
diff changeset
   277
          let
54448f5d151f improve detection of installed SPASS
blanchet
parents: 38028
diff changeset
   278
            fun do_run complete =
54448f5d151f improve detection of installed SPASS
blanchet
parents: 38028
diff changeset
   279
              let
54448f5d151f improve detection of installed SPASS
blanchet
parents: 38028
diff changeset
   280
                val command = command_line complete probfile
54448f5d151f improve detection of installed SPASS
blanchet
parents: 38028
diff changeset
   281
                val ((output, msecs), res_code) =
54448f5d151f improve detection of installed SPASS
blanchet
parents: 38028
diff changeset
   282
                  bash_output command
54448f5d151f improve detection of installed SPASS
blanchet
parents: 38028
diff changeset
   283
                  |>> (if overlord then
54448f5d151f improve detection of installed SPASS
blanchet
parents: 38028
diff changeset
   284
                         prefix ("% " ^ command ^ "\n% " ^ timestamp () ^ "\n")
54448f5d151f improve detection of installed SPASS
blanchet
parents: 38028
diff changeset
   285
                       else
54448f5d151f improve detection of installed SPASS
blanchet
parents: 38028
diff changeset
   286
                         I)
54448f5d151f improve detection of installed SPASS
blanchet
parents: 38028
diff changeset
   287
                  |>> (if Config.get ctxt measure_runtime then split_time
54448f5d151f improve detection of installed SPASS
blanchet
parents: 38028
diff changeset
   288
                       else rpair 0)
54448f5d151f improve detection of installed SPASS
blanchet
parents: 38028
diff changeset
   289
                val (proof, outcome) =
54448f5d151f improve detection of installed SPASS
blanchet
parents: 38028
diff changeset
   290
                  extract_proof_and_outcome complete res_code proof_delims
54448f5d151f improve detection of installed SPASS
blanchet
parents: 38028
diff changeset
   291
                                            known_failures output
54448f5d151f improve detection of installed SPASS
blanchet
parents: 38028
diff changeset
   292
              in (output, msecs, proof, outcome) end
54448f5d151f improve detection of installed SPASS
blanchet
parents: 38028
diff changeset
   293
            val readable_names = debug andalso overlord
38282
319c59682c51 move Sledgehammer's HOL -> FOL translation to separate file (sledgehammer_translate.ML)
blanchet
parents: 38277
diff changeset
   294
            val (problem, pool, conjecture_offset, axiom_names) =
319c59682c51 move Sledgehammer's HOL -> FOL translation to separate file (sledgehammer_translate.ML)
blanchet
parents: 38277
diff changeset
   295
              prepare_problem ctxt readable_names explicit_forall full_types
319c59682c51 move Sledgehammer's HOL -> FOL translation to separate file (sledgehammer_translate.ML)
blanchet
parents: 38277
diff changeset
   296
                              explicit_apply hyp_ts concl_t the_axioms
319c59682c51 move Sledgehammer's HOL -> FOL translation to separate file (sledgehammer_translate.ML)
blanchet
parents: 38277
diff changeset
   297
            val _ = File.write_list probfile (strings_for_tptp_problem problem)
38032
54448f5d151f improve detection of installed SPASS
blanchet
parents: 38028
diff changeset
   298
            val conjecture_shape =
54448f5d151f improve detection of installed SPASS
blanchet
parents: 38028
diff changeset
   299
              conjecture_offset + 1 upto conjecture_offset + length hyp_ts + 1
38040
174568533593 fix bug in the SPASS Flotter hack, when a conjecture FOF is translated to several CNF clauses
blanchet
parents: 38039
diff changeset
   300
              |> map single
38032
54448f5d151f improve detection of installed SPASS
blanchet
parents: 38028
diff changeset
   301
            val result =
54448f5d151f improve detection of installed SPASS
blanchet
parents: 38028
diff changeset
   302
              do_run false
54448f5d151f improve detection of installed SPASS
blanchet
parents: 38028
diff changeset
   303
              |> (fn (_, msecs0, _, SOME _) =>
54448f5d151f improve detection of installed SPASS
blanchet
parents: 38028
diff changeset
   304
                     do_run true
54448f5d151f improve detection of installed SPASS
blanchet
parents: 38028
diff changeset
   305
                     |> (fn (output, msecs, proof, outcome) =>
54448f5d151f improve detection of installed SPASS
blanchet
parents: 38028
diff changeset
   306
                            (output, msecs0 + msecs, proof, outcome))
54448f5d151f improve detection of installed SPASS
blanchet
parents: 38028
diff changeset
   307
                   | result => result)
38282
319c59682c51 move Sledgehammer's HOL -> FOL translation to separate file (sledgehammer_translate.ML)
blanchet
parents: 38277
diff changeset
   308
          in ((pool, conjecture_shape, axiom_names), result) end
38032
54448f5d151f improve detection of installed SPASS
blanchet
parents: 38028
diff changeset
   309
        else
54448f5d151f improve detection of installed SPASS
blanchet
parents: 38028
diff changeset
   310
          error ("Bad executable: " ^ Path.implode command ^ ".")
38023
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   311
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   312
    (* If the problem file has not been exported, remove it; otherwise, export
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   313
       the proof file too. *)
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   314
    fun cleanup probfile =
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   315
      if the_dest_dir = "" then try File.rm probfile else NONE
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   316
    fun export probfile (_, (output, _, _, _)) =
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   317
      if the_dest_dir = "" then
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   318
        ()
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   319
      else
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   320
        File.write (Path.explode (Path.implode probfile ^ "_proof")) output
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   321
38282
319c59682c51 move Sledgehammer's HOL -> FOL translation to separate file (sledgehammer_translate.ML)
blanchet
parents: 38277
diff changeset
   322
    val ((pool, conjecture_shape, axiom_names),
319c59682c51 move Sledgehammer's HOL -> FOL translation to separate file (sledgehammer_translate.ML)
blanchet
parents: 38277
diff changeset
   323
         (output, msecs, proof, outcome)) =
38023
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   324
      with_path cleanup export run_on (prob_pathname subgoal)
38282
319c59682c51 move Sledgehammer's HOL -> FOL translation to separate file (sledgehammer_translate.ML)
blanchet
parents: 38277
diff changeset
   325
    val (conjecture_shape, axiom_names) =
38023
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   326
      repair_conjecture_shape_and_theorem_names output conjecture_shape
38282
319c59682c51 move Sledgehammer's HOL -> FOL translation to separate file (sledgehammer_translate.ML)
blanchet
parents: 38277
diff changeset
   327
                                                axiom_names
38023
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   328
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   329
    val (message, used_thm_names) =
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   330
      case outcome of
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   331
        NONE =>
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   332
        proof_text isar_proof
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   333
            (pool, debug, isar_shrink_factor, ctxt, conjecture_shape)
38282
319c59682c51 move Sledgehammer's HOL -> FOL translation to separate file (sledgehammer_translate.ML)
blanchet
parents: 38277
diff changeset
   334
            (full_types, minimize_command, proof, axiom_names, th, subgoal)
38023
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   335
      | SOME failure => (string_for_failure failure ^ "\n", [])
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   336
  in
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   337
    {outcome = outcome, message = message, pool = pool,
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   338
     used_thm_names = used_thm_names, atp_run_time_in_msecs = msecs,
38282
319c59682c51 move Sledgehammer's HOL -> FOL translation to separate file (sledgehammer_translate.ML)
blanchet
parents: 38277
diff changeset
   339
     output = output, proof = proof, axiom_names = axiom_names,
38083
c4b57f68ddb3 remove the "extra_clauses" business introduced in 19a5f1c8a844;
blanchet
parents: 38061
diff changeset
   340
     conjecture_shape = conjecture_shape}
38023
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   341
  end
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   342
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   343
fun get_prover_fun thy name = prover_fun name (get_prover thy name)
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   344
37584
2e289dc13615 factor out thread creation
blanchet
parents: 37583
diff changeset
   345
fun start_prover_thread (params as {verbose, full_types, timeout, ...}) i n
2e289dc13615 factor out thread creation
blanchet
parents: 37583
diff changeset
   346
                        relevance_override minimize_command proof_state name =
36379
20ef039bccff make "ATP_Manager.get_prover" a total function, since we always want to show the same error text
blanchet
parents: 36373
diff changeset
   347
  let
38023
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   348
    val thy = Proof.theory_of proof_state
37584
2e289dc13615 factor out thread creation
blanchet
parents: 37583
diff changeset
   349
    val birth_time = Time.now ()
2e289dc13615 factor out thread creation
blanchet
parents: 37583
diff changeset
   350
    val death_time = Time.+ (birth_time, timeout)
38023
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   351
    val prover = get_prover_fun thy name
36379
20ef039bccff make "ATP_Manager.get_prover" a total function, since we always want to show the same error text
blanchet
parents: 36373
diff changeset
   352
    val {context = ctxt, facts, goal} = Proof.goal proof_state;
20ef039bccff make "ATP_Manager.get_prover" a total function, since we always want to show the same error text
blanchet
parents: 36373
diff changeset
   353
    val desc =
20ef039bccff make "ATP_Manager.get_prover" a total function, since we always want to show the same error text
blanchet
parents: 36373
diff changeset
   354
      "ATP " ^ quote name ^ " for subgoal " ^ string_of_int i ^ ":\n" ^
36392
c00c57850eb7 cosmetics: rename internal functions
blanchet
parents: 36383
diff changeset
   355
      Syntax.string_of_term ctxt (Thm.term_of (Thm.cprem_of goal i));
37584
2e289dc13615 factor out thread creation
blanchet
parents: 37583
diff changeset
   356
  in
37585
c2ed8112ce57 multiplexing
blanchet
parents: 37584
diff changeset
   357
    Async_Manager.launch das_Tool verbose birth_time death_time desc
37584
2e289dc13615 factor out thread creation
blanchet
parents: 37583
diff changeset
   358
        (fn () =>
2e289dc13615 factor out thread creation
blanchet
parents: 37583
diff changeset
   359
            let
2e289dc13615 factor out thread creation
blanchet
parents: 37583
diff changeset
   360
              val problem =
2e289dc13615 factor out thread creation
blanchet
parents: 37583
diff changeset
   361
                {subgoal = i, goal = (ctxt, (facts, goal)),
38084
e2aac207d13b "axiom_clauses" -> "axioms" (these are no longer clauses)
blanchet
parents: 38083
diff changeset
   362
                 relevance_override = relevance_override, axioms = NONE}
37584
2e289dc13615 factor out thread creation
blanchet
parents: 37583
diff changeset
   363
            in
38100
e458a0dd3dc1 use "explicit_apply" in the minimizer whenever it might make a difference to prevent freak failures;
blanchet
parents: 38098
diff changeset
   364
              prover params (minimize_command name) problem |> #message
37994
b04307085a09 make TPTP generator accept full first-order formulas
blanchet
parents: 37926
diff changeset
   365
              handle ERROR message => "Error: " ^ message ^ "\n"
38290
581a402a80f0 prevent ATP thread for staying around for 1 minute if an exception occurred earlier;
blanchet
parents: 38282
diff changeset
   366
                   | exn => "Internal error: \n" ^ ML_Compiler.exn_message exn ^
581a402a80f0 prevent ATP thread for staying around for 1 minute if an exception occurred earlier;
blanchet
parents: 38282
diff changeset
   367
                            "\n"
37584
2e289dc13615 factor out thread creation
blanchet
parents: 37583
diff changeset
   368
            end)
2e289dc13615 factor out thread creation
blanchet
parents: 37583
diff changeset
   369
  end
28582
c269a3045fdf info: back to plain printing;
wenzelm
parents: 28571
diff changeset
   370
38044
463177795c49 minor refactoring
blanchet
parents: 38040
diff changeset
   371
fun run_sledgehammer {atps = [], ...} _ _ _ _ = error "No ATP is set."
463177795c49 minor refactoring
blanchet
parents: 38040
diff changeset
   372
  | run_sledgehammer (params as {atps, ...}) i relevance_override
463177795c49 minor refactoring
blanchet
parents: 38040
diff changeset
   373
                     minimize_command state =
463177795c49 minor refactoring
blanchet
parents: 38040
diff changeset
   374
    case subgoal_count state of
463177795c49 minor refactoring
blanchet
parents: 38040
diff changeset
   375
      0 => priority "No subgoal!"
463177795c49 minor refactoring
blanchet
parents: 38040
diff changeset
   376
    | n =>
463177795c49 minor refactoring
blanchet
parents: 38040
diff changeset
   377
      let
463177795c49 minor refactoring
blanchet
parents: 38040
diff changeset
   378
        val _ = kill_atps ()
463177795c49 minor refactoring
blanchet
parents: 38040
diff changeset
   379
        val _ = priority "Sledgehammering..."
463177795c49 minor refactoring
blanchet
parents: 38040
diff changeset
   380
        val _ = app (start_prover_thread params i n relevance_override
463177795c49 minor refactoring
blanchet
parents: 38040
diff changeset
   381
                                         minimize_command state) atps
463177795c49 minor refactoring
blanchet
parents: 38040
diff changeset
   382
      in () end
463177795c49 minor refactoring
blanchet
parents: 38040
diff changeset
   383
38023
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   384
val setup =
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   385
  dest_dir_setup
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   386
  #> problem_prefix_setup
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   387
  #> measure_runtime_setup
962b0a7f544b more refactoring
blanchet
parents: 38021
diff changeset
   388
28582
c269a3045fdf info: back to plain printing;
wenzelm
parents: 28571
diff changeset
   389
end;