Germs of functions between topological spaces #
In this file, we prove basic properties of germs of functions between topological spaces,
with respect to the neighbourhood filter π x
.
Main definitions and results #
Filter.Germ.value Ο f
: value associated to the germΟ
at a pointx
, w.r.t. the neighbourhood filter atx
. This is the common value of all representatives ofΟ
atx
.Filter.Germ.valueOrderRingHom
and friends: the mapGerm (π x) E β E
is a monoid homomorphism, π-module homomorphism, ring homomorphism, monotone ring homomorphismRestrictGermPredicate
: given a predicate on germsP : Ξ x : X, germ (π x) Y β Prop
andA : set X
, build a new predicate on germsrestrictGermPredicate P A
such that(β x, RestrictGermPredicate P A x f) β βαΆ x near A, P x f
;forall_restrictRermPredicate_iff
is this equivalence.Filter.Germ.sliceLeft, sliceRight
: map the germ of functionsX Γ Y β Z
atp = (x,y) β X Γ Y
to the corresponding germ of functionsX β Z
atx β X
resp.Y β Z
aty β Y
.eq_of_germ_isConstant
: if each germ off : X β Y
is constant andX
is pre-connected,f
is constant.
The value associated to a germ at a point. This is the common value shared by all representatives at the given point.
Equations
- Ο.value = Quotient.liftOn' Ο (fun (f : X β Ξ±) => f x) β―
Instances For
The map Germ (π x) E β E
into a monoid E
as a monoid homomorphism
Equations
- Filter.Germ.valueMulHom = { toFun := Filter.Germ.value, map_one' := β―, map_mul' := β― }
Instances For
The map Germ (π x) E β E
as an additive monoid homomorphism
Equations
- Filter.Germ.valueAddHom = { toFun := Filter.Germ.value, map_zero' := β―, map_add' := β― }
Instances For
The map Germ (π x) E β E
into a π
-module E
as a π
-linear map
Equations
- Filter.Germ.valueβ = { toFun := (βFilter.Germ.valueAddHom).toFun, map_add' := β―, map_smul' := β― }
Instances For
The map Germ (π x) E β E
as a ring homomorphism
Equations
- Filter.Germ.valueRingHom = { toMonoidHom := Filter.Germ.valueMulHom, map_zero' := β―, map_add' := β― }
Instances For
The map Germ (π x) E β E
as a monotone ring homomorphism
Equations
- Filter.Germ.valueOrderRingHom = { toRingHom := Filter.Germ.valueRingHom, monotone' := β― }
Instances For
Given a predicate on germs P : Ξ x : X, germ (π x) Y β Prop
and A : set X
,
build a new predicate on germs RestrictGermPredicate P A
such that
(β x, RestrictGermPredicate P A x f) β βαΆ x near A, P x f
, see
forall_restrictGermPredicate_iff
for this equivalence.
Equations
- RestrictGermPredicate P A x Ο = Ο.liftOn (fun (f : X β Y) => x β A β βαΆ (y : X) in nhds x, P y βf) β―
Instances For
Map the germ of functions X Γ Y β Z
at p = (x,y) β X Γ Y
to the corresponding germ
of functions X β Z
at x β X
Equations
- P.sliceLeft = P.compTendsto (fun (x : X) => (x, p.2)) β―
Instances For
Map the germ of functions X Γ Y β Z
at p = (x,y) β X Γ Y
to the corresponding germ
of functions Y β Z
at y β Y
Instances For
If the germ of f
w.r.t. each π x
is constant, f
is locally constant.