Subdirect irreducibility and simplicity of lattices #
We prove that there exists a lattice that is subdirectly irreducible but not simple.
0
/
| 4
3 |
| 2
\ /
1
A lattice L is subdirectly irreducible if it contains two elements
a, b that are identified by any nontrivial congruence.
(We also allow the trivial case |L| ≤ 1.)
Equations
- SubdirectlyIrreducible l = ((∀ (a b : A), a = b) ∨ ∃ (a : A) (b : A), a ≠ b ∧ ∀ (R : A → A → Prop), congruence l R → R ≠ Eq → R a b)
Instances For
theorem
preserve_sup_of_indiscernible
{A : Type u_1}
(l : Lattice A)
(x y : A)
(hxy' : ∀ z ∉ Set.Icc x y, ∀ w₀ ∈ Set.Icc x y, ∀ w₁ ∈ Set.Icc x y, (w₀ ≤ z ↔ w₁ ≤ z) ∧ (z ≤ w₀ ↔ z ≤ w₁))
(x₀ x₁ y₀ y₁ : A)
:
An interval [x,y] is indiscernible if its elements u agree on
whether they are above or below a given element z ∉ [x,y].
The equivalence relation formed by collapsing such an interval
preserves ∨.
Simple implies subdirectly irreducible. ((D 5) is an example of the failure of the converse.) M₃ is simple.
The principal equivalence relation with block {2,4}
preserves ∧ in (D 5).
There exists a lattice that is subdirectly irreducible
but not simple, namely N₅.