Zulip Chat Archive

Stream: Is there code for X?

Topic: Continuity and inducing


Thomas Browning (Aug 30 2022 at 04:53):

Is this lemma in mathlib, or is there an easier proof using mathlib?

import topology.order

example (W X Y Z : Type*) [topological_space W] [topological_space X] [topological_space Y]
  [topological_space Z] (f : X  Y) (g : W  Z) (i : W  X) (j : Z  Y)
  (hi : inducing i) (hj : inducing j) (h : f  i = j  g) (hg : continuous f) :
  continuous g :=
begin
  rw [continuous_iff_le_induced, hj.induced, induced_compose, h, induced_compose],
  rw continuous_iff_le_induced at hg,
  rw hi.induced,
  exact induced_mono hg,
end

Patrick Massot (Aug 30 2022 at 07:27):

example (W X Y Z : Type*) [topological_space W] [topological_space X] [topological_space Y]
  [topological_space Z] (f : X  Y) (g : W  Z) (i : W  X) (j : Z  Y)
  (hi : inducing i) (hj : inducing j) (h : f  i = j  g) (hg : continuous f) :
  continuous g :=
begin
  rw [hj.continuous_iff,  h],
  exact hg.comp hi.continuous,
end

Patrick Massot (Aug 30 2022 at 07:27):

It would have been faster if hg had been named hf

Patrick Massot (Aug 30 2022 at 07:28):

Also note the assumption on i is way too strong, continuity is enough.


Last updated: Dec 20 2023 at 11:08 UTC