src/HOL/Algebra/Embedded_Algebras.thy
changeset 80914 d97fdabd9e2b
parent 70160 8e9100dcde52
child 81438 95c9af7483b1
--- a/src/HOL/Algebra/Embedded_Algebras.thy	Fri Sep 20 19:07:10 2024 +0200
+++ b/src/HOL/Algebra/Embedded_Algebras.thy	Fri Sep 20 19:51:08 2024 +0200
@@ -38,7 +38,7 @@
 abbreviation (in ring) dependent ::  "'a set \<Rightarrow> 'a list \<Rightarrow> bool"
   where "dependent K U \<equiv> \<not> independent K U"
 
-definition over :: "('a \<Rightarrow> 'b) \<Rightarrow> 'a \<Rightarrow> 'b" (infixl "over" 65)
+definition over :: "('a \<Rightarrow> 'b) \<Rightarrow> 'a \<Rightarrow> 'b" (infixl \<open>over\<close> 65)
   where "f over a = f a"