Skip to content

Commit

Permalink
chore: fix a name (#6015)
Browse files Browse the repository at this point in the history
Rename `LocalHomeomorph.trans_equiv_eq_trans`
to `LocalHomeomorph.transHomeomorph_eq_trans`.

Also fix the module docstring.
  • Loading branch information
urkud committed Jul 20, 2023
1 parent 11832fa commit 5070d54
Showing 1 changed file with 10 additions and 9 deletions.
19 changes: 10 additions & 9 deletions Mathlib/Topology/LocalHomeomorph.lean
Expand Up @@ -22,14 +22,14 @@ instead of `e.toFun x` and `e.invFun x`.
## Main definitions
`Homeomorph.toLocalHomeomorph`: associating a local homeomorphism to a homeomorphism, with
source = target = univ
`LocalHomeomorph.symm` : the inverse of a local homeomorphism
`Homeomorph.toLocalHomeomorph` : associating a local homeomorphism to a homeomorphism, with
`source = target = Set.univ`;
`LocalHomeomorph.symm` : the inverse of a local homeomorphism
`LocalHomeomorph.trans` : the composition of two local homeomorphisms
`LocalHomeomorph.refl` : the identity local homeomorphism
`LocalHomeomorph.ofSet`: the identity on a set `s`
`eq_on_source` : equivalence relation describing the "right" notion of equality for local
homeomorphisms
`LocalHomeomorph.refl` : the identity local homeomorphism
`LocalHomeomorph.ofSet` : the identity on a set `s`
`LocalHomeomorph.EqOnSource` : equivalence relation describing the "right" notion of equality
for local homeomorphisms
## Implementation notes
Expand Down Expand Up @@ -901,9 +901,10 @@ def transHomeomorph (e' : β ≃ₜ γ) : LocalHomeomorph α γ where
continuous_invFun := e.symm.continuousOn.comp e'.symm.continuous.continuousOn fun _ => id
#align local_homeomorph.trans_homeomorph LocalHomeomorph.transHomeomorph

theorem trans_equiv_eq_trans (e' : β ≃ₜ γ) : e.transHomeomorph e' = e.trans e'.toLocalHomeomorph :=
theorem transHomeomorph_eq_trans (e' : β ≃ₜ γ) :
e.transHomeomorph e' = e.trans e'.toLocalHomeomorph :=
toLocalEquiv_injective <| LocalEquiv.transEquiv_eq_trans _ _
#align local_homeomorph.trans_equiv_eq_trans LocalHomeomorph.trans_equiv_eq_trans
#align local_homeomorph.trans_equiv_eq_trans LocalHomeomorph.transHomeomorph_eq_trans

/-- Precompose a local homeomorphism with a homeomorphism.
We modify the source and target to have better definitional behavior. -/
Expand Down

0 comments on commit 5070d54

Please sign in to comment.