src/HOL/Quickcheck_Examples/Quickcheck_Examples.thy
changeset 67613 ce654b0e6d69
parent 67443 3abf6a722518
child 68249 949d93804740
equal deleted inserted replaced
67610:4939494ed791 67613:ce654b0e6d69
   301 quickcheck[exhaustive, expect = counterexample]
   301 quickcheck[exhaustive, expect = counterexample]
   302 oops
   302 oops
   303 
   303 
   304 (* FIXME: some dramatic performance decrease after changing the code equation of the ntrancl *)
   304 (* FIXME: some dramatic performance decrease after changing the code equation of the ntrancl *)
   305 lemma
   305 lemma
   306   "(x, z) : rtrancl (R Un S) ==> \<exists> y. (x, y) : rtrancl R & (y, z) : rtrancl S"
   306   "(x, z) \<in> rtrancl (R Un S) \<Longrightarrow> \<exists>y. (x, y) \<in> rtrancl R \<and> (y, z) \<in> rtrancl S"
   307 (*quickcheck[exhaustive, expect = counterexample]*)
   307 (*quickcheck[exhaustive, expect = counterexample]*)
   308 oops
   308 oops
   309 
   309 
   310 lemma
   310 lemma
   311   "wf (R :: ('a * 'a) set) ==> wf S ==> wf (R Un S)"
   311   "wf (R :: ('a * 'a) set) ==> wf S ==> wf (R Un S)"