Skip to content
New issue

Have a question about this project? Sign up for a free GitHub account to open an issue and contact its maintainers and the community.

By clicking “Sign up for GitHub”, you agree to our terms of service and privacy statement. We’ll occasionally send you account related emails.

Already on GitHub? Sign in to your account

Porting note: added proof #10888

Open
pitmonticone opened this issue Feb 23, 2024 · 0 comments
Open

Porting note: added proof #10888

pitmonticone opened this issue Feb 23, 2024 · 0 comments
Labels
porting-notes Mathlib3 to Mathlib4 porting notes.

Comments

@pitmonticone
Copy link
Collaborator

Classifies porting notes claiming added proof.

Examples

/-- In a paracompact space, every open covering of a closed set admits a locally finite refinement
indexed by the same type. -/
theorem precise_refinement_set [ParacompactSpace X] {s : Set X} (hs : IsClosed s) (u : ι → Set X)
(uo : ∀ i, IsOpen (u i)) (us : s ⊆ ⋃ i, u i) :
∃ v : ι → Set X, (∀ i, IsOpen (v i)) ∧ (s ⊆ ⋃ i, v i) ∧ LocallyFinite v ∧ ∀ i, v i ⊆ u i := by
-- Porting note: Added proof of uc
have uc : (iUnion fun i => Option.elim' sᶜ u i) = univ := by
apply Subset.antisymm (subset_univ _)
· simp_rw [← compl_union_self s, Option.elim', iUnion_option]
apply union_subset_union_right sᶜ us
rcases precise_refinement (Option.elim' sᶜ u) (Option.forall.2 ⟨isOpen_compl_iff.2 hs, uo⟩)
uc with
⟨v, vo, vc, vf, vu⟩
refine' ⟨v ∘ some, fun i ↦ vo _, _, vf.comp_injective (Option.some_injective _), fun i ↦ vu _⟩
· simp only [iUnion_option, ← compl_subset_iff_union] at vc
exact Subset.trans (subset_compl_comm.1 <| vu Option.none) vc
#align precise_refinement_set precise_refinement_set

/-- (Impl) A preliminary definition to avoid timeouts. -/
@[simps]
def conesEquivFunctor (B : C) {J : Type w} (F : Discrete J ⥤ Over B) :
Cone (widePullbackDiagramOfDiagramOver B F) ⥤ Cone F where
obj c :=
{ pt := Over.mk (c.π.app none)
π :=
{ app := fun ⟨j⟩ => Over.homMk (c.π.app (some j)) (c.w (WidePullbackShape.Hom.term j))
-- Porting note: Added a proof for `naturality`
naturality := fun ⟨X⟩ ⟨Y⟩ ⟨⟨f⟩⟩ => by dsimp at f ⊢; aesop_cat } }

@pitmonticone pitmonticone added the porting-notes Mathlib3 to Mathlib4 porting notes. label Feb 23, 2024
mathlib-bors bot pushed a commit that referenced this issue Feb 23, 2024
Classifies by adding issue number (#10888) to porting notes claiming `added proof`.
thorimur pushed a commit that referenced this issue Feb 24, 2024
Classifies by adding issue number (#10888) to porting notes claiming `added proof`.
thorimur pushed a commit that referenced this issue Feb 26, 2024
Classifies by adding issue number (#10888) to porting notes claiming `added proof`.
riccardobrasca pushed a commit that referenced this issue Mar 1, 2024
Classifies by adding issue number (#10888) to porting notes claiming `added proof`.
dagurtomas pushed a commit that referenced this issue Mar 22, 2024
Classifies by adding issue number (#10888) to porting notes claiming `added proof`.
Louddy pushed a commit that referenced this issue Apr 15, 2024
Classifies by adding issue number (#10888) to porting notes claiming `added proof`.
Sign up for free to join this conversation on GitHub. Already have an account? Sign in to comment
Labels
porting-notes Mathlib3 to Mathlib4 porting notes.
Projects
None yet
Development

No branches or pull requests

1 participant