Units of continuous functions #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
This file concerns itself with C(X, M)ˣ
and C(X, Mˣ)
when X
is a topological space
and M
has some monoid structure compatible with its topology.
Equivalence between continuous maps into the additive units of an additive monoid with continuous addition and the additive units of the additive monoid of continuous maps.
Equations
- continuous_map.add_units_lift = {to_fun := λ (f : C(X, add_units M)), {val := {to_fun := λ (x : X), ↑(⇑f x), continuous_to_fun := _}, neg := {to_fun := λ (x : X), ↑-⇑f x, continuous_to_fun := _}, val_neg := _, neg_val := _}, inv_fun := λ (f : add_units C(X, M)), {to_fun := λ (x : X), {val := ⇑f x, neg := (⇑-f) x, val_neg := _, neg_val := _}, continuous_to_fun := _}, left_inv := _, right_inv := _}
Equivalence between continuous maps into the units of a monoid with continuous multiplication and the units of the monoid of continuous maps.
Equations
- continuous_map.units_lift = {to_fun := λ (f : C(X, Mˣ)), {val := {to_fun := λ (x : X), ↑(⇑f x), continuous_to_fun := _}, inv := {to_fun := λ (x : X), ↑(⇑f x)⁻¹, continuous_to_fun := _}, val_inv := _, inv_val := _}, inv_fun := λ (f : C(X, M)ˣ), {to_fun := λ (x : X), {val := ⇑f x, inv := ⇑f⁻¹ x, val_inv := _, inv_val := _}, continuous_to_fun := _}, left_inv := _, right_inv := _}
Construct a continuous map into the group of units of a normed ring from a function into the normed ring and a proof that every element of the range is a unit.
Equations
- continuous_map.units_of_forall_is_unit h = {to_fun := λ (x : X), _.unit, continuous_to_fun := _}
Equations
- continuous_map.can_lift = {prf := _}