diff -r 46f59511b7bb -r d97fdabd9e2b src/HOL/Analysis/Abstract_Topology_2.thy --- a/src/HOL/Analysis/Abstract_Topology_2.thy Fri Sep 20 19:07:10 2024 +0200 +++ b/src/HOL/Analysis/Abstract_Topology_2.thy Fri Sep 20 19:51:08 2024 +0200 @@ -311,7 +311,7 @@ subsection\<^marker>\tag unimportant\ \A function constant on a set\ -definition constant_on (infixl "(constant'_on)" 50) +definition constant_on (infixl \(constant'_on)\ 50) where "f constant_on A \ \y. \x\A. f x = y" lemma constant_on_subset: "\f constant_on A; B \ A\ \ f constant_on B" @@ -892,7 +892,7 @@ where "retraction S T r \ T \ S \ continuous_on S r \ r \ S \ T \ (\x\T. r x = x)" -definition\<^marker>\tag important\ retract_of (infixl "retract'_of" 50) where +definition\<^marker>\tag important\ retract_of (infixl \retract'_of\ 50) where "T retract_of S \ (\r. retraction S T r)" lemma retraction_idempotent: "retraction S T r \ x \ S \ r (r x) = r x" @@ -1111,7 +1111,7 @@ subsection\Retractions on a topological space\ -definition retract_of_space :: "'a set \ 'a topology \ bool" (infix "retract'_of'_space" 50) +definition retract_of_space :: "'a set \ 'a topology \ bool" (infix \retract'_of'_space\ 50) where "S retract_of_space X \ S \ topspace X \ (\r. continuous_map X (subtopology X S) r \ (\x \ S. r x = x))"