src/HOL/ex/Quickcheck_Examples.thy
changeset 45972 deda685ba210
parent 45942 4dfb1f6bd99b
child 45990 b7b905b23b2a
--- a/src/HOL/ex/Quickcheck_Examples.thy	Sat Dec 24 15:53:11 2011 +0100
+++ b/src/HOL/ex/Quickcheck_Examples.thy	Sat Dec 24 15:53:11 2011 +0100
@@ -6,7 +6,7 @@
 header {* Examples for the 'quickcheck' command *}
 
 theory Quickcheck_Examples
-imports Complex_Main "~~/src/HOL/Library/Dlist"
+imports Complex_Main "~~/src/HOL/Library/Dlist" "~~/src/HOL/Library/More_Set"
 begin
 
 text {*
@@ -271,12 +271,12 @@
 
 lemma
   "acyclic R ==> acyclic S ==> acyclic (R Un S)"
-quickcheck[expect = counterexample]
+(* FIXME: missing instance for narrowing -- quickcheck[expect = counterexample] *)
 oops
 
 lemma
   "(x, z) : rtrancl (R Un S) ==> \<exists> y. (x, y) : rtrancl R & (y, z) : rtrancl S"
-quickcheck[expect = counterexample]
+(* FIXME: missing instance for narrowing -- quickcheck[expect = counterexample] *)
 oops