diff -r e957b2dd8983 -r 6c81cdca5b82 src/HOL/Analysis/Infinite_Set_Sum.thy --- a/src/HOL/Analysis/Infinite_Set_Sum.thy Wed Oct 02 10:34:41 2024 +0200 +++ b/src/HOL/Analysis/Infinite_Set_Sum.thy Wed Oct 02 10:35:44 2024 +0200 @@ -96,10 +96,10 @@ syntax (ASCII) "_infsetsum" :: "pttrn \ 'a set \ 'b \ 'b::{banach, second_countable_topology}" - (\(3INFSETSUM _:_./ _)\ [0, 51, 10] 10) + (\(\indent=3 notation=\binder INFSETSUM\\INFSETSUM _:_./ _)\ [0, 51, 10] 10) syntax "_infsetsum" :: "pttrn \ 'a set \ 'b \ 'b::{banach, second_countable_topology}" - (\(2\\<^sub>a_\_./ _)\ [0, 51, 10] 10) + (\(\indent=2 notation=\binder \\<^sub>a\\\\<^sub>a_\_./ _)\ [0, 51, 10] 10) syntax_consts "_infsetsum" \ infsetsum translations \ \Beware of argument permutation!\ @@ -107,10 +107,10 @@ syntax (ASCII) "_uinfsetsum" :: "pttrn \ 'a set \ 'b \ 'b::{banach, second_countable_topology}" - (\(3INFSETSUM _:_./ _)\ [0, 51, 10] 10) + (\(\indent=3 notation=\binder INFSETSUM\\INFSETSUM _:_./ _)\ [0, 51, 10] 10) syntax "_uinfsetsum" :: "pttrn \ 'b \ 'b::{banach, second_countable_topology}" - (\(2\\<^sub>a_./ _)\ [0, 10] 10) + (\(\indent=2 notation=\binder \\<^sub>a\\\\<^sub>a_./ _)\ [0, 10] 10) syntax_consts "_uinfsetsum" \ infsetsum translations \ \Beware of argument permutation!\ @@ -118,10 +118,10 @@ syntax (ASCII) "_qinfsetsum" :: "pttrn \ bool \ 'a \ 'a::{banach, second_countable_topology}" - (\(3INFSETSUM _ |/ _./ _)\ [0, 0, 10] 10) + (\(\indent=3 notation=\binder INFSETSUM\\INFSETSUM _ |/ _./ _)\ [0, 0, 10] 10) syntax "_qinfsetsum" :: "pttrn \ bool \ 'a \ 'a::{banach, second_countable_topology}" - (\(2\\<^sub>a_ | (_)./ _)\ [0, 0, 10] 10) + (\(\indent=2 notation=\binder \\<^sub>a\\\\<^sub>a_ | (_)./ _)\ [0, 0, 10] 10) syntax_consts "_qinfsetsum" \ infsetsum translations