src/HOL/Nitpick_Examples/Induct_Nits.thy
changeset 34083 652719832159
parent 33197 de6285ebcc05
child 35076 cc19e2aef17e
--- a/src/HOL/Nitpick_Examples/Induct_Nits.thy	Mon Dec 14 10:31:35 2009 +0100
+++ b/src/HOL/Nitpick_Examples/Induct_Nits.thy	Mon Dec 14 10:59:46 2009 +0100
@@ -11,7 +11,7 @@
 imports Main
 begin
 
-nitpick_params [show_all]
+nitpick_params [sat_solver = MiniSatJNI, max_threads = 1, timeout = 60 s]
 
 inductive p1 :: "nat \<Rightarrow> bool" where
 "p1 0" |