diff -r 46f59511b7bb -r d97fdabd9e2b src/HOL/Analysis/Locally.thy --- a/src/HOL/Analysis/Locally.thy Fri Sep 20 19:07:10 2024 +0200 +++ b/src/HOL/Analysis/Locally.thy Fri Sep 20 19:51:08 2024 +0200 @@ -945,7 +945,7 @@ text\Basic definition of the small inductive dimension relation. Works in any topological space.\ -inductive dimension_le :: "['a topology, int] \ bool" (infix "dim'_le" 50) +inductive dimension_le :: "['a topology, int] \ bool" (infix \dim'_le\ 50) where "\-1 \ n; \V a. \openin X V; a \ V\ \ \U. a \ U \ U \ V \ openin X U \ (subtopology X (X frontier_of U)) dim_le (n-1)\ \ X dim_le (n::int)"