Computational realization of filters (experimental) #
This file provides infrastructure to compute with filters.
Main declarations #
Equations
- instInhabitedCFilter = { default := { f := id, pt := default, inf := fun (x1 x2 : α) => x1 ⊓ x2, inf_le_left := ⋯, inf_le_right := ⋯ } }
Equations
- CFilter.instCoeFunForall = { coe := CFilter.f }
theorem
CFilter.coe_mk
{α : Type u_1}
{σ : Type u_3}
[PartialOrder α]
(f : σ → α)
(pt : σ)
(inf : σ → σ → σ)
(h₁ : ∀ (a b : σ), f (inf a b) ≤ f a)
(h₂ : ∀ (a b : σ), f (inf a b) ≤ f b)
(a : σ)
:
Map a CFilter
to an equivalent representation type.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The filter represented by a CFilter
is the collection of supersets of
elements of the filter base.
Equations
Instances For
A filter realizes itself.
Equations
- One or more equations did not get rendered due to their size.
Instances For
@[simp]
@[simp]
Equations
- Filter.Realizer.instInhabitedPrincipal s = { default := Filter.Realizer.principal s }
Unit
is a realizer for the top filter
Instances For
@[simp]
@[simp]
theorem
Filter.Realizer.map_σ
{α : Type u_1}
{β : Type u_2}
(m : α → β)
{f : Filter α}
(F : f.Realizer)
:
@[simp]
theorem
Filter.Realizer.map_F
{α : Type u_1}
{β : Type u_2}
(m : α → β)
{f : Filter α}
(F : f.Realizer)
(s : (Realizer.map m F).σ)
:
Construct a realizer for the cofinite filter
Equations
- One or more equations did not get rendered due to their size.
Instances For
Construct a realizer for the product of filters
Equations
- F.prod G = (Filter.Realizer.comap Prod.fst F).inf (Filter.Realizer.comap Prod.snd G)