diff -r e43bff789ac0 -r 53e61087bc6f src/HOL/Set.thy --- a/src/HOL/Set.thy Fri Nov 22 14:54:00 2024 +0000 +++ b/src/HOL/Set.thy Fri Nov 22 16:05:42 2024 +0000 @@ -1834,14 +1834,13 @@ lemma the_elem_image_unique: assumes "A \ {}" - and *: "\y. y \ A \ f y = f x" - shows "the_elem (f ` A) = f x" + and *: "\y. y \ A \ f y = a" + shows "the_elem (f ` A) = a" unfolding the_elem_def proof (rule the1_equality) from \A \ {}\ obtain y where "y \ A" by auto - with * have "f x = f y" by simp - with \y \ A\ have "f x \ f ` A" by blast - with * show "f ` A = {f x}" by auto + with * \y \ A\ have "a \ f ` A" by blast + with * show "f ` A = {a}" by auto then show "\!x. f ` A = {x}" by auto qed