src/HOL/Hahn_Banach/Subspace.thy
changeset 80914 d97fdabd9e2b
parent 66453 cc19f7ca2ed6
child 81464 2575f1bd226b
--- a/src/HOL/Hahn_Banach/Subspace.thy	Fri Sep 20 19:07:10 2024 +0200
+++ b/src/HOL/Hahn_Banach/Subspace.thy	Fri Sep 20 19:51:08 2024 +0200
@@ -23,7 +23,7 @@
     and mult_closed [iff]: "x \<in> U \<Longrightarrow> a \<cdot> x \<in> U"
 
 notation (symbols)
-  subspace  (infix "\<unlhd>" 50)
+  subspace  (infix \<open>\<unlhd>\<close> 50)
 
 declare vectorspace.intro [intro?] subspace.intro [intro?]