src/HOL/Nitpick_Examples/Manual_Nits.thy
changeset 42421 6bc725d60593
parent 42208 02513eb26eb7
child 42959 ee829022381d
--- a/src/HOL/Nitpick_Examples/Manual_Nits.thy	Wed Apr 20 07:44:23 2011 +0200
+++ b/src/HOL/Nitpick_Examples/Manual_Nits.thy	Wed Apr 20 10:14:24 2011 +0200
@@ -70,7 +70,7 @@
 oops
 
 lemma "\<forall>n. Suc n \<noteq> n \<Longrightarrow> P"
-nitpick [card nat = 100, check_potential, expect = genuine]
+nitpick [card nat = 100, check_potential, tac_timeout = 5, expect = genuine]
 oops
 
 lemma "P Suc"