bounded lattices #
This file defines top and bottom elements (greatest and least elements) of a type, the bounded
variants of different kinds of lattices, sets up the typeclass hierarchy between them and provides
instances for Prop
and fun
.
Common lattices #
- Distributive lattices with a bottom element. Notated by
[DistribLattice α] [OrderBot α]
It captures the properties ofDisjoint
that are common toGeneralizedBooleanAlgebra
andDistribLattice
whenOrderBot
. - Bounded and distributive lattice. Notated by
[DistribLattice α] [BoundedOrder α]
. Typical examples includeProp
andDet α
.
Top, bottom element #
In this section we prove some properties about monotone and antitone operations on Prop
#
theorem
exists_ge_and_iff_exists
{α : Type u}
[SemilatticeSup α]
{P : α → Prop}
{x₀ : α}
(hP : Monotone P)
:
theorem
exists_and_iff_of_monotone
{α : Type u}
[SemilatticeSup α]
{P Q : α → Prop}
(hP : Monotone P)
(hQ : Monotone Q)
:
theorem
exists_le_and_iff_exists
{α : Type u}
[SemilatticeInf α]
{P : α → Prop}
{x₀ : α}
(hP : Antitone P)
:
theorem
exists_and_iff_of_antitone
{α : Type u}
[SemilatticeInf α]
{P Q : α → Prop}
(hP : Antitone P)
(hQ : Antitone Q)
: