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.valueOrderRingHomand friends: the mapGerm (π x) E β Eis a monoid homomorphism, π-linear map, ring homomorphism, monotone ring homomorphismRestrictGermPredicate: given a predicate on germsP : Ξ x : X, germ (π x) Y β PropandA : set X, build a new predicate on germsrestrictGermPredicate P Asuch that(β x, RestrictGermPredicate P A x f) β βαΆ x near A, P x f;forall_restrictRermPredicate_iffis this equivalence.Filter.Germ.sliceLeft, sliceRight: map the germ of functionsX Γ Y β Zatp = (x,y) β X Γ Yto the corresponding germ of functionsX β Zatx β Xresp.Y β Zaty β Y.eq_of_germ_isConstant: if each germ off : X β Yis constant andXis pre-connected,fis 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
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
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
Equations
- P.sliceRight = P.compTendsto (Prod.mk p.1) β―
Instances For
If the germ of f w.r.t. each π x is constant, f is locally constant.