diff -r 6ce0c8d59f5a -r ec121999a9cb src/HOL/GCD.thy --- a/src/HOL/GCD.thy Sun Oct 06 22:56:07 2024 +0200 +++ b/src/HOL/GCD.thy Tue Oct 08 12:10:35 2024 +0200 @@ -2851,7 +2851,7 @@ definition (in semiring_1) semiring_char :: "'a itself \ nat" where "semiring_char _ = Gcd {n. of_nat n = (0 :: 'a)}" -syntax "_type_char" :: "type => nat" (\(\indent=1 notation=\prefix CHAR\\CHAR/(1'(_')))\) +syntax "_type_char" :: "type => nat" (\(\indent=1 notation=\mixfix CHAR\\CHAR/(1'(_')))\) syntax_consts "_type_char" \ semiring_char translations "CHAR('t)" \ "CONST semiring_char (CONST Pure.type :: 't itself)" print_translation \