src/HOL/Hilbert_Choice.thy
changeset 63807 5f77017055a3
parent 63630 b2a6a1a49d39
child 63980 f8e556c8ad6f
--- a/src/HOL/Hilbert_Choice.thy	Mon Sep 05 23:11:00 2016 +0200
+++ b/src/HOL/Hilbert_Choice.thy	Mon Sep 05 23:39:15 2016 +0200
@@ -244,15 +244,12 @@
 lemma o_inv_distrib: "bij f \<Longrightarrow> bij g \<Longrightarrow> inv (f \<circ> g) = inv g \<circ> inv f"
   by (rule inv_equality) (auto simp add: bij_def surj_f_inv_f)
 
-lemma image_surj_f_inv_f: "surj f \<Longrightarrow> f ` (inv f ` A) = A"
+lemma image_f_inv_f: "surj f \<Longrightarrow> f ` (inv f ` A) = A"
   by (simp add: surj_f_inv_f image_comp comp_def)
 
 lemma image_inv_f_f: "inj f \<Longrightarrow> inv f ` (f ` A) = A"
   by simp
 
-lemma inv_image_comp: "inj f \<Longrightarrow> inv f ` (f ` X) = X"
-  by (fact image_inv_f_f)
-
 lemma bij_image_Collect_eq: "bij f \<Longrightarrow> f ` Collect P = {y. P (inv f y)}"
   apply auto
    apply (force simp add: bij_is_inj)