LESSWRONG
LW

Wikitags
Main
2
Exercises
1
Examples

Lattice (Order Theory)

Edited by Kevin Clancy, et al. last updated 6th Dec 2016
Requires: Join and meet, Partially ordered set

A lattice is a partially ordered set that is closed under binary joins and meets.

Let L be a lattice. Then for all p,q,r∈L the following properties are necessarily satisfied.

  • Associativity of joins and meets: (p∨q)∨r=p∨(q∨r), and (p∧q)∧r=p∧(q∧r)
  • Commutativity of joins and meets: p∨q=q∨p and p∧q=q∧p
  • Idempotency of joins and and meets: p∨p=p and p∧p=p
  • Absorption: p∨(p∧q)=p and p∧(p∨q)=p

Proofs

Lemma 1: Let P be a poset, S⊆P, and p∈P. If both ⋁S and (⋁S)∨p exist then ⋁(S∪{p}) exists as well, and (⋁S)∨p=⋁(S∪{p}).

Proof: See the Join fu exercise in Join and meet: Exercises.

Associativity

Let L be a lattice and p,q,r,s∈L such that s=p∨(q∨r). We apply the above lemma, along with commutativity and closure of lattices under binary joins, to get p∨(q∨r)=(q∨r)∨p=(⋁{q,r})∨p=⋁({q,r}∪{p})= ⋁{q,r,p}=⋁({p,q}∪{r})=(⋁{p,q})∨r=(p∨q)∨r.

By duality, we also have the associativity of binary meets.

Commutativity

Let L be a lattice and p,q∈L. Then p∨q=⋁{p,q}=q∨p. Binary joins are therefore commutative. By duality, binary meets are also commutative.

Idempotency

Let L be a lattice and p∈L. Then p∨p=⋁{p}=p. The property that for all p∈L, p∨p=p is called idempotency. By duality, we also have the idempotency of meets: for all p∈L, p∧p=p.

Absorption

Since p∧q is the greatest lower bound of {p,q}, p∧q≤p. Because p≤p and (p∧q)≤p, p is an upper bound of {p,p∧q}, and so p∨(p∧q)≤p. On the other hand, p∨(p∧q) is the least upper bound of {p,p∧q}, and so p≤p∨(p∧q). By anti-symmetry, p=p∨(p∧q).

Closure under finite joins and meets

Let L be a lattice and S={s1,...,sn} be some finite subset of L. Then an inductive argument shows that ⋁S exists.

Proof

Here again, we will need Lemma 1, stated in the proofs of the four lattice properties.

Our proof proceeds by induction on the cardinality of S.

The base case is ⋁{s1}=s1∈L. For the inductive step, we suppose that ⋁{s1,...,si} exists. Then, applying lemma 1, we have ⋁{s1,...,si+1}=⋁{s1,...,si}∨si+1. Applying our inductive hypothesis and closure under binary joins, we have ⋁{s1,...,si}∨si+1 exists. Lattices are therefore closed under all finite joins, not just binary ones. Dually, lattices are closed under all finite meets.

Basic positive examples

Here are two Hasse diagrams of posets which are lattices.

A diamond shaped lattice

A cube shaped lattice

Basic negative examples

Here are two Hasse diagrams of posets which are not lattices.

A simple non-lattice

In the above diagram, the two bottom elements have no common lower bounds. Therefore they have no meet, and so the depicted poset is not a lattice. However, it should be easy to verify that this poset is closed under binary joins.

Another simple non-lattice

The Hasse diagram of this poset has two connected components. No element from the left component will have a meet or a join with any element from the right component. The depicted poset is therefore not a lattice.

The connecting lemma

The connecting lemma states that for any lattice L and p,q∈L, p∨q=p⇔q≤p and dually, p∧q=p⇔q≥p. This simple but important lemma is so named because it establishes a connection between the lattice's join operator and its underlying poset order.

Proof

We prove p∨q=p⇔q≤p; the other part follows from duality. If p∨q=p, then p is an upper bound of both p and q, and so q≤p. Going the other direction, suppose q≤p. Since p is and upper bound of itself by reflexivity, it then follows that p is an upper bound of {p,q}. There cannot be a lesser upper bound of {p,q} because it would not be an upper bound of p. Hence, p∨q=p.

Lattices as algebraic structures

It's also possible to formulate lattices as algebraic structures ⟨L,∨,∧⟩ satisfying the associativity, commutativity, idempotency, and absorption laws described above. A poset ⟨L,≤⟩ can then be defined such that for p,q∈L, p≤q whenever p∨q=q. It can be shown that this poset is closed under binary meets and joins, and that these meets and joins are equal to the corresponding meets and joins of the algebraic lattice.

Additional material

For more examples of lattices, see Lattice: Examples. For some exercises involving the concepts introduced on this page, see Lattice: Exercises.

Parents:
Order theory
Children:
Lattice: Exercises
Lattice: Examples
2
2
Discussion0
Discussion0