src/HOL/Tools/Sledgehammer/sledgehammer_provers.ML
changeset 52150 41c885784e04
parent 52125 ac7830871177
child 52196 2281f33e8da6
equal deleted inserted replaced
52149:32b1dbda331c 52150:41c885784e04
   910     fun clean_up () =
   910     fun clean_up () =
   911       if dest_dir = "" then (try File.rm prob_path; ()) else ()
   911       if dest_dir = "" then (try File.rm prob_path; ()) else ()
   912     fun export (_, (output, _, _, _, _)) =
   912     fun export (_, (output, _, _, _, _)) =
   913       if dest_dir = "" then ()
   913       if dest_dir = "" then ()
   914       else File.write (Path.explode (Path.implode prob_path ^ "_proof")) output
   914       else File.write (Path.explode (Path.implode prob_path ^ "_proof")) output
   915     val ((_, (_, pool, fact_names, _, sym_tab)),
   915     val ((_, (_, pool, fact_names, lifted, sym_tab)),
   916          (output, run_time, used_from, atp_proof, outcome)) =
   916          (output, run_time, used_from, atp_proof, outcome)) =
   917       with_cleanup clean_up run () |> tap export
   917       with_cleanup clean_up run () |> tap export
   918     val important_message =
   918     val important_message =
   919       if mode = Normal andalso
   919       if mode = Normal andalso
   920          random_range 0 (atp_important_message_keep_quotient - 1) = 0 then
   920          random_range 0 (atp_important_message_keep_quotient - 1) = 0 then
   949                     Output.urgent_message "Generating proof text..."
   949                     Output.urgent_message "Generating proof text..."
   950                   else
   950                   else
   951                     ()
   951                     ()
   952                 val isar_params =
   952                 val isar_params =
   953                   (debug, verbose, preplay_timeout, preplay_trace, isar_compress,
   953                   (debug, verbose, preplay_timeout, preplay_trace, isar_compress,
   954                    pool, fact_names, sym_tab, atp_proof, goal)
   954                    pool, fact_names, lifted, sym_tab, atp_proof, goal)
   955                 val one_line_params =
   955                 val one_line_params =
   956                   (preplay, proof_banner mode name, used_facts,
   956                   (preplay, proof_banner mode name, used_facts,
   957                    choose_minimize_command ctxt params minimize_command name
   957                    choose_minimize_command ctxt params minimize_command name
   958                                            preplay,
   958                                            preplay,
   959                    subgoal, subgoal_count)
   959                    subgoal, subgoal_count)