src/HOL/Analysis/Locally.thy
changeset 80914 d97fdabd9e2b
parent 78480 b22f39c54e8c
--- 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\<open>Basic definition of the small inductive dimension relation. Works in any topological space.\<close>
 
-inductive dimension_le :: "['a topology, int] \<Rightarrow> bool" (infix "dim'_le" 50) 
+inductive dimension_le :: "['a topology, int] \<Rightarrow> bool" (infix \<open>dim'_le\<close> 50) 
   where "\<lbrakk>-1 \<le> n;
         \<And>V a. \<lbrakk>openin X V; a \<in> V\<rbrakk> \<Longrightarrow> \<exists>U. a \<in> U \<and> U \<subseteq> V \<and> openin X U \<and> (subtopology X (X frontier_of U)) dim_le (n-1)\<rbrakk>
               \<Longrightarrow> X dim_le (n::int)"