src/HOL/ex/set.thy
changeset 36319 8feb2c4bef1a
parent 34055 fdf294ee08b2
child 40928 ace26e2cee91
--- a/src/HOL/ex/set.thy	Fri Apr 23 23:33:48 2010 +0200
+++ b/src/HOL/ex/set.thy	Fri Apr 23 23:35:43 2010 +0200
@@ -26,7 +26,7 @@
   Trivial example of term synthesis: apparently hard for some provers!
 *}
 
-lemma "a \<noteq> b \<Longrightarrow> a \<in> ?X \<and> b \<notin> ?X"
+schematic_lemma "a \<noteq> b \<Longrightarrow> a \<in> ?X \<and> b \<notin> ?X"
   by blast
 
 
@@ -60,15 +60,15 @@
   -- {* Requires best-first search because it is undirectional. *}
   by best
 
-lemma "\<forall>f:: 'a \<Rightarrow> 'a set. \<forall>x. f x \<noteq> ?S f"
+schematic_lemma "\<forall>f:: 'a \<Rightarrow> 'a set. \<forall>x. f x \<noteq> ?S f"
   -- {*This form displays the diagonal term. *}
   by best
 
-lemma "?S \<notin> range (f :: 'a \<Rightarrow> 'a set)"
+schematic_lemma "?S \<notin> range (f :: 'a \<Rightarrow> 'a set)"
   -- {* This form exploits the set constructs. *}
   by (rule notI, erule rangeE, best)
 
-lemma "?S \<notin> range (f :: 'a \<Rightarrow> 'a set)"
+schematic_lemma "?S \<notin> range (f :: 'a \<Rightarrow> 'a set)"
   -- {* Or just this! *}
   by best