src/FOLP/ex/Intro.thy
changeset 36319 8feb2c4bef1a
parent 35762 af3ff2ba4c54
child 41526 54b4686704af
--- a/src/FOLP/ex/Intro.thy	Fri Apr 23 23:33:48 2010 +0200
+++ b/src/FOLP/ex/Intro.thy	Fri Apr 23 23:35:43 2010 +0200
@@ -13,7 +13,7 @@
 
 subsubsection {* Some simple backward proofs *}
 
-lemma mythm: "?p : P|P --> P"
+schematic_lemma mythm: "?p : P|P --> P"
 apply (rule impI)
 apply (rule disjE)
 prefer 3 apply (assumption)
@@ -21,7 +21,7 @@
 apply assumption
 done
 
-lemma "?p : (P & Q) | R --> (P | R)"
+schematic_lemma "?p : (P & Q) | R --> (P | R)"
 apply (rule impI)
 apply (erule disjE)
 apply (drule conjunct1)
@@ -31,7 +31,7 @@
 done
 
 (*Correct version, delaying use of "spec" until last*)
-lemma "?p : (ALL x y. P(x,y)) --> (ALL z w. P(w,z))"
+schematic_lemma "?p : (ALL x y. P(x,y)) --> (ALL z w. P(w,z))"
 apply (rule impI)
 apply (rule allI)
 apply (rule allI)
@@ -43,13 +43,13 @@
 
 subsubsection {* Demonstration of @{text "fast"} *}
 
-lemma "?p : (EX y. ALL x. J(y,x) <-> ~J(x,x))
+schematic_lemma "?p : (EX y. ALL x. J(y,x) <-> ~J(x,x))
         -->  ~ (ALL x. EX y. ALL z. J(z,y) <-> ~ J(z,x))"
 apply (tactic {* fast_tac FOLP_cs 1 *})
 done
 
 
-lemma "?p : ALL x. P(x,f(x)) <->
+schematic_lemma "?p : ALL x. P(x,f(x)) <->
         (EX y. (ALL z. P(z,y) --> P(z,f(x))) & P(x,y))"
 apply (tactic {* fast_tac FOLP_cs 1 *})
 done
@@ -57,7 +57,7 @@
 
 subsubsection {* Derivation of conjunction elimination rule *}
 
-lemma
+schematic_lemma
   assumes major: "p : P&Q"
     and minor: "!!x y. [| x : P; y : Q |] ==> f(x, y) : R"
   shows "?p : R"
@@ -71,7 +71,7 @@
 
 text {* Derivation of negation introduction *}
 
-lemma
+schematic_lemma
   assumes "!!x. x : P ==> f(x) : False"
   shows "?p : ~ P"
 apply (unfold not_def)
@@ -80,7 +80,7 @@
 apply assumption
 done
 
-lemma
+schematic_lemma
   assumes major: "p : ~P"
     and minor: "q : P"
   shows "?p : R"
@@ -91,7 +91,7 @@
 done
 
 text {* Alternative proof of the result above *}
-lemma
+schematic_lemma
   assumes major: "p : ~P"
     and minor: "q : P"
   shows "?p : R"