src/HOL/Tools/Sledgehammer/sledgehammer_run.ML
author blanchet
Thu, 21 Apr 2011 18:39:22 +0200
changeset 43314 724e612ba248
parent 43232 23f352990944
child 43315 8e5438dc70bb
permissions -rw-r--r--
implemented general slicing for ATPs, especially E 1.2w and above
blanchet@41335
     1
(*  Title:      HOL/Tools/Sledgehammer/sledgehammer_run.ML
wenzelm@28477
     2
    Author:     Fabian Immler, TU Muenchen
wenzelm@32996
     3
    Author:     Makarius
blanchet@35967
     4
    Author:     Jasmin Blanchette, TU Muenchen
wenzelm@28477
     5
blanchet@38255
     6
Sledgehammer's heart.
wenzelm@28477
     7
*)
wenzelm@28477
     8
blanchet@41335
     9
signature SLEDGEHAMMER_RUN =
wenzelm@28477
    10
sig
blanchet@39232
    11
  type relevance_override = Sledgehammer_Filter.relevance_override
blanchet@40249
    12
  type minimize_command = Sledgehammer_ATP_Reconstruct.minimize_command
blanchet@41335
    13
  type params = Sledgehammer_Provers.params
blanchet@41511
    14
  type prover = Sledgehammer_Provers.prover
blanchet@39733
    15
blanchet@41583
    16
  val auto_minimize_min_facts : int Unsynchronized.ref
blanchet@43314
    17
  val get_minimizing_prover : Proof.context -> bool -> bool -> string -> prover
blanchet@38290
    18
  val run_sledgehammer :
blanchet@43314
    19
    params -> bool -> bool -> int -> relevance_override
blanchet@43314
    20
    -> (string -> minimize_command) -> Proof.state -> bool * Proof.state
wenzelm@28477
    21
end;
wenzelm@28477
    22
blanchet@41335
    23
structure Sledgehammer_Run : SLEDGEHAMMER_RUN =
wenzelm@28477
    24
struct
wenzelm@28477
    25
blanchet@38257
    26
open Sledgehammer_Util
blanchet@39232
    27
open Sledgehammer_Filter
blanchet@40249
    28
open Sledgehammer_ATP_Translate
blanchet@41335
    29
open Sledgehammer_Provers
blanchet@41339
    30
open Sledgehammer_Minimize
blanchet@40253
    31
blanchet@41456
    32
fun prover_description ctxt ({verbose, blocking, ...} : params) name num_facts i
blanchet@41337
    33
                       n goal =
blanchet@41337
    34
  quote name ^
blanchet@41337
    35
  (if verbose then
blanchet@41337
    36
     " with " ^ string_of_int num_facts ^ " fact" ^ plural_s num_facts
blanchet@41337
    37
   else
blanchet@41337
    38
     "") ^
blanchet@42614
    39
  " on " ^ (if n = 1 then "goal" else "subgoal " ^ string_of_int i) ^
blanchet@41337
    40
  (if blocking then
blanchet@42614
    41
     "."
blanchet@41337
    42
   else
blanchet@42614
    43
     ":\n" ^ Syntax.string_of_term ctxt (Thm.term_of (Thm.cprem_of goal i)))
blanchet@41337
    44
blanchet@41583
    45
val auto_minimize_min_facts = Unsynchronized.ref (!binary_min_facts)
blanchet@41339
    46
blanchet@43314
    47
fun get_minimizing_prover ctxt auto may_slice name
blanchet@42613
    48
        (params as {debug, verbose, explicit_apply, ...}) minimize_command
blanchet@41511
    49
        (problem as {state, subgoal, subgoal_count, facts, ...}) =
blanchet@43314
    50
  get_prover ctxt auto may_slice name params minimize_command problem
blanchet@41511
    51
  |> (fn result as {outcome, used_facts, run_time_in_msecs, message} =>
blanchet@41511
    52
         if is_some outcome then
blanchet@41511
    53
           result
blanchet@41511
    54
         else
blanchet@41511
    55
           let
blanchet@41511
    56
             val (used_facts, message) =
blanchet@41583
    57
               if length used_facts >= !auto_minimize_min_facts then
blanchet@42613
    58
                 minimize_facts name params (SOME explicit_apply) (not verbose)
blanchet@42613
    59
                     subgoal subgoal_count state
blanchet@41511
    60
                     (filter_used_facts used_facts
blanchet@41511
    61
                          (map (apsnd single o untranslated_fact) facts))
blanchet@41511
    62
                 |>> Option.map (map fst)
blanchet@41511
    63
               else
blanchet@41511
    64
                 (SOME used_facts, message)
blanchet@41511
    65
           in
blanchet@41511
    66
             case used_facts of
blanchet@41511
    67
               SOME used_facts =>
blanchet@41511
    68
               (if debug andalso not (null used_facts) then
blanchet@41511
    69
                  facts ~~ (0 upto length facts - 1)
blanchet@41511
    70
                  |> map (fn (fact, j) =>
blanchet@41511
    71
                             fact |> untranslated_fact |> apsnd (K j))
blanchet@41511
    72
                  |> filter_used_facts used_facts
blanchet@41511
    73
                  |> map (fn ((name, _), j) => name ^ "@" ^ string_of_int j)
blanchet@41511
    74
                  |> commas
blanchet@41511
    75
                  |> enclose ("Fact" ^ plural_s (length facts) ^ " in " ^
blanchet@41511
    76
                              quote name ^ " proof (of " ^
blanchet@41511
    77
                              string_of_int (length facts) ^ "): ") "."
blanchet@41511
    78
                  |> Output.urgent_message
blanchet@41511
    79
                else
blanchet@41511
    80
                  ();
blanchet@41511
    81
                {outcome = NONE, used_facts = used_facts,
blanchet@41511
    82
                 run_time_in_msecs = run_time_in_msecs, message = message})
blanchet@41511
    83
             | NONE => result
blanchet@41511
    84
           end)
blanchet@41510
    85
blanchet@43314
    86
fun launch_prover (params as {debug, blocking, max_relevant, slicing, timeout,
blanchet@43314
    87
                              expect, ...})
blanchet@43314
    88
        auto may_slice minimize_command only
blanchet@42612
    89
        {state, goal, subgoal, subgoal_count, facts, smt_filter} name =
blanchet@41337
    90
  let
blanchet@41337
    91
    val ctxt = Proof.context_of state
blanchet@43314
    92
    val slicing = may_slice andalso slicing
blanchet@41337
    93
    val birth_time = Time.now ()
blanchet@41337
    94
    val death_time = Time.+ (birth_time, timeout)
blanchet@41337
    95
    val max_relevant =
blanchet@43314
    96
      max_relevant
blanchet@43314
    97
      |> the_default (default_max_relevant_for_prover ctxt slicing name)
blanchet@41337
    98
    val num_facts = length facts |> not only ? Integer.min max_relevant
blanchet@41337
    99
    val desc =
blanchet@41337
   100
      prover_description ctxt params name num_facts subgoal subgoal_count goal
blanchet@41337
   101
    val problem =
blanchet@41337
   102
      {state = state, goal = goal, subgoal = subgoal,
blanchet@41483
   103
       subgoal_count = subgoal_count, facts = take num_facts facts,
blanchet@42612
   104
       smt_filter = smt_filter}
blanchet@41501
   105
    fun really_go () =
blanchet@41511
   106
      problem
blanchet@43314
   107
      |> get_minimizing_prover ctxt auto may_slice name params
blanchet@43314
   108
                               (minimize_command name)
blanchet@41510
   109
      |> (fn {outcome, message, ...} =>
blanchet@41510
   110
             (if is_some outcome then "none" else "some" (* sic *), message))
blanchet@41337
   111
    fun go () =
blanchet@41337
   112
      let
blanchet@41337
   113
        val (outcome_code, message) =
blanchet@41337
   114
          if debug then
blanchet@41337
   115
            really_go ()
blanchet@41337
   116
          else
blanchet@41337
   117
            (really_go ()
blanchet@41337
   118
             handle ERROR message => ("unknown", "Error: " ^ message ^ "\n")
blanchet@41337
   119
                  | exn =>
blanchet@41337
   120
                    if Exn.is_interrupt exn then
blanchet@41337
   121
                      reraise exn
blanchet@41337
   122
                    else
blanchet@41337
   123
                      ("unknown", "Internal error:\n" ^
blanchet@41337
   124
                                  ML_Compiler.exn_message exn ^ "\n"))
blanchet@41337
   125
        val _ =
blanchet@41390
   126
          (* The "expect" argument is deliberately ignored if the prover is
blanchet@41390
   127
             missing so that the "Metis_Examples" can be processed on any
blanchet@41390
   128
             machine. *)
blanchet@41390
   129
          if expect = "" orelse outcome_code = expect orelse
blanchet@41390
   130
             not (is_prover_installed ctxt name) then
blanchet@41337
   131
            ()
blanchet@41337
   132
          else if blocking then
blanchet@41337
   133
            error ("Unexpected outcome: " ^ quote outcome_code ^ ".")
blanchet@41337
   134
          else
blanchet@41337
   135
            warning ("Unexpected outcome: " ^ quote outcome_code ^ ".");
blanchet@41337
   136
      in (outcome_code = "some", message) end
blanchet@41337
   137
  in
blanchet@41337
   138
    if auto then
blanchet@41337
   139
      let val (success, message) = TimeLimit.timeLimit timeout go () in
blanchet@41337
   140
        (success, state |> success ? Proof.goal_message (fn () =>
blanchet@41339
   141
             Pretty.chunks [Pretty.str "",
blanchet@41339
   142
                            Pretty.mark Markup.hilite (Pretty.str message)]))
blanchet@41337
   143
      end
blanchet@41337
   144
    else if blocking then
blanchet@41337
   145
      let val (success, message) = TimeLimit.timeLimit timeout go () in
blanchet@41337
   146
        List.app Output.urgent_message
blanchet@41337
   147
                 (Async_Manager.break_into_chunks [desc ^ "\n" ^ message]);
blanchet@41337
   148
        (success, state)
blanchet@41337
   149
      end
blanchet@41337
   150
    else
blanchet@41337
   151
      (Async_Manager.launch das_Tool birth_time death_time desc (snd o go);
blanchet@41337
   152
       (false, state))
blanchet@41337
   153
  end
blanchet@41337
   154
blanchet@41483
   155
fun class_of_smt_solver ctxt name =
blanchet@41483
   156
  ctxt |> select_smt_solver name
blanchet@41483
   157
       |> SMT_Config.solver_class_of |> SMT_Utils.string_of_class
blanchet@41483
   158
blanchet@41483
   159
(* Makes backtraces more transparent and might be more efficient as well. *)
blanchet@41483
   160
fun smart_par_list_map _ [] = []
blanchet@41483
   161
  | smart_par_list_map f [x] = [f x]
blanchet@41483
   162
  | smart_par_list_map f xs = Par_List.map f xs
blanchet@41483
   163
blanchet@41502
   164
fun dest_SMT_Weighted_Fact (SMT_Weighted_Fact p) = p
blanchet@41502
   165
  | dest_SMT_Weighted_Fact _ = raise Fail "dest_SMT_Weighted_Fact"
blanchet@41502
   166
blanchet@40946
   167
(* FUDGE *)
blanchet@40946
   168
val auto_max_relevant_divisor = 2
blanchet@40241
   169
blanchet@43051
   170
fun run_sledgehammer (params as {debug, blocking, provers, monomorphize,
blanchet@43051
   171
                                 type_sys, relevance_thresholds, max_relevant,
blanchet@43314
   172
                                 slicing, timeout, ...})
blanchet@43314
   173
                     auto may_slice i (relevance_override as {only, ...})
blanchet@43314
   174
                     minimize_command state =
blanchet@40240
   175
  if null provers then
blanchet@40240
   176
    error "No prover is set."
blanchet@39564
   177
  else case subgoal_count state of
wenzelm@40392
   178
    0 => (Output.urgent_message "No subgoal!"; (false, state))
blanchet@39564
   179
  | n =>
blanchet@39564
   180
    let
blanchet@39610
   181
      val _ = Proof.assert_backward state
blanchet@42644
   182
      val print = if auto then K () else Output.urgent_message
blanchet@41483
   183
      val state =
blanchet@41483
   184
        state |> Proof.map_context (Config.put SMT_Config.verbose debug)
blanchet@40441
   185
      val ctxt = Proof.context_of state
wenzelm@43232
   186
      val thy = Proof_Context.theory_of ctxt
blanchet@43314
   187
      val slicing = may_slice andalso slicing
blanchet@40441
   188
      val {facts = chained_ths, goal, ...} = Proof.goal state
blanchet@40241
   189
      val (_, hyp_ts, concl_t) = strip_subgoal goal i
blanchet@41386
   190
      val no_dangerous_types = types_dangerous_types type_sys
blanchet@40240
   191
      val _ = () |> not blocking ? kill_provers
blanchet@42591
   192
      val _ = case find_first (not o is_prover_supported ctxt) provers of
blanchet@41189
   193
                SOME name => error ("No such prover: " ^ name ^ ".")
blanchet@41189
   194
              | NONE => ()
blanchet@42644
   195
      val _ = print "Sledgehammering..."
blanchet@41189
   196
      val (smts, atps) = provers |> List.partition (is_smt_prover ctxt)
blanchet@42612
   197
      fun launch_provers state get_facts translate maybe_smt_filter provers =
blanchet@41502
   198
        let
blanchet@41502
   199
          val facts = get_facts ()
blanchet@41502
   200
          val num_facts = length facts
blanchet@41502
   201
          val facts = facts ~~ (0 upto num_facts - 1)
blanchet@41502
   202
                      |> map (translate num_facts)
blanchet@41502
   203
          val problem =
blanchet@41502
   204
            {state = state, goal = goal, subgoal = i, subgoal_count = n,
blanchet@41502
   205
             facts = facts,
blanchet@42612
   206
             smt_filter = maybe_smt_filter
blanchet@41502
   207
                  (fn () => map_filter (try dest_SMT_Weighted_Fact) facts) i}
blanchet@43314
   208
          val launch = launch_prover params auto may_slice minimize_command only
blanchet@41502
   209
        in
blanchet@41502
   210
          if auto then
blanchet@41502
   211
            fold (fn prover => fn (true, state) => (true, state)
blanchet@41510
   212
                                | (false, _) => launch problem prover)
blanchet@41502
   213
                 provers (false, state)
blanchet@41502
   214
          else
blanchet@41502
   215
            provers
blanchet@41510
   216
            |> (if blocking then smart_par_list_map else map) (launch problem)
blanchet@41502
   217
            |> exists fst |> rpair state
blanchet@41502
   218
        end
blanchet@41483
   219
      fun get_facts label no_dangerous_types relevance_fudge provers =
blanchet@41483
   220
        let
blanchet@41483
   221
          val max_max_relevant =
blanchet@41483
   222
            case max_relevant of
blanchet@41483
   223
              SOME n => n
blanchet@41483
   224
            | NONE =>
blanchet@43314
   225
              0 |> fold (Integer.max
blanchet@43314
   226
                         o default_max_relevant_for_prover ctxt slicing)
blanchet@41483
   227
                        provers
blanchet@41483
   228
                |> auto ? (fn n => n div auto_max_relevant_divisor)
blanchet@41483
   229
          val is_built_in_const =
blanchet@41483
   230
            is_built_in_const_for_prover ctxt (hd provers)
blanchet@41483
   231
        in
blanchet@41483
   232
          relevant_facts ctxt no_dangerous_types relevance_thresholds
blanchet@41483
   233
                         max_max_relevant is_built_in_const relevance_fudge
blanchet@41483
   234
                         relevance_override chained_ths hyp_ts concl_t
blanchet@41483
   235
          |> tap (fn facts =>
blanchet@41483
   236
                     if debug then
blanchet@41483
   237
                       label ^ plural_s (length provers) ^ ": " ^
blanchet@41483
   238
                       (if null facts then
blanchet@41483
   239
                          "Found no relevant facts."
blanchet@41483
   240
                        else
blanchet@41483
   241
                          "Including (up to) " ^ string_of_int (length facts) ^
blanchet@41483
   242
                          " relevant fact" ^ plural_s (length facts) ^ ":\n" ^
blanchet@41483
   243
                          (facts |> map (fst o fst) |> space_implode " ") ^ ".")
blanchet@42644
   244
                       |> print
blanchet@41483
   245
                     else
blanchet@41483
   246
                       ())
blanchet@41483
   247
        end
blanchet@42617
   248
      fun launch_atps accum =
blanchet@42617
   249
        if null atps then
blanchet@41502
   250
          accum
blanchet@41502
   251
        else
blanchet@41510
   252
          launch_provers state
blanchet@41502
   253
              (get_facts "ATP" no_dangerous_types atp_relevance_fudge o K atps)
blanchet@43051
   254
              (if monomorphize then
blanchet@43051
   255
                 K (Untranslated_Fact o fst)
blanchet@43051
   256
               else
blanchet@43051
   257
                 ATP_Translated_Fact oo K (translate_atp_fact ctxt false o fst))
blanchet@41502
   258
              (K (K NONE)) atps
blanchet@42617
   259
      fun launch_smts accum =
blanchet@42617
   260
        if null smts then
blanchet@41483
   261
          accum
blanchet@41483
   262
        else
blanchet@41483
   263
          let
blanchet@41483
   264
            val facts = get_facts "SMT solver" true smt_relevance_fudge smts
blanchet@41502
   265
            val weight = SMT_Weighted_Fact oo weight_smt_fact thy
blanchet@42612
   266
            fun smt_filter facts =
blanchet@42659
   267
              (if debug then curry (op o) SOME
blanchet@42659
   268
               else TimeLimit.timeLimit timeout o try)
boehmes@41680
   269
                  (SMT_Solver.smt_filter_preprocess state (facts ()))
blanchet@41483
   270
          in
blanchet@41483
   271
            smts |> map (`(class_of_smt_solver ctxt))
blanchet@41483
   272
                 |> AList.group (op =)
blanchet@42612
   273
                 |> map (launch_provers state (K facts) weight smt_filter o snd)
blanchet@41483
   274
                 |> exists fst |> rpair state
blanchet@41483
   275
          end
blanchet@41510
   276
      fun launch_atps_and_smt_solvers () =
blanchet@41510
   277
        [launch_atps, launch_smts]
blanchet@41483
   278
        |> smart_par_list_map (fn f => f (false, state) |> K ())
blanchet@42644
   279
        handle ERROR msg => (print ("Error: " ^ msg); error msg)
blanchet@40241
   280
    in
blanchet@40246
   281
      (false, state)
blanchet@41510
   282
      |> (if blocking then launch_atps #> not auto ? launch_smts
blanchet@41510
   283
          else (fn p => Future.fork (tap launch_atps_and_smt_solvers) |> K p))
blanchet@42644
   284
      handle TimeLimit.TimeOut =>
blanchet@42644
   285
             (print "Sledgehammer ran out of time."; (false, state))
blanchet@40241
   286
    end
blanchet@38290
   287
wenzelm@28582
   288
end;