src/HOL/Tools/Sledgehammer/sledgehammer_prover.ML
changeset 75031 ae4dc5ac983f
parent 75026 b61949cba32a
child 75034 890b70f96fe4
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_prover.ML	Mon Jan 31 16:09:23 2022 +0100
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_prover.ML	Mon Jan 31 16:09:23 2022 +0100
@@ -40,6 +40,7 @@
      fact_thresholds : real * real,
      max_mono_iters : int option,
      max_new_mono_instances : int option,
+     max_proofs : int,
      isar_proofs : bool option,
      compress : real option,
      try0 : bool,
@@ -51,7 +52,6 @@
      expect : string}
 
   val string_of_params : params -> string
-  val set_params_provers : params -> string list -> params
   val slice_timeout : int -> Time.time -> Time.time
 
   type prover_problem =
@@ -141,6 +141,7 @@
    fact_thresholds : real * real,
    max_mono_iters : int option,
    max_new_mono_instances : int option,
+   max_proofs : int,
    isar_proofs : bool option,
    compress : real option,
    try0 : bool,
@@ -158,33 +159,6 @@
     induction_rules = Exclude ?
       filter_out (fn ((_, (_, ATP_Problem_Generate.Induction)), _) => true | _ => false)
 
-fun set_params_provers params provers =
-  {debug = #debug params,
-   verbose = #verbose params,
-   overlord = #overlord params,
-   spy = #spy params,
-   provers = provers,
-   type_enc = #type_enc params,
-   strict = #strict params,
-   lam_trans = #lam_trans params,
-   uncurried_aliases = #uncurried_aliases params,
-   learn = #learn params,
-   fact_filter = #fact_filter params,
-   induction_rules = #induction_rules params,
-   max_facts = #max_facts params,
-   fact_thresholds = #fact_thresholds params,
-   max_mono_iters = #max_mono_iters params,
-   max_new_mono_instances = #max_new_mono_instances params,
-   isar_proofs = #isar_proofs params,
-   compress = #compress params,
-   try0 = #try0 params,
-   smt_proofs = #smt_proofs params,
-   minimize = #minimize params,
-   slices = #slices params,
-   timeout = #timeout params,
-   preplay_timeout = #preplay_timeout params,
-   expect = #expect params}
-
 fun slice_timeout slices timeout =
   Time.toReal timeout * Real.fromInt (Multithreading.max_threads ()) / Real.fromInt slices
   |> seconds