src/HOL/Nitpick_Examples/Refute_Nits.thy
changeset 74641 6f801e1073fa
parent 69597 ff784d5a5bfb
--- a/src/HOL/Nitpick_Examples/Refute_Nits.thy	Sat Oct 30 19:23:01 2021 +0200
+++ b/src/HOL/Nitpick_Examples/Refute_Nits.thy	Sat Oct 30 19:41:09 2021 +0200
@@ -12,7 +12,7 @@
 begin
 
 nitpick_params [verbose, card = 1-6, max_potential = 0,
-                sat_solver = MiniSat_JNI, max_threads = 1, timeout = 240]
+                sat_solver = MiniSat, max_threads = 1, timeout = 240]
 
 lemma "P \<and> Q"
 apply (rule conjI)