src/HOL/Codatatype/BNF_Library.thy
changeset 49276 59fa53ed7507
parent 49274 ddd606ec45b9
--- a/src/HOL/Codatatype/BNF_Library.thy	Tue Sep 11 13:06:14 2012 +0200
+++ b/src/HOL/Codatatype/BNF_Library.thy	Tue Sep 11 13:06:14 2012 +0200
@@ -843,10 +843,6 @@
   "\<lbrakk>\<forall>x. s = f (Inr (Inl x)) \<longrightarrow> P; \<forall>x. s = f (Inr (Inr x)) \<longrightarrow> P\<rbrakk> \<Longrightarrow> \<forall>x. s = f (Inr x) \<longrightarrow> P"
 by (metis obj_sumE)
 
-lemma sum_map_if:
-"sum_map f g (if p then Inl x else Inr y) = (if p then Inl (f x) else Inr (g y))"
-by simp
-
 lemma sum_case_if:
 "sum_case f g (if p then Inl x else Inr y) = (if p then f x else g y)"
 by simp