diff -r c2ee8f5a5652 -r 7e6cdcd113a2 src/HOL/Library/FuncSet.thy --- a/src/HOL/Library/FuncSet.thy Fri Sep 27 13:24:29 2002 +0200 +++ b/src/HOL/Library/FuncSet.thy Fri Sep 27 16:44:50 2002 +0200 @@ -39,6 +39,7 @@ compose :: "['a set, 'b => 'c, 'a => 'b] => ('a => 'c)" "compose A g f == \x\A. g (f x)" +print_translation {* [("Pi", dependent_tr' ("@Pi", "funcset"))] *} subsection{*Basic Properties of @{term Pi}*} @@ -105,7 +106,6 @@ lemma restrict_in_funcset: "(!!x. x \ A ==> f x \ B) ==> (\x\A. f x) \ A -> B" by (simp add: Pi_def restrict_def) - lemma restrictI: "(!!x. x \ A ==> f x \ B x) ==> (\x\A. f x) \ Pi A B" by (simp add: Pi_def restrict_def)