Lattice operations on finsets of functions #
This file is concerned with folding binary lattice operations over finsets.
theorem
Finset.inf_sup
{α : Type u_1}
{ι : Type u_2}
[DistribLattice α]
[BoundedOrder α]
[DecidableEq ι]
{κ : ι → Type u_3}
(s : Finset ι)
(t : (i : ι) → Finset (κ i))
(f : (i : ι) → κ i → α)
:
theorem
Finset.sup_inf
{α : Type u_1}
{ι : Type u_2}
[DistribLattice α]
[BoundedOrder α]
[DecidableEq ι]
{κ : ι → Type u_3}
(s : Finset ι)
(t : (i : ι) → Finset (κ i))
(f : (i : ι) → κ i → α)
: