src/HOL/Library/Quotient_Product.thy
changeset 40541 7850b4cc1507
parent 40465 2989f9f3aa10
child 40607 30d512bf47a7
--- a/src/HOL/Library/Quotient_Product.thy	Mon Nov 15 00:20:36 2010 +0100
+++ b/src/HOL/Library/Quotient_Product.thy	Mon Nov 15 14:14:38 2010 +0100
@@ -9,7 +9,7 @@
 begin
 
 definition
-  prod_rel :: "('a \<Rightarrow> 'a \<Rightarrow> bool) \<Rightarrow> ('b \<Rightarrow> 'b \<Rightarrow> bool) \<Rightarrow> 'a \<times> 'b \<Rightarrow> 'a \<times> 'b \<Rightarrow> bool"
+  prod_rel :: "('a \<Rightarrow> 'b \<Rightarrow> bool) \<Rightarrow> ('c \<Rightarrow> 'd \<Rightarrow> bool) \<Rightarrow> 'a \<times> 'c \<Rightarrow> 'b \<times> 'd \<Rightarrow> bool"
 where
   "prod_rel R1 R2 = (\<lambda>(a, b) (c, d). R1 a c \<and> R2 b d)"