diff -r e957b2dd8983 -r 6c81cdca5b82 src/HOL/Analysis/Bounded_Linear_Function.thy --- a/src/HOL/Analysis/Bounded_Linear_Function.thy Wed Oct 02 10:34:41 2024 +0200 +++ b/src/HOL/Analysis/Bounded_Linear_Function.thy Wed Oct 02 10:35:44 2024 +0200 @@ -116,7 +116,7 @@ subsection \Type of bounded linear functions\ -typedef\<^marker>\tag important\ (overloaded) ('a, 'b) blinfun (\(_ \\<^sub>L /_)\ [22, 21] 21) = +typedef\<^marker>\tag important\ (overloaded) ('a, 'b) blinfun (\(\notation=\infix \\<^sub>L\\_ \\<^sub>L /_)\ [22, 21] 21) = "{f::'a::real_normed_vector\'b::real_normed_vector. bounded_linear f}" morphisms blinfun_apply Blinfun by (blast intro: bounded_linear_intros)