diff -r 46f59511b7bb -r d97fdabd9e2b src/HOL/Analysis/Homotopy.thy --- a/src/HOL/Analysis/Homotopy.thy Fri Sep 20 19:07:10 2024 +0200 +++ b/src/HOL/Analysis/Homotopy.thy Fri Sep 20 19:51:08 2024 +0200 @@ -3340,7 +3340,7 @@ subsection\Homotopy equivalence of topological spaces.\ definition\<^marker>\tag important\ homotopy_equivalent_space - (infix "homotopy'_equivalent'_space" 50) + (infix \homotopy'_equivalent'_space\ 50) where "X homotopy_equivalent_space Y \ (\f g. continuous_map X Y f \ continuous_map Y X g \ @@ -3781,7 +3781,7 @@ abbreviation\<^marker>\tag important\ homotopy_eqv :: "'a::topological_space set \ 'b::topological_space set \ bool" - (infix "homotopy'_eqv" 50) + (infix \homotopy'_eqv\ 50) where "S homotopy_eqv T \ top_of_set S homotopy_equivalent_space top_of_set T" lemma homeomorphic_imp_homotopy_eqv: "S homeomorphic T \ S homotopy_eqv T"