src/HOL/Library/FuncSet.thy
changeset 14745 94be403deb84
parent 14706 71590b7733b7
child 14762 bd349ff7907a
equal deleted inserted replaced
14744:7ccfc167e451 14745:94be403deb84
   163   apply (simp add: compose_def)
   163   apply (simp add: compose_def)
   164   apply (rule restrict_ext)
   164   apply (rule restrict_ext)
   165   apply (simp add: f_Inv_f)
   165   apply (simp add: f_Inv_f)
   166   done
   166   done
   167 
   167 
       
   168 
       
   169 subsection{*Cardinality*}
       
   170 
       
   171 lemma card_inj: "[|f \<in> A\<rightarrow>B; inj_on f A; finite B|] ==> card(A) \<le> card(B)"
       
   172 apply (rule card_inj_on_le)
       
   173 apply (auto simp add: Pi_def)
       
   174 done
       
   175 
       
   176 lemma card_bij:
       
   177      "[|f \<in> A\<rightarrow>B; inj_on f A;
       
   178         g \<in> B\<rightarrow>A; inj_on g B; finite A; finite B|] ==> card(A) = card(B)"
       
   179 by (blast intro: card_inj order_antisym)
       
   180 
   168 end
   181 end