src/HOL/Library/Quotient_Product.thy
changeset 37678 0040bafffdef
parent 36695 b434506fb0d4
child 39198 f967a16dfcdd
--- a/src/HOL/Library/Quotient_Product.thy	Thu Jul 01 16:54:42 2010 +0200
+++ b/src/HOL/Library/Quotient_Product.thy	Thu Jul 01 16:54:44 2010 +0200
@@ -13,7 +13,7 @@
 where
   "prod_rel R1 R2 = (\<lambda>(a, b) (c, d). R1 a c \<and> R2 b d)"
 
-declare [[map * = (prod_fun, prod_rel)]]
+declare [[map prod = (prod_fun, prod_rel)]]
 
 
 lemma prod_equivp[quot_equiv]: