Added lemma
authornipkow
Wed, 02 Apr 2025 16:56:36 +0200
changeset 82394 00a83dd88141
parent 82393 88064da0ae76
child 82395 918c50e0447e
Added lemma
src/HOL/Library/Infinite_Typeclass.thy
--- a/src/HOL/Library/Infinite_Typeclass.thy	Tue Apr 01 12:10:45 2025 +0200
+++ b/src/HOL/Library/Infinite_Typeclass.thy	Wed Apr 02 16:56:36 2025 +0200
@@ -27,6 +27,9 @@
     by auto
 qed
 
+lemma arb_inj_on_finite_infinite: "finite(A :: 'b set) \<Longrightarrow> \<exists>f :: 'b \<Rightarrow> 'a. inj_on f A"
+by (meson arb_finite_subset card_le_inj infinite_imp_nonempty)
+
 lemma arb_countable_map: "finite Y \<Longrightarrow> \<exists>f :: (nat \<Rightarrow> 'a). inj f \<and> range f \<subseteq> UNIV - Y"
   using infinite_UNIV
   by (auto simp: infinite_countable_subset)