Documentation

Mathlib.Topology.Algebra.Indicator

Continuity of indicator functions #

theorem continuous_mulIndicator {α : Type u_1} {β : Type u_2} [TopologicalSpace α] [TopologicalSpace β] {f : αβ} {s : Set α} [One β] (hs : afrontier s, f a = 1) (hf : ContinuousOn f (closure s)) :
theorem continuous_indicator {α : Type u_1} {β : Type u_2} [TopologicalSpace α] [TopologicalSpace β] {f : αβ} {s : Set α} [Zero β] (hs : afrontier s, f a = 0) (hf : ContinuousOn f (closure s)) :
theorem Continuous.mulIndicator {α : Type u_1} {β : Type u_2} [TopologicalSpace α] [TopologicalSpace β] {f : αβ} {s : Set α} [One β] (hs : afrontier s, f a = 1) (hf : Continuous f) :
theorem Continuous.indicator {α : Type u_1} {β : Type u_2} [TopologicalSpace α] [TopologicalSpace β] {f : αβ} {s : Set α} [Zero β] (hs : afrontier s, f a = 0) (hf : Continuous f) :
theorem ContinuousOn.continuousAt_mulIndicator {α : Type u_1} {β : Type u_2} [TopologicalSpace α] [TopologicalSpace β] {f : αβ} {s : Set α} [One β] (hf : ContinuousOn f (interior s)) {x : α} (hx : xfrontier s) :
theorem ContinuousOn.continuousAt_indicator {α : Type u_1} {β : Type u_2} [TopologicalSpace α] [TopologicalSpace β] {f : αβ} {s : Set α} [Zero β] (hf : ContinuousOn f (interior s)) {x : α} (hx : xfrontier s) :
theorem IsClopen.continuous_mulIndicator {α : Type u_1} {β : Type u_2} [TopologicalSpace α] [TopologicalSpace β] {f : αβ} {s : Set α} [One β] (hs : IsClopen s) (hf : Continuous f) :
theorem IsClopen.continuous_indicator {α : Type u_1} {β : Type u_2} [TopologicalSpace α] [TopologicalSpace β] {f : αβ} {s : Set α} [Zero β] (hs : IsClopen s) (hf : Continuous f) :