tuned
authornipkow
Sat, 20 Jun 2009 14:00:36 +0200
changeset 31731 7ffc1a901eea
parent 31730 d74830dc3e4a
child 31732 052399f580cf
child 31735 a00292a5587d
tuned
src/HOL/Library/FuncSet.thy
--- a/src/HOL/Library/FuncSet.thy	Sat Jun 20 13:34:54 2009 +0200
+++ b/src/HOL/Library/FuncSet.thy	Sat Jun 20 14:00:36 2009 +0200
@@ -51,9 +51,12 @@
 
 subsection{*Basic Properties of @{term Pi}*}
 
-lemma Pi_I[simp]: "(!!x. x \<in> A ==> f x \<in> B x) ==> f \<in> Pi A B"
+lemma Pi_I: "(!!x. x \<in> A ==> f x \<in> B x) ==> f \<in> Pi A B"
   by (simp add: Pi_def)
 
+lemma Pi_I'[simp]: "(!!x. x : A --> f x : B x) ==> f : Pi A B"
+by(simp add:Pi_def)
+
 lemma funcsetI: "(!!x. x \<in> A ==> f x \<in> B) ==> f \<in> A -> B"
   by (simp add: Pi_def)