src/HOL/Tools/Sledgehammer/sledgehammer_provers.ML
changeset 52697 6fb98a20c349
parent 52632 23393c31c7fe
child 52754 d9d90d29860e
equal deleted inserted replaced
52696:38466f4f3483 52697:6fb98a20c349
   971                    choose_minimize_command ctxt params minimize_command name
   971                    choose_minimize_command ctxt params minimize_command name
   972                                            preplay,
   972                                            preplay,
   973                    subgoal, subgoal_count)
   973                    subgoal, subgoal_count)
   974                 val num_chained = length (#facts (Proof.goal state))
   974                 val num_chained = length (#facts (Proof.goal state))
   975               in
   975               in
   976                 proof_text ctxt isar_proofs isar_params num_chained
   976                 proof_text ctxt (mode = Auto_Try) isar_proofs isar_params num_chained
   977                            one_line_params
   977                            one_line_params
   978               end,
   978               end,
   979            (if verbose then
   979            (if verbose then
   980               "\nATP real CPU time: " ^ string_of_time run_time ^ "."
   980               "\nATP real CPU time: " ^ string_of_time run_time ^ "."
   981             else
   981             else
  1175                 (preplay, proof_banner mode name, used_facts,
  1175                 (preplay, proof_banner mode name, used_facts,
  1176                  choose_minimize_command ctxt params minimize_command name
  1176                  choose_minimize_command ctxt params minimize_command name
  1177                                          preplay,
  1177                                          preplay,
  1178                  subgoal, subgoal_count)
  1178                  subgoal, subgoal_count)
  1179               val num_chained = length (#facts (Proof.goal state))
  1179               val num_chained = length (#facts (Proof.goal state))
  1180             in one_line_proof_text num_chained one_line_params end,
  1180             in one_line_proof_text (mode = Auto_Try) num_chained one_line_params end,
  1181          if verbose then
  1181          if verbose then
  1182            "\nSMT solver real CPU time: " ^ string_of_time run_time ^ "."
  1182            "\nSMT solver real CPU time: " ^ string_of_time run_time ^ "."
  1183          else
  1183          else
  1184            "")
  1184            "")
  1185       | SOME failure =>
  1185       | SOME failure =>
  1220               val one_line_params =
  1220               val one_line_params =
  1221                 (play, proof_banner mode name, used_facts,
  1221                 (play, proof_banner mode name, used_facts,
  1222                  minimize_command override_params name, subgoal,
  1222                  minimize_command override_params name, subgoal,
  1223                  subgoal_count)
  1223                  subgoal_count)
  1224               val num_chained = length (#facts (Proof.goal state))
  1224               val num_chained = length (#facts (Proof.goal state))
  1225             in one_line_proof_text num_chained one_line_params end,
  1225             in one_line_proof_text (mode = Auto_Try) num_chained one_line_params end,
  1226        message_tail = ""}
  1226        message_tail = ""}
  1227     | play =>
  1227     | play =>
  1228       let
  1228       let
  1229         val failure = case play of Failed_to_Play _ => GaveUp | _ => TimedOut
  1229         val failure = case play of Failed_to_Play _ => GaveUp | _ => TimedOut
  1230       in
  1230       in