src/HOL/Library/RBT_Impl.thy
changeset 80914 d97fdabd9e2b
parent 77061 5de3772609ea
--- a/src/HOL/Library/RBT_Impl.thy	Fri Sep 20 19:07:10 2024 +0200
+++ b/src/HOL/Library/RBT_Impl.thy	Fri Sep 20 19:51:08 2024 +0200
@@ -74,10 +74,10 @@
 where
   rbt_less_prop: "rbt_less k t \<longleftrightarrow> (\<forall>x\<in>set (keys t). x < k)"
 
-abbreviation rbt_less_symbol (infix "|\<guillemotleft>" 50)
+abbreviation rbt_less_symbol (infix \<open>|\<guillemotleft>\<close> 50)
 where "t |\<guillemotleft> x \<equiv> rbt_less x t"
 
-definition rbt_greater :: "'a \<Rightarrow> ('a, 'b) rbt \<Rightarrow> bool" (infix "\<guillemotleft>|" 50) 
+definition rbt_greater :: "'a \<Rightarrow> ('a, 'b) rbt \<Rightarrow> bool" (infix \<open>\<guillemotleft>|\<close> 50) 
 where
   rbt_greater_prop: "rbt_greater k t = (\<forall>x\<in>set (keys t). k < x)"