src/HOL/BNF_FP_Base.thy
changeset 55966 972f0aa7091b
parent 55945 e96383acecf9
child 56640 0a35354137a5
--- a/src/HOL/BNF_FP_Base.thy	Thu Mar 06 22:15:01 2014 +0100
+++ b/src/HOL/BNF_FP_Base.thy	Fri Mar 07 01:02:21 2014 +0100
@@ -28,12 +28,6 @@
 lemma unit_all_impI: "(P () \<Longrightarrow> Q ()) \<Longrightarrow> \<forall>x. P x \<longrightarrow> Q x"
 by simp
 
-lemma prod_all_impI: "(\<And>x y. P (x, y) \<Longrightarrow> Q (x, y)) \<Longrightarrow> \<forall>x. P x \<longrightarrow> Q x"
-by clarify
-
-lemma prod_all_impI_step: "(\<And>x. \<forall>y. P (x, y) \<longrightarrow> Q (x, y)) \<Longrightarrow> \<forall>x. P x \<longrightarrow> Q x"
-by auto
-
 lemma pointfree_idE: "f \<circ> g = id \<Longrightarrow> f (g x) = x"
 unfolding comp_def fun_eq_iff by simp
 
@@ -58,9 +52,6 @@
 "case_sum f (case_sum f' g') (Inr p) = case_sum f' g' p"
 by auto
 
-lemma one_pointE: "\<lbrakk>\<And>x. s = x \<Longrightarrow> P\<rbrakk> \<Longrightarrow> P"
-by simp
-
 lemma obj_one_pointE: "\<forall>x. s = x \<longrightarrow> P \<Longrightarrow> P"
 by blast
 
@@ -76,9 +67,6 @@
   fix x from assms show "s = f x \<longrightarrow> P" by (cases x) auto
 qed
 
-lemma obj_sumE: "\<lbrakk>\<forall>x. s = Inl x \<longrightarrow> P; \<forall>x. s = Inr x \<longrightarrow> P\<rbrakk> \<Longrightarrow> P"
-by (cases s) auto
-
 lemma case_sum_if:
 "case_sum f g (if p then Inl x else Inr y) = (if p then f x else g y)"
 by simp