src/HOL/Fun.thy
changeset 69700 7a92cbec7030
parent 69661 a03a63b81f44
child 69735 8230dca028eb
equal deleted inserted replaced
69699:82f57315cade 69700:7a92cbec7030
   179   by (auto simp: inj_on_def)
   179   by (auto simp: inj_on_def)
   180 
   180 
   181 lemma inj_on_strict_subset: "inj_on f B \<Longrightarrow> A \<subset> B \<Longrightarrow> f ` A \<subset> f ` B"
   181 lemma inj_on_strict_subset: "inj_on f B \<Longrightarrow> A \<subset> B \<Longrightarrow> f ` A \<subset> f ` B"
   182   unfolding inj_on_def by blast
   182   unfolding inj_on_def by blast
   183 
   183 
   184 lemma inj_comp: "inj f \<Longrightarrow> inj g \<Longrightarrow> inj (f \<circ> g)"
   184 lemma inj_compose: "inj f \<Longrightarrow> inj g \<Longrightarrow> inj (f \<circ> g)"
   185   by (simp add: inj_def)
   185   by (simp add: inj_def)
   186 
   186 
   187 lemma inj_fun: "inj f \<Longrightarrow> inj (\<lambda>x y. f x)"
   187 lemma inj_fun: "inj f \<Longrightarrow> inj (\<lambda>x y. f x)"
   188   by (simp add: inj_def fun_eq_iff)
   188   by (simp add: inj_def fun_eq_iff)
   189 
   189