src/HOL/Nitpick_Examples/Special_Nits.thy
changeset 34083 652719832159
parent 33737 e441fede163d
child 34124 c4628a1dcf75
--- a/src/HOL/Nitpick_Examples/Special_Nits.thy	Mon Dec 14 10:31:35 2009 +0100
+++ b/src/HOL/Nitpick_Examples/Special_Nits.thy	Mon Dec 14 10:59:46 2009 +0100
@@ -11,7 +11,8 @@
 imports Main
 begin
 
-nitpick_params [card = 4, debug, show_consts, timeout = 10 s]
+nitpick_params [sat_solver = MiniSatJNI, max_threads = 1, timeout = 60 s,
+                card = 4]
 
 fun f1 :: "nat \<Rightarrow> nat \<Rightarrow> nat \<Rightarrow> nat \<Rightarrow> nat \<Rightarrow> nat" where
 "f1 a b c d e = a + b + c + d + e"