changeset 20770 | 2c583720436e |
parent 20362 | bbff23c3e2ca |
child 21210 | c17fd2df4e9e |
--- a/src/HOL/Library/FuncSet.thy Thu Sep 28 23:42:39 2006 +0200 +++ b/src/HOL/Library/FuncSet.thy Thu Sep 28 23:42:43 2006 +0200 @@ -39,8 +39,8 @@ "_lam" :: "[pttrn, 'a set, 'a => 'b] => ('a=>'b)" ("(3\<lambda>_\<in>_./ _)" [0,0,3] 3) translations - "PI x:A. B" == "Pi A (%x. B)" - "%x:A. f" == "restrict (%x. f) A" + "PI x:A. B" == "CONST Pi A (%x. B)" + "%x:A. f" == "CONST restrict (%x. f) A" definition "compose" :: "['a set, 'b => 'c, 'a => 'b] => ('a => 'c)"