src/HOL/Algebra/FiniteProduct.thy
changeset 62105 686681f69d5e
parent 61384 9f5145281888
child 63167 0909deb8059b
--- a/src/HOL/Algebra/FiniteProduct.thy	Fri Jan 08 18:18:40 2016 +0100
+++ b/src/HOL/Algebra/FiniteProduct.thy	Fri Jan 08 19:46:30 2016 +0100
@@ -298,7 +298,7 @@
   "_finprod" :: "index => idt => 'a set => 'b => 'b"
       ("(3\<Otimes>__\<in>_. _)" [1000, 0, 51, 10] 10)
 translations
-  "\<Otimes>\<index>i\<in>A. b" \<rightleftharpoons> "CONST finprod \<struct>\<index> (%i. b) A"
+  "\<Otimes>\<^bsub>G\<^esub>i\<in>A. b" \<rightleftharpoons> "CONST finprod G (%i. b) A"
   -- \<open>Beware of argument permutation!\<close>
 
 lemma (in comm_monoid) finprod_empty [simp]: