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