diff -r 079fe4292526 -r c7723cc15de8 src/HOL/Library/FuncSet.thy --- a/src/HOL/Library/FuncSet.thy Sun Aug 25 20:54:20 2024 +0200 +++ b/src/HOL/Library/FuncSet.thy Sun Aug 25 21:10:01 2024 +0200 @@ -25,6 +25,9 @@ syntax "_Pi" :: "pttrn \ 'a set \ 'b set \ ('a \ 'b) set" ("(3\ _\_./ _)" 10) "_lam" :: "pttrn \ 'a set \ ('a \ 'b) \ ('a \ 'b)" ("(3\_\_./ _)" [0,0,3] 3) +syntax_consts + "_Pi" \ Pi and + "_lam" \ restrict translations "\ x\A. B" \ "CONST Pi A (\x. B)" "\x\A. f" \ "CONST restrict (\x. f) A" @@ -350,6 +353,8 @@ syntax "_PiE" :: "pttrn \ 'a set \ 'b set \ ('a \ 'b) set" ("(3\\<^sub>E _\_./ _)" 10) +syntax_consts + "_PiE" \ Pi\<^sub>E translations "\\<^sub>E x\A. B" \ "CONST Pi\<^sub>E A (\x. B)"