11 replacing = |
11 replacing = |
12 [(("appendP", "limited_appendP"), "quickcheck"), |
12 [(("appendP", "limited_appendP"), "quickcheck"), |
13 (("revP", "limited_revP"), "quickcheck"), |
13 (("revP", "limited_revP"), "quickcheck"), |
14 (("appendP", "limited_appendP"), "lim_revP")], |
14 (("appendP", "limited_appendP"), "lim_revP")], |
15 manual_reorder = [], |
15 manual_reorder = [], |
|
16 timeout = Time.fromSeconds 10, |
16 prolog_system = Code_Prolog.SWI_PROLOG}) *} |
17 prolog_system = Code_Prolog.SWI_PROLOG}) *} |
17 |
18 |
18 lemma "(xs :: nat list) = ys @ ys --> rev xs = xs" |
19 lemma "(xs :: nat list) = ys @ ys --> rev xs = xs" |
19 quickcheck[generator = code, iterations = 200000, expect = counterexample] |
20 quickcheck[generator = code, iterations = 200000, expect = counterexample] |
20 quickcheck[generator = predicate_compile_wo_ff, iterations = 1, expect = counterexample] |
21 quickcheck[generator = predicate_compile_wo_ff, iterations = 1, expect = counterexample] |