# HG changeset patch # User bulwahn # Date 1299836263 -3600 # Node ID 34360908cb78fbc103dfb040526bd180430cd3eb # Parent 1848775589e597c1c71aba6b9e50374bc1250175 increasing timeout of example for counterexample generation diff -r 1848775589e5 -r 34360908cb78 src/HOL/ex/LSC_Examples.thy --- a/src/HOL/ex/LSC_Examples.thy Fri Mar 11 10:37:42 2011 +0100 +++ b/src/HOL/ex/LSC_Examples.thy Fri Mar 11 10:37:43 2011 +0100 @@ -134,7 +134,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 = lazy_exhaustive, finite_types = false, default_type = nat, size = 1, timeout = 80, expect = counterexample] +quickcheck[tester = lazy_exhaustive, finite_types = false, default_type = nat, size = 1, timeout = 100, expect = counterexample] oops