src/HOL/Nitpick_Examples/Datatype_Nits.thy
changeset 34083 652719832159
parent 33199 6c9b2a94a69c
child 34126 8a2c5d7aff51
--- a/src/HOL/Nitpick_Examples/Datatype_Nits.thy	Mon Dec 14 10:31:35 2009 +0100
+++ b/src/HOL/Nitpick_Examples/Datatype_Nits.thy	Mon Dec 14 10:59:46 2009 +0100
@@ -11,6 +11,8 @@
 imports Main
 begin
 
+nitpick_params [sat_solver = MiniSatJNI, max_threads = 1, timeout = 60 s]
+
 primrec rot where
 "rot Nibble0 = Nibble1" |
 "rot Nibble1 = Nibble2" |