Documentation

Mathlib.Topology.ContinuousMap.Polynomial

Constructions relating polynomial functions and continuous functions. #

Main definitions #

Every polynomial with coefficients in a topological semiring gives a (bundled) continuous function.

Equations
Instances For

    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
    Instances For
      @[simp]
      @[simp]
      theorem Polynomial.aeval_continuousMap_apply {R : Type u_1} {α : Type u_2} [TopologicalSpace α] [CommSemiring R] [TopologicalSpace R] [IsTopologicalSemiring R] (g : Polynomial R) (f : C(α, R)) (x : α) :
      ((aeval f) g) x = eval (f x) g

      The algebra map from R[X] to continuous functions C(R, R).

      Equations
      Instances For

        The algebra map from R[X] to continuous functions C(X, R), for any subset X of R.

        Equations
        Instances For
          noncomputable def polynomialFunctions {R : Type u_1} [CommSemiring R] [TopologicalSpace R] [IsTopologicalSemiring R] (X : Set R) :

          The subalgebra of polynomial functions in C(X, R), for X a subset of some topological semiring R.

          Equations
          Instances For

            The preimage of polynomials on [0,1] under the pullback map by x ↦ (b-a) * x + a is the polynomials on [a,b].