mathlib documentation

topology.instances.real_vector_space

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 add_monoid_hom.map_real_smul {E : Type u_1} [add_comm_group E] [vector_space E] [topological_space E] [topological_vector_space E] {F : Type u_2} [add_comm_group F] [vector_space F] [topological_space F] [topological_vector_space F] [t2_space F] (f : E →+ F) (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