src/HOL/Library/Pattern_Aliases.thy
changeset 80914 d97fdabd9e2b
parent 80874 9af593e9e454
--- a/src/HOL/Library/Pattern_Aliases.thy	Fri Sep 20 19:07:10 2024 +0200
+++ b/src/HOL/Library/Pattern_Aliases.thy	Fri Sep 20 19:51:08 2024 +0200
@@ -160,7 +160,7 @@
 
 bundle pattern_aliases begin
 
-  notation as (infixr "=:" 1)
+  notation as (infixr \<open>=:\<close> 1)
 
   declaration \<open>K (Syntax_Phases.term_check 98 "pattern_syntax" (K (map check_pattern_syntax)))\<close>
   declaration \<open>K (Syntax_Phases.term_uncheck 98 "pattern_syntax" (map o uncheck_pattern_syntax))\<close>