Skip to content

Commit

Permalink
Update Mathlib/Geometry/Manifold/ChartedSpace.lean
Browse files Browse the repository at this point in the history
Co-authored-by: Winston Yin <[email protected]>
  • Loading branch information
grunweg and winstonyin committed Jan 20, 2024
1 parent cccbe5a commit c7417ce
Showing 1 changed file with 3 additions and 6 deletions.
9 changes: 3 additions & 6 deletions Mathlib/Geometry/Manifold/ChartedSpace.lean
Original file line number Diff line number Diff line change
Expand Up @@ -983,12 +983,9 @@ instance hasGroupoid_continuousGroupoid : HasGroupoid M (continuousGroupoid H) :
theorem StructureGroupoid.trans_restricted {e e' : PartialHomeomorph M H} {G : StructureGroupoid H}
(he : e ∈ atlas H M) (he' : e' ∈ atlas H M)
[HasGroupoid M G] [ClosedUnderRestriction G] (s : Opens M) [Nonempty s] :
(e.subtypeRestr s).symm ≫ₕ e'.subtypeRestr s ∈ G := by
apply G.eq_on_source ?_ (e.subtypeRestr_symm_trans_subtypeRestr s e')
let hopen := e.isOpen_inter_preimage_symm s.2
refine G.locality fun x' hx' ↦ ⟨e.target ∩ e.symm ⁻¹' s, hopen, ?_, ?_ ⟩
· exact interior_subset (mem_of_mem_inter_right hx')
· exact closedUnderRestriction' (closedUnderRestriction' (G.compatible he he') hopen) hopen
(e.subtypeRestr s).symm ≫ₕ e'.subtypeRestr s ∈ G :=
G.eq_on_source (closedUnderRestriction' (G.compatible he he') (e.isOpen_inter_preimage_symm s.2))
(e.subtypeRestr_symm_trans_subtypeRestr s e')

section MaximalAtlas

Expand Down

0 comments on commit c7417ce

Please sign in to comment.