src/HOL/Algebra/FiniteProduct.thy
changeset 35054 a5db9779b026
parent 32960 69916a850301
child 35416 d8d7d1b785af
--- a/src/HOL/Algebra/FiniteProduct.thy	Mon Feb 08 21:26:52 2010 +0100
+++ b/src/HOL/Algebra/FiniteProduct.thy	Mon Feb 08 21:28:27 2010 +0100
@@ -302,7 +302,7 @@
   "_finprod" :: "index => idt => 'a set => 'b => 'b"
       ("(3\<Otimes>__\<in>_. _)" [1000, 0, 51, 10] 10)
 translations
-  "\<Otimes>\<index>i:A. b" == "finprod \<struct>\<index> (%i. b) A"
+  "\<Otimes>\<index>i:A. b" == "CONST finprod \<struct>\<index> (%i. b) A"
   -- {* Beware of argument permutation! *}
 
 lemma (in comm_monoid) finprod_empty [simp]: