src/HOL/Nitpick_Examples/Special_Nits.thy
changeset 54680 93f6d33a754e
parent 54633 86e0b402994c
child 58889 5b7a9633cfa8
--- a/src/HOL/Nitpick_Examples/Special_Nits.thy	Thu Dec 05 23:13:54 2013 +0000
+++ b/src/HOL/Nitpick_Examples/Special_Nits.thy	Fri Dec 06 09:42:13 2013 +0100
@@ -11,7 +11,7 @@
 imports Main
 begin
 
-nitpick_params [verbose, card = 4, sat_solver = Riss3g, max_threads = 1,
+nitpick_params [verbose, card = 4, sat_solver = MiniSat_JNI, max_threads = 1,
                 timeout = 240]
 
 fun f1 :: "nat \<Rightarrow> nat \<Rightarrow> nat \<Rightarrow> nat \<Rightarrow> nat \<Rightarrow> nat" where