lemmas strip;
authorwenzelm
Thu, 01 Jun 2006 21:14:54 +0200
changeset 19756 61c4117345c6
parent 19755 90f80de04c46
child 19757 4a2a71c31968
lemmas strip;
src/FOL/IFOL.thy
--- a/src/FOL/IFOL.thy	Thu Jun 01 21:14:05 2006 +0200
+++ b/src/FOL/IFOL.thy	Thu Jun 01 21:14:54 2006 +0200
@@ -117,6 +117,9 @@
   iff_reflection: "(P<->Q) ==> (P==Q)"
 
 
+lemmas strip = impI allI
+
+
 text{*Thanks to Stephan Merz*}
 theorem subst:
   assumes eq: "a = b" and p: "P(a)"