Skip to content

Commit

Permalink
feat: two missing lemmas about restricting continuous maps (#6616)
Browse files Browse the repository at this point in the history
  • Loading branch information
ADedecker committed Aug 19, 2023
1 parent 0a3c012 commit a0d8b86
Showing 1 changed file with 13 additions and 2 deletions.
15 changes: 13 additions & 2 deletions Mathlib/Topology/Constructions.lean
Expand Up @@ -1099,9 +1099,10 @@ theorem closure_subtype {x : { a // p a }} {s : Set { a // p a }} :
closure_induced
#align closure_subtype closure_subtype

@[simp]
theorem continuousAt_codRestrict_iff {f : α → β} {t : Set β} (h1 : ∀ x, f x ∈ t) {x : α} :
ContinuousAt (codRestrict f t h1) x ↔ ContinuousAt f x := by
simp_rw [inducing_subtype_val.continuousAt_iff, Function.comp, val_codRestrict_apply]
ContinuousAt (codRestrict f t h1) x ↔ ContinuousAt f x :=
inducing_subtype_val.continuousAt_iff
#align continuous_at_cod_restrict_iff continuousAt_codRestrict_iff

alias continuousAt_codRestrict_iff ↔ _ ContinuousAt.codRestrict
Expand All @@ -1123,6 +1124,16 @@ theorem Continuous.codRestrict {f : α → β} {s : Set β} (hf : Continuous f)
hf.subtype_mk hs
#align continuous.cod_restrict Continuous.codRestrict

@[continuity]
theorem Continuous.restrict {f : α → β} {s : Set α} {t : Set β} (h1 : MapsTo f s t)
(h2 : Continuous f) : Continuous (h1.restrict f s t) :=
(h2.comp continuous_subtype_val).codRestrict _

@[continuity]
theorem Continuous.restrictPreimage {f : α → β} {s : Set β} (h : Continuous f) :
Continuous (s.restrictPreimage f) :=
h.restrict _

theorem Inducing.codRestrict {e : α → β} (he : Inducing e) {s : Set β} (hs : ∀ x, e x ∈ s) :
Inducing (codRestrict e s hs) :=
inducing_of_inducing_compose (he.continuous.codRestrict hs) continuous_subtype_val he
Expand Down

0 comments on commit a0d8b86

Please sign in to comment.