equal
deleted
inserted
replaced
476 lemma strong_bex_cong [cong]: |
476 lemma strong_bex_cong [cong]: |
477 "A = B ==> (!!x. x:B =simp=> P x = Q x) ==> |
477 "A = B ==> (!!x. x:B =simp=> P x = Q x) ==> |
478 (EX x:A. P x) = (EX x:B. Q x)" |
478 (EX x:A. P x) = (EX x:B. Q x)" |
479 by (simp add: simp_implies_def Bex_def cong: conj_cong) |
479 by (simp add: simp_implies_def Bex_def cong: conj_cong) |
480 |
480 |
|
481 lemma bex1_def: "(\<exists>!x\<in>X. P x) \<longleftrightarrow> (\<exists>x\<in>X. P x) \<and> (\<forall>x\<in>X. \<forall>y\<in>X. P x \<longrightarrow> P y \<longrightarrow> x = y)" |
|
482 by auto |
481 |
483 |
482 subsection {* Basic operations *} |
484 subsection {* Basic operations *} |
483 |
485 |
484 subsubsection {* Subsets *} |
486 subsubsection {* Subsets *} |
485 |
487 |