| changeset 34083 | 652719832159 |
| parent 33735 | 0c0e7b2ecf2e |
| child 35076 | cc19e2aef17e |
--- a/src/HOL/Nitpick_Examples/Refute_Nits.thy Mon Dec 14 10:31:35 2009 +0100 +++ b/src/HOL/Nitpick_Examples/Refute_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] + lemma "P \<and> Q" apply (rule conjI) nitpick [expect = genuine] 1