equal
deleted
inserted
replaced
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] |