--- a/src/HOL/Tools/Sledgehammer/sledgehammer_commands.ML Mon Jan 09 17:16:22 2023 +0000
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_commands.ML Tue Jan 10 11:06:20 2023 +0000
@@ -163,7 +163,7 @@
(* The first ATP of the list is used by Auto Sledgehammer. *)
fun default_provers_param_value ctxt =
\<comment> \<open>see also \<^system_option>\<open>sledgehammer_provers\<close>\<close>
- filter (is_prover_installed ctxt) (smts ctxt @ non_dummy_atps)
+ filter (is_prover_installed ctxt) (smts ctxt @ local_atps)
|> implode_param
fun set_default_raw_param param thy =