src/HOL/ex/Quickcheck_Examples.thy
changeset 43890 eba9c3b1f84a
parent 43803 06094d789512
child 43909 7feb72f7bc3e
--- a/src/HOL/ex/Quickcheck_Examples.thy	Mon Jul 18 10:34:21 2011 +0200
+++ b/src/HOL/ex/Quickcheck_Examples.thy	Mon Jul 18 11:38:14 2011 +0200
@@ -361,7 +361,7 @@
 begin
 
 lemma "False"
-quickcheck[expect = counterexample]
+quickcheck[exhaustive, expect = counterexample]
 oops
 
 end