src/FOL/ex/Quantifiers_Cla.thy
changeset 36319 8feb2c4bef1a
parent 31974 e81979a703a4
child 41777 1f7cbe39d425
--- a/src/FOL/ex/Quantifiers_Cla.thy	Fri Apr 23 23:33:48 2010 +0200
+++ b/src/FOL/ex/Quantifiers_Cla.thy	Fri Apr 23 23:35:43 2010 +0200
@@ -58,11 +58,11 @@
   apply fast?
   oops
 
-lemma "P(?a) --> (ALL x. P(x))"
+schematic_lemma "P(?a) --> (ALL x. P(x))"
   apply fast?
   oops
 
-lemma "(P(?a) --> (ALL x. Q(x))) --> (ALL x. P(x) --> Q(x))"
+schematic_lemma "(P(?a) --> (ALL x. Q(x))) --> (ALL x. P(x) --> Q(x))"
   apply fast?
   oops
 
@@ -76,7 +76,7 @@
 lemma "(P --> (EX x. Q(x))) & P --> (EX x. Q(x))"
   by fast
 
-lemma "(ALL x. P(x)-->Q(f(x))) & (ALL x. Q(x)-->R(g(x))) & P(d) --> R(?a)"
+schematic_lemma "(ALL x. P(x)-->Q(f(x))) & (ALL x. Q(x)-->R(g(x))) & P(d) --> R(?a)"
   by fast
 
 lemma "(ALL x. Q(x))  -->  (EX x. Q(x))"