src/HOL/Basic_BNFs.thy
changeset 58446 e89f57d1e46c
parent 56077 d397030fb27e
child 58889 5b7a9633cfa8
--- a/src/HOL/Basic_BNFs.thy	Thu Sep 25 16:35:51 2014 +0200
+++ b/src/HOL/Basic_BNFs.thy	Thu Sep 25 16:35:53 2014 +0200
@@ -21,14 +21,6 @@
 
 lemmas sum_set_defs = setl_def[abs_def] setr_def[abs_def]
 
-definition
-   rel_sum :: "('a \<Rightarrow> 'c \<Rightarrow> bool) \<Rightarrow> ('b \<Rightarrow> 'd \<Rightarrow> bool) \<Rightarrow> 'a + 'b \<Rightarrow> 'c + 'd \<Rightarrow> bool"
-where
-   "rel_sum R1 R2 x y =
-     (case (x, y) of (Inl x, Inl y) \<Rightarrow> R1 x y
-     | (Inr x, Inr y) \<Rightarrow> R2 x y
-     | _ \<Rightarrow> False)"
-
 lemma rel_sum_simps[simp]:
   "rel_sum R1 R2 (Inl a1) (Inl b1) = R1 a1 b1"
   "rel_sum R1 R2 (Inl a1) (Inr b2) = False"