src/HOL/Hilbert_Choice.thy
changeset 67613 ce654b0e6d69
parent 65955 0616ba637b14
child 67673 c8caefb20564
--- a/src/HOL/Hilbert_Choice.thy	Tue Feb 13 14:24:50 2018 +0100
+++ b/src/HOL/Hilbert_Choice.thy	Thu Feb 15 12:11:00 2018 +0100
@@ -144,7 +144,7 @@
 lemma inv_f_f: "inj f \<Longrightarrow> inv f (f x) = x"
   by simp
 
-lemma f_inv_into_f: "y : f`A \<Longrightarrow> f (inv_into A f y) = y"
+lemma f_inv_into_f: "y \<in> f`A \<Longrightarrow> f (inv_into A f y) = y"
   by (simp add: inv_into_def) (fast intro: someI2)
 
 lemma inv_into_f_eq: "inj_on f A \<Longrightarrow> x \<in> A \<Longrightarrow> f x = y \<Longrightarrow> inv_into A f y = x"