Documentation

Mathlib.Topology.Hom.ContinuousEval

Bundled maps with evaluation continuous in both variables #

In this file we define a class ContinuousEval F X Y saying that F is a bundled morphism class (in the sense of FunLike) with a topology such that fun (f, x) : F × X ↦ f x is a continuous function.

class ContinuousEval (F : Type u_1) (X : outParam (Type u_2)) (Y : outParam (Type u_3)) [FunLike F X Y] [TopologicalSpace F] [TopologicalSpace X] [TopologicalSpace Y] :

A typeclass saying that F is a bundled morphism class (in the sense of FunLike) with a topology such that fun (f, x) : F × X ↦ f x is a continuous function.

  • continuous_eval : Continuous fun (fx : F × X) => fx.1 fx.2

    Evaluation of a bundled morphism at a point is continuous in both variables.

Instances
    theorem ContinuousEval.continuous_eval {F : Type u_1} {X : outParam (Type u_2)} {Y : outParam (Type u_3)} :
    ∀ {inst : FunLike F X Y} {inst_1 : TopologicalSpace F} {inst_2 : TopologicalSpace X} {inst_3 : TopologicalSpace Y} [self : ContinuousEval F X Y], Continuous fun (fx : F × X) => fx.1 fx.2

    Evaluation of a bundled morphism at a point is continuous in both variables.

    theorem Continuous.eval {F : Type u_1} {X : Type u_2} {Y : Type u_3} {Z : Type u_4} [FunLike F X Y] [TopologicalSpace F] [TopologicalSpace X] [TopologicalSpace Y] [ContinuousEval F X Y] [TopologicalSpace Z] {f : ZF} {g : ZX} (hf : Continuous f) (hg : Continuous g) :
    Continuous fun (z : Z) => (f z) (g z)
    theorem ContinuousEval.of_continuous_forget {F : Type u_1} {X : Type u_2} {Y : Type u_3} [FunLike F X Y] [TopologicalSpace F] [TopologicalSpace X] [TopologicalSpace Y] [ContinuousEval F X Y] {F' : Type u_5} [FunLike F' X Y] [TopologicalSpace F'] {f : F'F} (hc : Continuous f) (hf : autoParam (∀ (g : F'), (f g) = g) _auto✝) :

    If a type F' of bundled morphisms admits a continuous projection to a type satisfying ContinuousEval, then F' satisfies this predicate too.

    The word "forget" in the name is motivated by the term "forgetful functor".

    @[instance 100]
    Equations
    • =
    @[instance 100]
    Equations
    • =
    theorem Filter.Tendsto.eval {F : Type u_1} {X : Type u_2} {Y : Type u_3} [FunLike F X Y] [TopologicalSpace F] [TopologicalSpace X] [TopologicalSpace Y] [ContinuousEval F X Y] {α : Type u_5} {l : Filter α} {f : αF} {f₀ : F} {g : αX} {x₀ : X} (hf : Filter.Tendsto f l (nhds f₀)) (hg : Filter.Tendsto g l (nhds x₀)) :
    Filter.Tendsto (fun (a : α) => (f a) (g a)) l (nhds (f₀ x₀))
    theorem ContinuousAt.eval {F : Type u_1} {X : Type u_2} {Y : Type u_3} {Z : Type u_4} [FunLike F X Y] [TopologicalSpace F] [TopologicalSpace X] [TopologicalSpace Y] [ContinuousEval F X Y] [TopologicalSpace Z] {f : ZF} {g : ZX} {z : Z} (hf : ContinuousAt f z) (hg : ContinuousAt g z) :
    ContinuousAt (fun (z : Z) => (f z) (g z)) z
    theorem ContinuousWithinAt.eval {F : Type u_1} {X : Type u_2} {Y : Type u_3} {Z : Type u_4} [FunLike F X Y] [TopologicalSpace F] [TopologicalSpace X] [TopologicalSpace Y] [ContinuousEval F X Y] [TopologicalSpace Z] {f : ZF} {g : ZX} {s : Set Z} {z : Z} (hf : ContinuousWithinAt f s z) (hg : ContinuousWithinAt g s z) :
    ContinuousWithinAt (fun (z : Z) => (f z) (g z)) s z
    theorem ContinuousOn.eval {F : Type u_1} {X : Type u_2} {Y : Type u_3} {Z : Type u_4} [FunLike F X Y] [TopologicalSpace F] [TopologicalSpace X] [TopologicalSpace Y] [ContinuousEval F X Y] [TopologicalSpace Z] {f : ZF} {g : ZX} {s : Set Z} (hf : ContinuousOn f s) (hg : ContinuousOn g s) :
    ContinuousOn (fun (z : Z) => (f z) (g z)) s