--- 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:
"\<lbrakk> is_ord(MKT (x :: nat) l r h); height l = height r + 2 \<rbrakk> \<Longrightarrow> 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