Documentation

Mathlib.Topology.Instances.RealVectorSpace

Continuous additive maps are -linear #

In this file we prove that a continuous map f : E →+ F between two topological vector spaces over is -linear

theorem map_real_smul {E : Type u_1} [AddCommGroup E] [Module E] [TopologicalSpace E] [ContinuousSMul E] {F : Type u_2} [AddCommGroup F] [Module F] [TopologicalSpace F] [ContinuousSMul F] [T2Space F] {G : Type u_3} [FunLike G E F] [AddMonoidHomClass G E F] (f : G) (hf : Continuous f) (c : ) (x : E) :
f (c x) = c f x

A continuous additive map between two vector spaces over is -linear.

Reinterpret a continuous additive homomorphism between two real vector spaces as a continuous real-linear map.

Equations
Instances For

    Reinterpret a continuous additive equivalence between two real vector spaces as a continuous real-linear map.

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For

      A topological group carries at most one structure of a topological -module, so for any topological -algebra A (e.g. A = ℂ) and any topological group that is both a topological -module and a topological A-module, these structures agree.

      Equations
      • =