src/HOL/Set.thy
changeset 59000 6eb0725503fc
parent 58963 26bf09b95dda
child 59498 50b60f501b05
child 59504 8c6747dba731
equal deleted inserted replaced
58997:fc571ebb04e1 59000:6eb0725503fc
   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