Constructions relating polynomial functions and continuous functions. #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
Main definitions #
polynomial.to_continuous_map_on p X
: forX : set R
, interprets a polynomialp
as a bundled continuous function inC(X, R)
.polynomial.to_continuous_map_on_alg_hom
: the same, as anR
-algebra homomorphism.polynomial_functions (X : set R) : subalgebra R C(X, R)
: polynomial functions as a subalgebra.polynomial_functions_separates_points (X : set R) : (polynomial_functions X).separates_points
: the polynomial functions separate points.
Every polynomial with coefficients in a topological semiring gives a (bundled) continuous function.
Equations
- p.to_continuous_map = {to_fun := λ (x : R), polynomial.eval x p, continuous_to_fun := _}
A polynomial as a continuous function, with domain restricted to some subset of the semiring of coefficients.
(This is particularly useful when restricting to compact sets, e.g. [0,1]
.)
Equations
- p.to_continuous_map_on X = {to_fun := λ (x : ↥X), ⇑(p.to_continuous_map) ↑x, continuous_to_fun := _}
The algebra map from R[X]
to continuous functions C(R, R)
.
Equations
- polynomial.to_continuous_map_alg_hom = {to_fun := λ (p : polynomial R), p.to_continuous_map, map_one' := _, map_mul' := _, map_zero' := _, map_add' := _, commutes' := _}
The algebra map from R[X]
to continuous functions C(X, R)
, for any subset X
of R
.
Equations
- polynomial.to_continuous_map_on_alg_hom X = {to_fun := λ (p : polynomial R), p.to_continuous_map_on X, map_one' := _, map_mul' := _, map_zero' := _, map_add' := _, commutes' := _}
The subalgebra of polynomial functions in C(X, R)
, for X
a subset of some topological semiring
R
.
Equations
The preimage of polynomials on [0,1]
under the pullback map by x ↦ (b-a) * x + a
is the polynomials on [a,b]
.