src/HOL/Algebra/AbelCoset.thy
changeset 45006 11a542f50fc3
parent 44655 fe0365331566
child 45388 121b2db078b1
--- a/src/HOL/Algebra/AbelCoset.thy	Mon Sep 19 23:18:18 2011 +0200
+++ b/src/HOL/Algebra/AbelCoset.thy	Mon Sep 19 23:24:32 2011 +0200
@@ -36,7 +36,7 @@
   where "A_SET_INV G H = SET_INV \<lparr>carrier = carrier G, mult = add G, one = zero G\<rparr> H"
 
 definition
-  a_r_congruent :: "[('a,'b)ring_scheme, 'a set] \<Rightarrow> ('a*'a)set"  ("racong\<index> _")
+  a_r_congruent :: "[('a,'b)ring_scheme, 'a set] \<Rightarrow> ('a*'a)set"  ("racong\<index>")
   where "a_r_congruent G = r_congruent \<lparr>carrier = carrier G, mult = add G, one = zero G\<rparr>"
 
 definition