Skip to content

Commit

Permalink
restore StoneWeierstrass
Browse files Browse the repository at this point in the history
  • Loading branch information
Benoît Guillemet committed Feb 21, 2025
1 parent 42d0007 commit a00977d
Show file tree
Hide file tree
Showing 2 changed files with 1 addition and 3 deletions.
1 change: 0 additions & 1 deletion Mathlib/Analysis/Calculus/FDeriv/MvPolynomial.lean
Original file line number Diff line number Diff line change
Expand Up @@ -9,7 +9,6 @@ import Mathlib.Analysis.Calculus.FDeriv.Mul
import Mathlib.Analysis.Calculus.Deriv.Pow
import Mathlib.Algebra.BigOperators.Group.Finset


/-!
# Derivatives of multivariate polynomials
Expand Down
3 changes: 1 addition & 2 deletions Mathlib/Topology/ContinuousMap/StoneWeierstrass.lean
Original file line number Diff line number Diff line change
Expand Up @@ -7,7 +7,6 @@ import Mathlib.Analysis.RCLike.Basic
import Mathlib.Topology.Algebra.StarSubalgebra
import Mathlib.Topology.ContinuousMap.ContinuousMapZero
import Mathlib.Topology.ContinuousMap.Weierstrass
import Mathlib.Topology.ContinuousMap.MvPolynomial
import Mathlib.Topology.ContinuousMap.Lattice

/-!
Expand Down Expand Up @@ -435,7 +434,7 @@ section PolynomialFunctions
open StarSubalgebra Polynomial
open scoped Polynomial

/-- Polynomial functions are dense in `C(s, ℝ)` when `s` is compact.
/-- Polynomial functions in are dense in `C(s, ℝ)` when `s` is compact.
See `polynomialFunctions_closure_eq_top` for the special case `s = Set.Icc a b` which does not use
the full Stone-Weierstrass theorem. Of course, that version could be used to prove this one as
Expand Down

0 comments on commit a00977d

Please sign in to comment.