changeset 54633 | 86e0b402994c |
parent 46095 | cd5c72462bca |
child 54680 | 93f6d33a754e |
--- a/src/HOL/Nitpick_Examples/Pattern_Nits.thy Thu Dec 05 13:22:00 2013 +0100 +++ b/src/HOL/Nitpick_Examples/Pattern_Nits.thy Thu Dec 05 13:38:20 2013 +0100 @@ -11,7 +11,7 @@ imports Main begin -nitpick_params [verbose, card = 8, max_potential = 0, sat_solver = MiniSat_JNI, +nitpick_params [verbose, card = 8, max_potential = 0, sat_solver = Riss3g, max_threads = 1, timeout = 240] lemma "x = (case u of () \<Rightarrow> y)"