Skip to content

Commit

Permalink
chore(Geometry/Manifold/SmoothPartitionOfUnity): remove autoImplicit (#…
Browse files Browse the repository at this point in the history
…9634)

It's just used once for one variable. That's not pulling its weight.
  • Loading branch information
grunweg committed Jan 11, 2024
1 parent 1e0cd87 commit 702f3fe
Showing 1 changed file with 1 addition and 4 deletions.
5 changes: 1 addition & 4 deletions Mathlib/Geometry/Manifold/PartitionOfUnity.lean
Expand Up @@ -85,9 +85,6 @@ any `U : M → Set M` such that `∀ x ∈ s, U x ∈ 𝓝 x` there exists a `Sm
subordinate to `U`. Then we use this fact to prove a version of the Whitney embedding theorem: any
compact real manifold can be embedded into `ℝ^n` for large enough `n`. -/

set_option autoImplicit true


variable (ι M)

/-- We say that a collection of `SmoothBumpFunction`s is a `SmoothBumpCovering` of a set `s` if
Expand Down Expand Up @@ -634,7 +631,7 @@ lemma IsOpen.exists_msmooth_support_eq_aux {s : Set H} (hs : IsOpen s) :

/-- Given an open set in a finite-dimensional real manifold, there exists a nonnegative smooth
function with support equal to `s`. -/
theorem IsOpen.exists_msmooth_support_eq (hs : IsOpen s) :
theorem IsOpen.exists_msmooth_support_eq {s : Set M} (hs : IsOpen s) :
∃ f : M → ℝ, f.support = s ∧ Smooth I 𝓘(ℝ) f ∧ ∀ x, 0 ≤ f x := by
rcases SmoothPartitionOfUnity.exists_isSubordinate_chartAt_source I M with ⟨f, hf⟩
have A : ∀ (c : M), ∃ g : H → ℝ,
Expand Down

0 comments on commit 702f3fe

Please sign in to comment.