Results filters related to finiteness. #
Lattice equations #
theorem
Pairwise.exists_mem_filter_of_disjoint
{α : Type u}
{ι : Type u_2}
[Finite ι]
{l : ι → Filter α}
(hd : Pairwise (Function.onFun Disjoint l))
:
theorem
Set.PairwiseDisjoint.exists_mem_filter
{α : Type u}
{ι : Type u_2}
{l : ι → Filter α}
{t : Set ι}
(hd : t.PairwiseDisjoint l)
(ht : t.Finite)
:
∃ (s : ι → Set α), (∀ (i : ι), s i ∈ l i) ∧ t.PairwiseDisjoint s
@[reducible, inline]
The dual version does not hold! Filter α
is not a CompleteDistribLattice
.
Instances For
principal
equations #
@[simp]
A special case of iInf_principal
that is safe to mark simp
.