src/HOL/Computational_Algebra/Formal_Laurent_Series.thy
changeset 80914 d97fdabd9e2b
parent 80175 200107cdd3ac
child 81107 ad5fc948e053
--- a/src/HOL/Computational_Algebra/Formal_Laurent_Series.thy	Fri Sep 20 19:07:10 2024 +0200
+++ b/src/HOL/Computational_Algebra/Formal_Laurent_Series.thy	Fri Sep 20 19:51:08 2024 +0200
@@ -26,7 +26,7 @@
 setup_lifting type_definition_fls
 
 unbundle fps_notation
-notation fls_nth (infixl "$$" 75)
+notation fls_nth (infixl \<open>$$\<close> 75)
 
 lemmas fls_eqI = iffD1[OF fls_nth_inject, OF iffD2, OF fun_eq_iff, OF allI]
 
@@ -4601,11 +4601,11 @@
 
 subsection \<open>Notation\<close>
 
-no_notation fls_nth (infixl "$$" 75)
+no_notation fls_nth (infixl \<open>$$\<close> 75)
 
 bundle fls_notation
 begin
-notation fls_nth (infixl "$$" 75)
+notation fls_nth (infixl \<open>$$\<close> 75)
 end
 
 end
\ No newline at end of file