diff -r aaecdaef4c04 -r 2e901da7cd3a src/HOL/ex/set.thy --- a/src/HOL/ex/set.thy Tue Dec 13 15:34:02 2005 +0100 +++ b/src/HOL/ex/set.thy Tue Dec 13 15:34:21 2005 +0100 @@ -40,18 +40,20 @@ -- {* Inter-image, called @{text Int_Inter_image} in Main HOL *} by blast -text{*Both of the singleton examples can be proved very quickly by @{text -"blast del: UNIV_I"} but not by @{text blast} alone. For some reason, @{text -UNIV_I} greatly increases the search space.*} - lemma singleton_example_1: "\S::'a set set. \x \ S. \y \ S. x \ y \ \z. S \ {z}" + by blast +(*With removal of negated equality literals, this no longer works: by (meson subsetI subset_antisym insertCI) +*) lemma singleton_example_2: "\x \ S. \S \ x \ \z. S \ {z}" -- {*Variant of the problem above. *} + by blast +(*With removal of negated equality literals, this no longer works: by (meson subsetI subset_antisym insertCI UnionI) +*) lemma "\!x. f (g x) = x \ \!y. g (f y) = y"