src/HOL/ex/Quickcheck_Narrowing_Examples.thy
changeset 45658 c2c647a4c237
parent 45441 fb4ac1dd4fde
child 45773 7f2366dc8c0f
--- a/src/HOL/ex/Quickcheck_Narrowing_Examples.thy	Sun Nov 27 23:12:03 2011 +0100
+++ b/src/HOL/ex/Quickcheck_Narrowing_Examples.thy	Mon Nov 28 12:13:27 2011 +0100
@@ -98,7 +98,7 @@
 
 lemma
   "list_all2 P (rev xs) (rev ys) = list_all2 P xs (rev ys)"
-  quickcheck[tester = narrowing, finite_types = false, expect = counterexample]
+  quickcheck[tester = narrowing, finite_types = false, expect = counterexample, timeout = 60]
 oops
 
 lemma "map f xs = F f xs"