src/HOL/ex/Quickcheck_Examples.thy
changeset 45507 6975db7fd6f0
parent 45441 fb4ac1dd4fde
child 45684 3d6ee9c7d7ef
--- a/src/HOL/ex/Quickcheck_Examples.thy	Tue Nov 15 15:38:49 2011 +0100
+++ b/src/HOL/ex/Quickcheck_Examples.thy	Tue Nov 15 15:38:50 2011 +0100
@@ -304,12 +304,22 @@
 quickcheck[random, size = 10]
 oops
 
+lemma "(x :: rat) >= 0"
+quickcheck[random, expect = counterexample]
+quickcheck[exhaustive, expect = counterexample]
+oops
+
 lemma
   "(x :: real) > 0 ==> y > 0 ==> z > 0 ==> x * x + y * y \<noteq> z * z"
 quickcheck[exhaustive, size = 10, expect = counterexample]
 quickcheck[random, size = 10]
 oops
 
+lemma "(x :: real) >= 0"
+quickcheck[random, expect = counterexample]
+quickcheck[exhaustive, expect = counterexample]
+oops
+
 subsubsection {* floor and ceiling functions *}
 
 lemma