Germ of a function at a filter #
The germ of a function f : α → β
at a filter l : Filter α
is the equivalence class of f
with respect to the equivalence relation EventuallyEq l
: f ≈ g
means ∀ᶠ x in l, f x = g x
.
Main definitions #
We define
Filter.Germ l β
to be the space of germs of functionsα → β
at a filterl : Filter α
;- coercion from
α → β
toGerm l β
:(f : Germ l β)
is the germ off : α → β
atl : Filter α
; this coercion is declared asCoeTC
; (const l c : Germ l β)
is the germ of the constant functionfun x : α ↦ c
at a filterl
;- coercion from
β
toGerm l β
:(↑c : Germ l β)
is the germ of the constant functionfun x : α ↦ c
at a filterl
; this coercion is declared asCoeTC
; map (F : β → γ) (f : Germ l β)
to be the composition of a functionF
and a germf
;map₂ (F : β → γ → δ) (f : Germ l β) (g : Germ l γ)
to be the germ offun x ↦ F (f x) (g x)
atl
;f.Tendsto lb
: we say that a germf : Germ l β
tends to a filterlb
if its representatives tend tolb
alongl
;f.compTendsto g hg
andf.compTendsto' g hg
: givenf : Germ l β
and a functiong : γ → α
(resp., a germg : Germ lc α
), ifg
tends tol
alonglc
, then the compositionf ∘ g
is a well-defined germ atlc
;Germ.liftPred
,Germ.liftRel
: lift a predicate or a relation to the space of germs:(f : Germ l β).liftPred p
means∀ᶠ x in l, p (f x)
, and similarly for a relation.
We also define map (F : β → γ) : Germ l β → Germ l γ
sending each germ f
to F ∘ f
.
For each of the following structures we prove that if β
has this structure, then so does
Germ l β
:
- one-operation algebraic structures up to
CommGroup
; MulZeroClass
,Distrib
,Semiring
,CommSemiring
,Ring
,CommRing
;MulAction
,DistribMulAction
,Module
;Preorder
,PartialOrder
, andLattice
structures, as well asBoundedOrder
;OrderedCancelCommMonoid
andOrderedCancelAddCommMonoid
.
Tags #
filter, germ
Setoid used to define the filter product. This is a dependent version of
Filter.germSetoid
.
Instances For
The filter product (a : α) → ε a
at a filter l
. This is a dependent version of
Filter.Germ
.
Instances For
Instances For
Instances For
Given a map F : (α → β) → (γ → δ)
that sends functions eventually equal at l
to functions
eventually equal at lc
, returns a map from Germ l β
to Germ lc δ
.
Instances For
Given a germ f : Germ l β
and a function F : (α → β) → γ
sending eventually equal functions
to the same value, returns the value F
takes on functions having germ f
at l
.
Instances For
Alias of the reverse direction of Filter.Germ.coe_eq
.
Lift a function β → γ
to a function Germ l β → Germ l γ
.
Instances For
Lift a binary function β → γ → δ
to a function Germ l β → Germ l γ → Germ l δ
.
Instances For
A germ at l
of maps from α
to β
tends to lb : Filter β
if it is represented by a map
which tends to lb
along l
.
Instances For
Alias of the reverse direction of Filter.Germ.coe_tendsto
.
Given two germs f : Germ l β
, and g : Germ lc α
, where l : Filter α
, if g
tends to l
,
then the composition f ∘ g
is well-defined as a germ at lc
.
Instances For
Given a germ f : Germ l β
and a function g : γ → α
, where l : Filter α
, if g
tends
to l
along lc : Filter γ
, then the composition f ∘ g
is well-defined as a germ at lc
.
Instances For
Lift a predicate on β
to Germ l β
.
Instances For
Lift a relation r : β → γ → Prop
to Germ l β → Germ l γ → Prop
.
Instances For
Coercion from functions to germs as an additive monoid homomorphism.
Instances For
Coercion from functions to germs as a monoid homomorphism.
Instances For
Coercion (α → R) → Germ l R
as a RingHom
.