bij <--> bij_betw
authorhoelzl
Thu, 02 Sep 2010 10:36:45 +0200
changeset 39074 211e4f6aad63
parent 39073 8520a1f89db1
child 39075 a18e5946d63c
bij <--> bij_betw
src/HOL/Fun.thy
--- a/src/HOL/Fun.thy	Thu Sep 02 10:18:15 2010 +0200
+++ b/src/HOL/Fun.thy	Thu Sep 02 10:36:45 2010 +0200
@@ -262,6 +262,15 @@
 apply (drule_tac x = x in spec, blast)
 done
 
+lemma surj_range_iff: "surj f \<longleftrightarrow> range f = UNIV"
+  unfolding expand_set_eq image_iff surj_def by auto
+
+lemma bij_betw_imp_surj: "bij_betw f A UNIV \<Longrightarrow> surj f"
+  unfolding bij_betw_def surj_range_iff by auto
+
+lemma bij_eq_bij_betw: "bij f \<longleftrightarrow> bij_betw f UNIV UNIV"
+  unfolding bij_def surj_range_iff bij_betw_def ..
+
 lemma bijI: "[| inj f; surj f |] ==> bij f"
 by (simp add: bij_def)