Documentation

Mathlib.Topology.Homotopy.Affine

Affine homotopy between two continuous maps #

In this file we define ContinuousMap.Homotopy.affine f g to be the homotopy between f and g such that affine f g (t, x) = AffineMap.lineMap (f x) (g x) t.

The homotopy between f and g such that affine f g (t, x) = AffineMap.lineMap (f x) (g x) t.

Equations
Instances For
    @[simp]
    theorem ContinuousMap.Homotopy.affine_apply {X : Type u_1} {E : Type u_2} [TopologicalSpace X] [AddCommGroup E] [TopologicalSpace E] [IsTopologicalAddGroup E] [Module E] [ContinuousSMul E] (f g : C(X, E)) (x : unitInterval × X) :
    (affine f g) x = (AffineMap.lineMap (f x.2) (g x.2)) x.1
    @[simp]