src/HOL/Quickcheck_Examples/Quickcheck_Examples.thy
changeset 58813 625d04d4fd2a
parent 58310 91ea607a34d8
child 58889 5b7a9633cfa8
equal deleted inserted replaced
58812:5a9a2d3b9f8b 58813:625d04d4fd2a
   542 quickcheck[random, report = true, expect = no_counterexample]
   542 quickcheck[random, report = true, expect = no_counterexample]
   543 oops
   543 oops
   544 
   544 
   545 text {* with the simple testing scheme *}
   545 text {* with the simple testing scheme *}
   546 
   546 
   547 setup {* Exhaustive_Generators.setup_exhaustive_datatype_interpretation *}
   547 setup Exhaustive_Generators.setup_exhaustive_datatype_interpretation
   548 declare [[quickcheck_full_support = false]]
   548 declare [[quickcheck_full_support = false]]
   549 
   549 
   550 lemma
   550 lemma
   551   "xs = [] ==> hd xs \<noteq> x"
   551   "xs = [] ==> hd xs \<noteq> x"
   552 quickcheck[exhaustive, expect = no_counterexample]
   552 quickcheck[exhaustive, expect = no_counterexample]