src/HOL/BNF_Fixpoint_Base.thy
changeset 62158 c25c62055180
parent 61551 078c9fd2e052
child 62325 7e4d31eefe60
--- a/src/HOL/BNF_Fixpoint_Base.thy	Wed Jan 13 00:12:43 2016 +0100
+++ b/src/HOL/BNF_Fixpoint_Base.thy	Wed Jan 13 09:09:37 2016 +0100
@@ -17,11 +17,8 @@
 lemma conj_imp_eq_imp_imp: "(P \<and> Q \<Longrightarrow> PROP R) \<equiv> (P \<Longrightarrow> Q \<Longrightarrow> PROP R)"
   by standard simp_all
 
-lemma mp_conj: "(P \<longrightarrow> Q) \<and> R \<Longrightarrow> P \<Longrightarrow> R \<and> Q"
-  by auto
-
-lemma predicate2D_conj: "P \<le> Q \<and> R \<Longrightarrow> P x y \<Longrightarrow> R \<and> Q x y"
-  by auto
+lemma predicate2D_conj: "P \<le> Q \<and> R \<Longrightarrow> R \<and> (P x y \<longrightarrow> Q x y)"
+  by blast
 
 lemma eq_sym_Unity_conv: "(x = (() = ())) = x"
   by blast