src/HOL/ex/Quickcheck_Examples.thy
changeset 45762 daf57640d4df
parent 45720 d8fbd3fa0375
child 45765 cb6ddee6a463
--- a/src/HOL/ex/Quickcheck_Examples.thy	Mon Dec 05 12:36:06 2011 +0100
+++ b/src/HOL/ex/Quickcheck_Examples.thy	Mon Dec 05 12:36:19 2011 +0100
@@ -411,10 +411,9 @@
 
 lemma
   "xs = [] ==> hd xs \<noteq> x"
-quickcheck[exhaustive, potential = false, expect = no_counterexample]
-quickcheck[exhaustive, potential = true, expect = counterexample]
-quickcheck[random, potential = false, report = false, expect = no_counterexample]
-quickcheck[random, potential = true, report = false, expect = counterexample]
+quickcheck[exhaustive, expect = no_counterexample]
+quickcheck[random, report = false, expect = no_counterexample]
+quickcheck[random, report = true, expect = counterexample]
 oops
 
 lemma