meson no longer does these examples
authorpaulson
Tue, 13 Dec 2005 15:34:21 +0100
changeset 18391 2e901da7cd3a
parent 18390 aaecdaef4c04
child 18392 fdefc3cd45c5
meson no longer does these examples
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:
      "\<And>S::'a set set. \<forall>x \<in> S. \<forall>y \<in> S. x \<subseteq> y \<Longrightarrow> \<exists>z. S \<subseteq> {z}"
+  by blast
+(*With removal of negated equality literals, this no longer works:
   by (meson subsetI subset_antisym insertCI)
+*)
 
 lemma singleton_example_2:
      "\<forall>x \<in> S. \<Union>S \<subseteq> x \<Longrightarrow> \<exists>z. S \<subseteq> {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 "\<exists>!x. f (g x) = x \<Longrightarrow> \<exists>!y. g (f y) = y"