Skip to content

Commit

Permalink
Bump mathlib again. PRs emptying two files were merged.
Browse files Browse the repository at this point in the history
  • Loading branch information
grunweg committed Jan 24, 2024
1 parent d91dd15 commit efe99f8
Show file tree
Hide file tree
Showing 6 changed files with 9 additions and 80 deletions.
2 changes: 0 additions & 2 deletions SphereEversion.lean
Original file line number Diff line number Diff line change
Expand Up @@ -43,7 +43,6 @@ import SphereEversion.ToMathlib.Data.Set.Lattice
import SphereEversion.ToMathlib.Data.Set.Prod
import SphereEversion.ToMathlib.Equivariant
import SphereEversion.ToMathlib.ExistsOfConvex
import SphereEversion.ToMathlib.Geometry.Manifold.Algebra.LieGroup
import SphereEversion.ToMathlib.Geometry.Manifold.Algebra.SmoothGerm
import SphereEversion.ToMathlib.Geometry.Manifold.Metrizable
import SphereEversion.ToMathlib.Geometry.Manifold.MiscManifold
Expand All @@ -69,4 +68,3 @@ import SphereEversion.ToMathlib.Topology.Paracompact
import SphereEversion.ToMathlib.Topology.Path
import SphereEversion.ToMathlib.Topology.Periodic
import SphereEversion.ToMathlib.Topology.Separation
import SphereEversion.ToMathlib.Topology.Support
46 changes: 0 additions & 46 deletions SphereEversion/ToMathlib/Geometry/Manifold/Algebra/LieGroup.lean

This file was deleted.

10 changes: 5 additions & 5 deletions SphereEversion/ToMathlib/Partition.lean
Original file line number Diff line number Diff line change
@@ -1,10 +1,10 @@
import Mathlib.Geometry.Manifold.PartitionOfUnity
import Mathlib.Geometry.Manifold.ContMDiff.Basic
import SphereEversion.ToMathlib.Geometry.Manifold.Algebra.SmoothGerm
import SphereEversion.ToMathlib.Geometry.Manifold.Algebra.LieGroup
import SphereEversion.ToMathlib.Analysis.Convex.Basic
import SphereEversion.ToMathlib.Topology.Support
import SphereEversion.ToMathlib.Topology.LocallyFinite
import Mathlib.Geometry.Manifold.PartitionOfUnity
import Mathlib.Geometry.Manifold.ContMDiff.Basic
import Mathlib.Geometry.Manifold.Algebra.LieGroup
import Mathlib.Topology.Support

noncomputable section

Expand All @@ -26,7 +26,7 @@ theorem SmoothPartitionOfUnity.contMDiffAt_sum (ρ : SmoothPartitionOfUnity ι I
refine' contMDiffAt_finsum (ρ.locallyFinite.smul_left _) fun i => _
by_cases hx : x₀ ∈ tsupport (ρ i)
· exact ContMDiffAt.smul ((ρ i).smooth.of_le le_top).contMDiffAt (hφ i hx)
· exact contMDiffAt_of_not_mem (compl_subset_compl.mpr (tsupport_smul_left (ρ i) (φ i)) hx) n
· exact contMDiffAt_of_not_mem (compl_subset_compl.mpr (tsupport_smul_subset_left (ρ i) (φ i)) hx) n

theorem SmoothPartitionOfUnity.contDiffAt_sum {s : Set E}
(ρ : SmoothPartitionOfUnity ι 𝓘(ℝ, E) E s) {n : ℕ∞} {x₀ : E} {φ : ι → E → F}
Expand Down
2 changes: 1 addition & 1 deletion SphereEversion/ToMathlib/Topology/LocallyFinite.lean
Original file line number Diff line number Diff line change
Expand Up @@ -39,7 +39,7 @@ open scoped Topology

open Filter

-- submitted as PR #9813
-- submitted as PR mathlib4#9813
theorem LocallyFinite.eventually_subset {ι X : Type*} [TopologicalSpace X] {s : ι → Set X}
(hs : LocallyFinite s) (hs' : ∀ i, IsClosed (s i)) (x : X) :
∀ᶠ y in 𝓝 x, {i | y ∈ s i} ⊆ {i | x ∈ s i} := by
Expand Down
23 changes: 0 additions & 23 deletions SphereEversion/ToMathlib/Topology/Support.lean

This file was deleted.

6 changes: 3 additions & 3 deletions lake-manifest.json
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@
[{"url": "https://github.com/leanprover/std4",
"type": "git",
"subDir": null,
"rev": "1972e073b3e6bc0776ad5b544bfa7db7fc3f7c36",
"rev": "0d0ac1c43e1ec1965e0806af9e7a32999ea31096",
"name": "std",
"manifestFile": "lake-manifest.json",
"inputRev": "main",
Expand All @@ -22,7 +22,7 @@
{"url": "https://github.com/leanprover-community/aesop",
"type": "git",
"subDir": null,
"rev": "1c638703ed1c0c42aed2687acbeda67cec801454",
"rev": "24a4e8fea81999723bfc38bebf7adc86c2f26c6c",
"name": "aesop",
"manifestFile": "lake-manifest.json",
"inputRev": "master",
Expand Down Expand Up @@ -58,7 +58,7 @@
{"url": "https://github.com/leanprover-community/mathlib4.git",
"type": "git",
"subDir": null,
"rev": "e3c20cbbbbe7a771a4579587bc2326669e992ae1",
"rev": "a686ba8279292ac8c50a644ee7ee3c9ab178a649",
"name": "mathlib",
"manifestFile": "lake-manifest.json",
"inputRev": null,
Expand Down

0 comments on commit efe99f8

Please sign in to comment.