src/HOL/Library/Quotient_Sum.thy
changeset 40542 9a173a22771c
parent 40465 2989f9f3aa10
child 40610 70776ecfe324
--- a/src/HOL/Library/Quotient_Sum.thy	Mon Nov 15 14:14:38 2010 +0100
+++ b/src/HOL/Library/Quotient_Sum.thy	Mon Nov 15 14:59:21 2010 +0100
@@ -9,7 +9,7 @@
 begin
 
 fun
-  sum_rel :: "('a \<Rightarrow> 'a \<Rightarrow> bool) \<Rightarrow> ('b \<Rightarrow> 'b \<Rightarrow> bool) \<Rightarrow> 'a + 'b \<Rightarrow> 'a + 'b \<Rightarrow> bool"
+  sum_rel :: "('a \<Rightarrow> 'c \<Rightarrow> bool) \<Rightarrow> ('b \<Rightarrow> 'd \<Rightarrow> bool) \<Rightarrow> 'a + 'b \<Rightarrow> 'c + 'd \<Rightarrow> bool"
 where
   "sum_rel R1 R2 (Inl a1) (Inl b1) = R1 a1 b1"
 | "sum_rel R1 R2 (Inl a1) (Inr b2) = False"