src/HOL/ex/Quickcheck_Examples.thy
changeset 46397 eef663f8242e
parent 46348 ee5009212793
child 46421 5ab496224729
--- a/src/HOL/ex/Quickcheck_Examples.thy	Thu Feb 02 10:12:30 2012 +0100
+++ b/src/HOL/ex/Quickcheck_Examples.thy	Thu Feb 02 10:16:10 2012 +0100
@@ -267,6 +267,14 @@
 oops
 
 
+subsection {* Examples with sets *}
+
+lemma
+  "{} = A Un - A"
+quickcheck[exhaustive, expect = counterexample]
+oops
+
+
 subsection {* Examples with relations *}
 
 lemma