Partial homeomorphisms: Images of sets #
Main definitions #
OpenPartialHomeomorph.IsImage: predicate for when one set is an image of anotherOpenPartialHomeomorph.ofSet: the identity on a setsOpenPartialHomeomorph.EqOnSource: equivalence relation describing the "right" notion of equality for open partial homeomorphisms
Implementation notes #
Most statements are copied from their PartialEquiv versions, although some care is required
especially when restricting to subsets, as these should be open subsets.
For design notes, see PartialEquiv.lean.
Local coding conventions #
If a lemma deals with the intersection of a set with either source or target of a PartialEquiv,
then it should use e.source ∩ s or e.target ∩ t, not s ∩ e.source or t ∩ e.target.
OpenPartialHomeomorph.IsImage relation #
We say that t : Set Y is an image of s : Set X under an open partial homeomorphism e if any of
the following equivalent conditions hold:
e '' (e.source ∩ s) = e.target ∩ t;e.source ∩ e ⁻¹ t = e.source ∩ s;∀ x ∈ e.source, e x ∈ t ↔ x ∈ s(this one is used in the definition).
This definition is a restatement of PartialEquiv.IsImage for open partial homeomorphisms.
In this section we transfer API about PartialEquiv.IsImage to open partial homeomorphisms and
add a few OpenPartialHomeomorph-specific lemmas like OpenPartialHomeomorph.IsImage.closure.
We say that t : Set Y is an image of s : Set X under an open partial homeomorphism e
if any of the following equivalent conditions hold:
e '' (e.source ∩ s) = e.target ∩ t;e.source ∩ e ⁻¹ t = e.source ∩ s;∀ x ∈ e.source, e x ∈ t ↔ x ∈ s(this one is used in the definition).
Instances For
Alias of the forward direction of OpenPartialHomeomorph.IsImage.iff_preimage_eq.
Alias of the reverse direction of OpenPartialHomeomorph.IsImage.iff_preimage_eq.
Alias of the reverse direction of OpenPartialHomeomorph.IsImage.iff_symm_preimage_eq.
Alias of the forward direction of OpenPartialHomeomorph.IsImage.iff_symm_preimage_eq.
Alias of the reverse direction of OpenPartialHomeomorph.IsImage.iff_symm_preimage_eq'.
Alias of the forward direction of OpenPartialHomeomorph.IsImage.iff_symm_preimage_eq'.
Alias of the forward direction of OpenPartialHomeomorph.IsImage.iff_preimage_eq'.
Alias of the reverse direction of OpenPartialHomeomorph.IsImage.iff_preimage_eq'.
Restrict an OpenPartialHomeomorph to a pair of corresponding open sets.
Equations
Instances For
Preimage of interior or interior of preimage coincide for open partial homeomorphisms, when restricted to the source.
Restriction #
Restricting an open partial homeomorphism e to e.source ∩ s when s is open.
This is sometimes hard to use because of the openness assumption, but it has the advantage that
when it can be used then its PartialEquiv is defeq to PartialEquiv.restr.
Instances For
Restricting an open partial homeomorphism e to e.source ∩ interior s. We use the interior to
make sure that the restriction is well defined whatever the set s, since open partial homeomorphisms
are by definition defined on open sets. In applications where s is open, this coincides with the
restriction of partial equivalences.
Instances For
ofSet #
The identity on a set s
The identity partial equivalence on a set s
Equations
- OpenPartialHomeomorph.ofSet s hs = { toPartialEquiv := PartialEquiv.ofSet s, open_source := hs, open_target := hs, continuousOn_toFun := ⋯, continuousOn_invFun := ⋯ }
Instances For
EqOnSource: equivalence on their source
EqOnSource e e' means that e and e' have the same source, and coincide there. They
should really be considered the same partial equivalence.
Instances For
EqOnSource is an equivalence relation.
Equations
- OpenPartialHomeomorph.eqOnSourceSetoid = { r := OpenPartialHomeomorph.EqOnSource, iseqv := ⋯ }
If two open partial homeomorphisms are equivalent, so are their inverses.
Two equivalent open partial homeomorphisms have the same source.
Two equivalent open partial homeomorphisms have the same target.
Two equivalent open partial homeomorphisms have coinciding toFun on the source
Two equivalent open partial homeomorphisms have coinciding invFun on the target
Restriction of open partial homeomorphisms respects equivalence
Two equivalent open partial homeomorphisms are equal when the source and target are univ.
Alias of Homeomorph.refl_toOpenPartialHomeomorph.
Alias of Homeomorph.symm_toOpenPartialHomeomorph.