src/HOL/Nitpick_Examples/Induct_Nits.thy
changeset 54680 93f6d33a754e
parent 54633 86e0b402994c
child 55893 aed17a173d16
--- a/src/HOL/Nitpick_Examples/Induct_Nits.thy	Thu Dec 05 23:13:54 2013 +0000
+++ b/src/HOL/Nitpick_Examples/Induct_Nits.thy	Fri Dec 06 09:42:13 2013 +0100
@@ -12,7 +12,7 @@
 begin
 
 nitpick_params [verbose, card = 1\<emdash>8, unary_ints,
-                sat_solver = Riss3g, max_threads = 1, timeout = 240]
+                sat_solver = MiniSat_JNI, max_threads = 1, timeout = 240]
 
 inductive p1 :: "nat \<Rightarrow> bool" where
 "p1 0" |