src/HOL/Library/Quotient_Sum.thy
changeset 53010 ec5e6f69bd65
parent 51994 82cc2aeb7d13
child 53012 cb82606b8215
--- a/src/HOL/Library/Quotient_Sum.thy	Tue Aug 13 14:20:22 2013 +0200
+++ b/src/HOL/Library/Quotient_Sum.thy	Tue Aug 13 15:59:22 2013 +0200
@@ -50,12 +50,6 @@
   "sum_rel (op =) (op =) = (op =)"
   by (simp add: sum_rel_unfold fun_eq_iff split: sum.split)
 
-lemma split_sum_all: "(\<forall>x. P x) \<longleftrightarrow> (\<forall>x. P (Inl x)) \<and> (\<forall>x. P (Inr x))"
-  by (metis sum.exhaust) (* TODO: move to Sum_Type.thy *)
-
-lemma split_sum_ex: "(\<exists>x. P x) \<longleftrightarrow> (\<exists>x. P (Inl x)) \<or> (\<exists>x. P (Inr x))"
-  by (metis sum.exhaust) (* TODO: move to Sum_Type.thy *)
-
 lemma sum_rel_mono[relator_mono]:
   assumes "A \<le> C"
   assumes "B \<le> D"