src/HOL/Quickcheck_Examples/Quickcheck_Examples.thy
changeset 63901 4ce989e962e0
parent 63882 018998c00003
child 66453 cc19f7ca2ed6
equal deleted inserted replaced
63899:dc036b1a2a6f 63901:4ce989e962e0
   268 lemma "(\<forall>x. \<exists>y. P x y) \<longrightarrow> (\<exists>y. \<forall>x. P x y)"
   268 lemma "(\<forall>x. \<exists>y. P x y) \<longrightarrow> (\<exists>y. \<forall>x. P x y)"
   269   quickcheck[random, expect = counterexample]
   269   quickcheck[random, expect = counterexample]
   270   quickcheck[expect = counterexample]
   270   quickcheck[expect = counterexample]
   271 oops
   271 oops
   272 
   272 
   273 lemma "(\<exists>x. P x) \<longrightarrow> (EX! x. P x)"
   273 lemma "(\<exists>x. P x) \<longrightarrow> (\<exists>!x. P x)"
   274   quickcheck[random, expect = counterexample]
   274   quickcheck[random, expect = counterexample]
   275   quickcheck[expect = counterexample]
   275   quickcheck[expect = counterexample]
   276 oops
   276 oops
   277 
   277 
   278 
   278