src/HOL/Algebra/Ideal_Product.thy
changeset 80914 d97fdabd9e2b
parent 75963 884dbbc8e1b3
child 81438 95c9af7483b1
--- a/src/HOL/Algebra/Ideal_Product.thy	Fri Sep 20 19:07:10 2024 +0200
+++ b/src/HOL/Algebra/Ideal_Product.thy	Fri Sep 20 19:51:08 2024 +0200
@@ -11,7 +11,7 @@
 text \<open>In this section, we study the structure of the set of ideals of a given ring.\<close>
 
 inductive_set
-  ideal_prod :: "[ ('a, 'b) ring_scheme, 'a set, 'a set ] \<Rightarrow> 'a set" (infixl "\<cdot>\<index>" 80)
+  ideal_prod :: "[ ('a, 'b) ring_scheme, 'a set, 'a set ] \<Rightarrow> 'a set" (infixl \<open>\<cdot>\<index>\<close> 80)
   for R and I and J (* both I and J are supposed ideals *) where
     prod: "\<lbrakk> i \<in> I; j \<in> J \<rbrakk> \<Longrightarrow> i \<otimes>\<^bsub>R\<^esub> j \<in> ideal_prod R I J"
   |  sum: "\<lbrakk> s1 \<in> ideal_prod R I J; s2 \<in> ideal_prod R I J \<rbrakk> \<Longrightarrow> s1 \<oplus>\<^bsub>R\<^esub> s2 \<in> ideal_prod R I J"