Zulip Chat Archive
Stream: Is there code for X?
Topic: Image equals image after surjection
Pedro Minicz (Jul 13 2022 at 17:53):
Do we have the following in mathlib? I looked for it but I nor library_search
could find it.
import data.set.basic
example {α β γ : Type*} (f : β → α) {g : γ → β} :
function.surjective g → set.range f = set.range (f ∘ g) :=
begin
intro hg,
ext a,
split; intro h,
{ rcases h with ⟨b, rfl⟩,
specialize hg b,
rcases hg with ⟨c, rfl⟩,
exact ⟨c, rfl⟩ },
{ rcases h with ⟨c, rfl⟩,
exact ⟨g c, rfl⟩ }
end
Yaël Dillies (Jul 13 2022 at 18:00):
You can get there faster using docs#set.range_comp
Last updated: Dec 20 2023 at 11:08 UTC