src/HOL/Predicate_Compile_Examples/IMP_1.thy
changeset 43686 bc7d63c7fd6f
parent 42397 13798dcbdca5
child 45451 74515e8e6046
equal deleted inserted replaced
43656:9ece73262746 43686:bc7d63c7fd6f
    24   "s ==> exec c1 s t ==> exec (IF c1 c2) s t" |
    24   "s ==> exec c1 s t ==> exec (IF c1 c2) s t" |
    25   "\<not> s ==> exec c2 s t ==> exec (IF c1 c2) s t"
    25   "\<not> s ==> exec c2 s t ==> exec (IF c1 c2) s t"
    26 
    26 
    27 lemma
    27 lemma
    28   "exec c s s' ==> exec (Seq c c) s s'"
    28   "exec c s s' ==> exec (Seq c c) s s'"
    29 quickcheck[tester = predicate_compile_wo_ff, size = 2, iterations = 10, timeout = 600.0, expect = counterexample]
    29 quickcheck[tester = predicate_compile_wo_ff, size = 2, iterations = 100, timeout = 600.0, expect = counterexample]
    30 oops
    30 oops
    31 
    31 
    32 
    32 
    33 end
    33 end