diff -r c007e6d9941d -r c92efbf32bfe src/HOL/HOL.thy --- a/src/HOL/HOL.thy Tue Oct 01 20:39:16 2024 +0200 +++ b/src/HOL/HOL.thy Tue Oct 01 21:30:59 2024 +0200 @@ -191,11 +191,11 @@ nonterminal case_syn and cases_syn syntax "_case_syntax" :: "['a, cases_syn] \ 'b" (\(\notation=\mixfix case expression\\case _ of/ _)\ 10) - "_case1" :: "['a, 'b] \ case_syn" (\(\indent=2 notation=\mixfix case pattern\\_ \/ _)\ 10) + "_case1" :: "['a, 'b] \ case_syn" (\(\indent=2 notation=\mixfix case clause\\_ \/ _)\ 10) "" :: "case_syn \ cases_syn" (\_\) "_case2" :: "[case_syn, cases_syn] \ cases_syn" (\_/ | _\) syntax (ASCII) - "_case1" :: "['a, 'b] \ case_syn" (\(\indent=2 notation=\mixfix case pattern\\_ =>/ _)\ 10) + "_case1" :: "['a, 'b] \ case_syn" (\(\indent=2 notation=\mixfix case clause\\_ =>/ _)\ 10) notation (ASCII) All (binder \ALL \ 10) and