src/HOL/Analysis/Bounded_Continuous_Function.thy
changeset 81097 6c81cdca5b82
parent 80914 d97fdabd9e2b
--- 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>\<open>tag important\<close> "bcontfun = {f. continuous_on UNIV f \<and> bounded (range f)}"
 
-typedef (overloaded) ('a, 'b) bcontfun (\<open>(_ \<Rightarrow>\<^sub>C /_)\<close> [22, 21] 21) =
+typedef (overloaded) ('a, 'b) bcontfun (\<open>(\<open>notation=\<open>infix \<Rightarrow>\<^sub>C\<close>\<close>_ \<Rightarrow>\<^sub>C /_)\<close> [22, 21] 21) =
   "bcontfun::('a::topological_space \<Rightarrow> 'b::metric_space) set"
   morphisms apply_bcontfun Bcontfun
   by (auto intro: continuous_intros simp: bounded_def bcontfun_def)