diff -r 6ce0c8d59f5a -r ec121999a9cb src/ZF/func.thy --- a/src/ZF/func.thy Sun Oct 06 22:56:07 2024 +0200 +++ b/src/ZF/func.thy Tue Oct 08 12:10:35 2024 +0200 @@ -448,10 +448,10 @@ nonterminal updbinds and updbind syntax - "_updbind" :: "[i, i] \ updbind" (\(\indent=2 notation=\infix update\\_ :=/ _)\) - "" :: "updbind \ updbinds" (\_\) - "_updbinds" :: "[updbind, updbinds] \ updbinds" (\_,/ _\) - "_Update" :: "[i, updbinds] \ i" (\_/'((_)')\ [900,0] 900) + "_updbind" :: "[i, i] \ updbind" (\(\indent=2 notation=\infix update\\_ :=/ _)\) + "" :: "updbind \ updbinds" (\_\) + "_updbinds" :: "[updbind, updbinds] \ updbinds" (\_,/ _\) + "_Update" :: "[i, updbinds] \ i" (\(\open_block notation=\mixfix function update\\_/'((_)'))\ [900,0] 900) translations "_Update (f, _updbinds(b,bs))" == "_Update (_Update(f,b), bs)" "f(x:=y)" == "CONST update(f,x,y)"