src/HOL/Algebra/FiniteProduct.thy
changeset 80914 d97fdabd9e2b
parent 80768 c7723cc15de8
child 81142 6ad2c917dd2e
--- a/src/HOL/Algebra/FiniteProduct.thy	Fri Sep 20 19:07:10 2024 +0200
+++ b/src/HOL/Algebra/FiniteProduct.thy	Fri Sep 20 19:51:08 2024 +0200
@@ -66,7 +66,7 @@
 locale LCD =
   fixes B :: "'b set"
   and D :: "'a set"
-  and f :: "'b \<Rightarrow> 'a \<Rightarrow> 'a"    (infixl "\<cdot>" 70)
+  and f :: "'b \<Rightarrow> 'a \<Rightarrow> 'a"    (infixl \<open>\<cdot>\<close> 70)
   assumes left_commute:
     "\<lbrakk>x \<in> B; y \<in> B; z \<in> D\<rbrakk> \<Longrightarrow> x \<cdot> (y \<cdot> z) = y \<cdot> (x \<cdot> z)"
   and f_closed [simp, intro!]: "!!x y. \<lbrakk>x \<in> B; y \<in> D\<rbrakk> \<Longrightarrow> f x y \<in> D"
@@ -246,7 +246,7 @@
 
 locale ACeD =
   fixes D :: "'a set"
-    and f :: "'a \<Rightarrow> 'a \<Rightarrow> 'a"    (infixl "\<cdot>" 70)
+    and f :: "'a \<Rightarrow> 'a \<Rightarrow> 'a"    (infixl \<open>\<cdot>\<close> 70)
     and e :: 'a
   assumes ident [simp]: "x \<in> D \<Longrightarrow> x \<cdot> e = x"
     and commute: "\<lbrakk>x \<in> D; y \<in> D\<rbrakk> \<Longrightarrow> x \<cdot> y = y \<cdot> x"
@@ -307,7 +307,7 @@
 
 syntax
   "_finprod" :: "index \<Rightarrow> idt \<Rightarrow> 'a set \<Rightarrow> 'b \<Rightarrow> 'b"
-      ("(3\<Otimes>__\<in>_. _)" [1000, 0, 51, 10] 10)
+      (\<open>(3\<Otimes>__\<in>_. _)\<close> [1000, 0, 51, 10] 10)
 syntax_consts
   "_finprod" \<rightleftharpoons> finprod
 translations