diff -r e957b2dd8983 -r 6c81cdca5b82 src/HOL/Analysis/Bounded_Continuous_Function.thy --- a/src/HOL/Analysis/Bounded_Continuous_Function.thy Wed Oct 02 10:34:41 2024 +0200 +++ b/src/HOL/Analysis/Bounded_Continuous_Function.thy Wed Oct 02 10:35:44 2024 +0200 @@ -10,7 +10,7 @@ definition\<^marker>\tag important\ "bcontfun = {f. continuous_on UNIV f \ bounded (range f)}" -typedef (overloaded) ('a, 'b) bcontfun (\(_ \\<^sub>C /_)\ [22, 21] 21) = +typedef (overloaded) ('a, 'b) bcontfun (\(\notation=\infix \\<^sub>C\\_ \\<^sub>C /_)\ [22, 21] 21) = "bcontfun::('a::topological_space \ 'b::metric_space) set" morphisms apply_bcontfun Bcontfun by (auto intro: continuous_intros simp: bounded_def bcontfun_def)