# HG changeset patch # User bulwahn # Date 1323181396 -3600 # Node ID 7f2366dc8c0f83d61217c1b4581f0c664c6ea01c # Parent 8a8f78ce0dcf0a0f07f3f8e4bb0002eea0c3f5d1 increasing quickcheck's timeout in the example theory to avoid failures on the testing infrastructure diff -r 8a8f78ce0dcf -r 7f2366dc8c0f src/HOL/ex/Quickcheck_Narrowing_Examples.thy --- a/src/HOL/ex/Quickcheck_Narrowing_Examples.thy Tue Dec 06 14:29:37 2011 +0100 +++ b/src/HOL/ex/Quickcheck_Narrowing_Examples.thy Tue Dec 06 15:23:16 2011 +0100 @@ -9,6 +9,8 @@ imports Main begin +declare [[quickcheck_timeout = 3600]] + subsection {* Minimalistic examples *} lemma @@ -98,7 +100,7 @@ lemma "list_all2 P (rev xs) (rev ys) = list_all2 P xs (rev ys)" - quickcheck[tester = narrowing, finite_types = false, expect = counterexample, timeout = 60] + quickcheck[tester = narrowing, finite_types = false, expect = counterexample] oops lemma "map f xs = F f xs" @@ -224,7 +226,7 @@ lemma is_ord_l_bal: "\ is_ord(MKT (x :: nat) l r h); height l = height r + 2 \ \ is_ord(l_bal(x,l,r))" -quickcheck[tester = narrowing, finite_types = false, default_type = nat, size = 6, timeout = 1000, expect = counterexample] +quickcheck[tester = narrowing, finite_types = false, default_type = nat, size = 6, expect = counterexample] oops