You are on page 1of 10

Chapter 2. Ordinals, well-founded relations.

2.1. Well-founded Relations.

We start with some definitions and rapidly reach the notion of a well-ordered set.

Definition. For any X and any binary relation < on X, (X, <) is a partially ordered set (p.o. set)
if < is a transitive and anti-symmetric relation on X:

∀x ∈ Xx 6< x and ∀x ∈ X ∀y ∈ X ∀z ∈ X (x < y & y < z −→ x < z).

Let us say that < partially orders X or < is a partial order of X.

(X, <) is a linearly ordered set (l.o. set) ou a totally ordered set (t.o. set) if (X, <) is a partially
ordered set and ∀x ∈ X ∀y ∈ X (x < y or x = y or y < x) as well.

Definition. Now let < be any binary relation on X. If Y ⊆ X, then (Y, <) is an initial segment
of (X, <) if ∀x ∈ X ∀y ∈ X (x < y & y ∈ Y −→ x ∈ Y ). Often we will just say that Y is an initial
segment of X when it is clear about which relation < we are talking. (Y, <) is a proper initial
segment of (X, <) if Y 6= X as well. For all s ∈ X and Y ⊆ X, we say that s is a successor of Y
if s ∈
/ Y and { y ∈ X | y < s } ⊆ Y . And if Y ⊆ X and y ∈ X we say that y is <-minimal in Y if
y ∈ Y and ∀x ∈ X (x < y −→ x ∈ / Y ).

Theorem. The following conditions are equivalent for any X and any binary relation on X.
(1) Each proper initial segment of X has a successor.
(2) Each non-empty subset of X has a <-minimal element.
(3) The principle of induction on < is true:  
∀x ∈ X ∀y ∈ X (y < x −→ φ(y)) −→ φ(x) −→ ∀x ∈ X φ(x).
 
Proof. (2) =⇒ (3). Suppose that ∀x ∈ X ∀y ∈ X (y < x −→ φ(y)) −→ φ(x) but
¬∀x ∈ X φ(x). Then {x ∈ X | ¬φ(x)} is non-empty and, by (2), has a member, let us say x0 ,
which is <-minimal. But then we have that ∀y < x0 φ(y) and hence φ(x), a contradiction.

(3) =⇒ (2). If Y ⊆ X and Y does not have a <-minimal element, then we have that

∀x ∈ X (∀y ∈ X(y < x & y ∈


/ Y )) −→ x ∈
/ Y.

Applying (3), we have that ∀x ∈ X x ∈


/ Y . Thus Y is empty.

(2) =⇒ (1). If Y is a proper initial segment of X, then X \ Y (= { x ∈ X | x ∈ / Y }) is non-empty,


and (2) says that there is a member, let us call it s, that is <-minimal. Hence s is a successor of Y .

(1) =⇒ (2). For all x, y ∈ X let x <∗ y if there are x0 , . . . , xn−1 ∈ X and x < x0 < . . . < xn−1 < y.
<∗ is the transitive closure of <: it is transitive, <⊆<∗ and if R is a transitive binary relation with
<⊆ R, then <∗ ⊆ R.

(In order to see that <∗ is transitive take x <∗ y and y <∗ z and suppose that we have this because
x < x0 < . . . < xn−1 < y and y < y0 < . . . < ym−1 < z for some x0 , . . . , xn−1 , y0 , . . . , ym−1 ∈ X.
Thus, x < x0 < . . . < xn−1 < y < y0 < . . . < ym−1 < z, and so x < z. It is clear that
x < y =⇒ x <∗ y: take n = 0 in the definition of <∗ . And if x <∗ y there are x0 < . . . < xn−1 with

version 1.1, 12/2/06

1
x < x0 < . . . < xn−1 < y, so if <⊆ R we have x R x0 R . . . Rxn−1 Ry, and hence, if R is transitive,
we have x R y.)

Now suppose that Y ⊆ X and Y is non-empty. { x ∈ X | x ∈ / Y & ∀y ∈ X (y <∗ x −→ y ∈ / Y )},


= Z, let us say, is an initial segment and is proper. If s is a successor of Z we have that s ∈ Y and
s is <-minimal in Y .

Definition. A binary relation < on a set X is well-founded if satisfies the conditions (1)-(3) of the
above theorem. A well-founded total order is called well-ordered or a well-ordering. (X, <) is then
a well-ordered set (a w.o. set).

2.2 Ordinals.

Thus, a well-ordered set is a set along which we can “count” one step at a time. The ordinals are
well-ordered sets that will be crucial for us. In fact we will see later that any well-ordered set is
isomorphic to some ordinal via an isomorphism which is order-preserving, hence one can say that
if we want to “count” we have to use the ordinals.

Definition. An ordinal is a transitive set that is well-ordered by ∈. (Frequently we will write <
instead of ∈ when we are dealing with ordinals.)

Examples. 0, 1, 2, 3, . . . , ω, . . . are (the first) ordinals. Exercise: if this is not apparent to you
then check it.

Proposition. If α is an ordinal and z ∈ α, then z is a transitive set and hence is a ordinal as well.

Proof. Let us suppose that x ∈ y ∈ z ∈ α. We have to show that x ∈ z. But α is transitive, so


y ∈ α, and thus x ∈ α. α is also well-ordered by ∈, hence ∈ is a transitive relation on α. Because
we have x ∈ y and y ∈ z, one has x ∈ z.

Definition. If α is an ordinal define s(α) = α ∪ {α }.

Proposition. If α is an ordinal, then s(α) is an ordinal as well.

Proof. If z ∈ y ∈ s(α), then either z ∈ y ∈ α or z ∈ y ∈ { α }. In the first case z ∈ α because ∈


is transitive on α, and in the second case z ∈ y = α. Hence, in any caso z ∈ s(α). Thus s(α) is
transitive. And it is clear that s(α) is well-ordered by ∈.
T
Proposition. If x 6= ∅ is a set of ordinals, then x is also an ordinal.
T
Proof. It is clear that any intersection of transitive sets is transitive. And if α ∈ x, then x⊆α
and must be well-ordered by ∈ α is well-ordered by ∈.

Proposition. If α, β are ordinals and α ⊆ β, then (a) α is an initial segment of β, and (b)
α 6= β =⇒ α ∈ β.

Proof. (a) If γ ∈ β, δ ∈ α and γ ∈ δ (i.e., γ comes before δ in the well-order of β by ∈), so


γ ∈ δ ∈ α, and thus γ ∈ α by the transitivity of ∈ on α.

(b) If α 6= β, then, by the equivalent of being well-founded, there is a sucessor, let us call it s, of
α as a subset of β. Note that s is unique because ∈ is a l.o. of β. Also, because ∈ is a l.o. of β,
γ ∈ α implies that γ ∈ s, thus α ⊆ s. On the other hand, S = α ∪ { s} is an initial segment of β
and, thus, it is transitive and, so, for any γ ∈ s(∈ S) we have γ ∈ S. Because s ∈/ s (by the axiom
of foundation), γ ∈ s implies γ ∈ α and s ⊆ α. Hence α = s, ∈ β.

2
2.3. Trichotomy.

Theorem. If α and β are ordinals one and exactly one of the following holds: α ∈ β or α = β or
β < α.

Proof. α ∩ β = α or α ∩ β ⊂ α and α ∩ β 6= α. Similarly α ∩ β = β or α ∩ β ⊂ β and α ∩ β 6= β,


giving four cases for us to consider.

(i) α ∩ β = α and α ∩ β = β. Then α = β.

(ii) α ∩ β = α and α ∩ β ⊂ β and α ∩ β 6= β. Then the last proposition of §2.2 immediately gives
that α ∈ β.

(iii) α ∩ β = β and α ∩ β ⊂ α and α ∩ β 6= α. Then the last proposition of §2.2 gives that β ∈ α.

(iv) α∩β ⊂ α, β, α∩β 6= α and α∩β 6= β. Note that we have already shown that α∩β is an ordinal.
Then the last proposition of §2.2 gives that α ∩ β ∈ α and that α ∩ β ∈ β. Henceα ∩ β ∈ α ∩ β, a
contradiction! (To the axiom of foundation.)

Corollary. For all ordinals α and β, α ⊆ β or β ⊆ α.

Proof. α ∈ β =⇒ α ⊆ β because β is transitive; β ∈ α =⇒ β ⊆ α because α is transitive;


α = β =⇒ α ⊆ β & β ⊆ α.

Notation. We write α ≤ β if α ∈ β or α = β.

Corollary. The collection of all ordinals is well-ordered by ∈.

Proof. It is easy to see that the collection is partially ordered by ∈ by the transitivity of ordinals.
The trichotomy theorem gives that ∈ totally orders the collection. Hence what remains to be shown
is that ∈ is well-founded on the collection.

Suppose that Z is a subset of the collection of all ordinals and Z 6= ∅. Let α ∈ Z. Either α is
∈-minimal (when we are finished), or Y = α ∩ Z 6= ∅. Y is a non-empty subset of α, hence there is
some β ∈ Y that is ∈-minimal. But β must be ∈-minimal in Z as well, because if γ ∈ β we have
that β ∈ α and, by the transitity of α, γ ∈ α. Hence γ ∈ Z.

Corollary. The collection of all ordinals is not a set: it is a proper class.

Proof. Suppose the collection was a set, x, let us say. Then we would have that x ∈ x by the
previous corollary and the definition of ordinal. This would contradict the axiom of foundation
(again).

This corollary is sometimes called the Burali-Forti paradox. As you’ve already see, as with Cantor’s
paradox, this is not in fact a true paradox. Again, as with V , it is convenient to have a name for
the (proper) class of all ordinals, and so we write On for this class.
S
Corollary. If x is a set of ordinals, then x is also an ordinal.
S S
Proof.SIt is clear that x is transitive.SAnd because x ⊆ On, trichotomy gives that ∈ totally
orders x. So, suppose that ∅ 6= Z ⊆ x. Take α ∈ Z. As in the corollary two ago, either α
already is ∈-minimal, or α ∩ Z has a member that is ∈-minimal and that is ∈-minimal in Z as well.

2.4. Successors and limits. Let α be an ordinal. There are two things that can happen.

3
Either there is a ∈-maximal element of α, i.e., a β ∈ α such that ∀γ ∈ α γ ≤ β. In this case
α = {β } ∪ {γ | γ < β }, = {β } ∪ β, = s(β). If there is some β such that α = s(β) we say that α is
a successor ordinal .

Or there is no ∈-maximal element (at the S i.e., ∀β ∈ α ∃γ ∈ α β < γ. In this case


S top) of α,
α = { β | β < α } = { β | ∃γ ∈ α β ∈ γ } = α. If α = α we say that α is a limit ordinal .
S
We must check that if α = s(β), then β = α.

Examples. 1, 2, 3, . . . are successor ordinals. ω is a limit ordinal. (And by our definition, 0 is a


limit ordinal as well, albeit that this is a special caso and is typically treated separately.)
S
In general, if x is a set of ordinals, x is the supremum of the ordinals in x, and if x is non-empty,
T
x is the infimum of the ordinals in x, and also the minimal element de x. (This latter is true
because we have already seen that x has ∈-minimal member Twhen ∅ 6= x ⊆ On, α, let us say, and
so ∀β ∈ x α ≤ β – i.e., ∀β ∈ x α ∈ β or α = β, whence α = x.)

2.5. Recursion Theorems. Now we want to define + and . on the ordinals, in a similar manner
to that in which we did on the natural numbers. But before we can do this we need to know that we
can make definitions using recursion and how to make these defintions. So this section is devoted
to that theme. Perhaps at first glance it will seem very technical, but it will be highly useful in the
end.

Weak recursion theorem. Let X, Y be two sets. Let < be a well-founded relation on X, and
let g : X × P (Y ) −→ Y be a function. Then there is a unique function f : X −→ Y such that
f (x) = g(x, { f (z) | z < x}) for all x ∈ X.

Proof. (Part 1.) We say that φ : Z −→ Y is an attempt if Z is an initial segment of X and


φ(x) = g(x, {φ(z) | z < x}) for all x ∈ Z. If φ0 : Z0 −→ Y and φ1 : Z1 −→ Y are two
attempts, they agree on Z1 ∩ Z2 : φ1  Z1 ∩ Z2 = φ2  Z1 ∩ Z2 . Because X1 ∩ X2 is clearly
an initial segment of X and if as attempts they do not agree there is some x0 which is <-minimal
in {x ∈ Z1 ∩ Z2 | φ1 (x) 6= φ2 (x)}. But in that case we have φ1 (x0 ) = g(x0 , { φ0 (x) | x < x0 }) =
g(x0 , {φ1 (x) | x < x0 }) = φ2 (x), a contradiction!
S
(Part 2.) Now let f = { φ | φ is an attempt S }, so f (x) = φ(x) if there is an attempt φ with
x ∈ dom(φ). It is clear that dom(f ) = { dom(φ) | φ is an attempt } is an initial segment of X,
and that f satisfies f (x) = g(x, { f (z) | z < x}) for allx ∈ dom(f ). So all that remains to be shown
is that dom(f ) = X.

But if dom(f ) 6= X there is some x0 that is <-minimal in {x ∈ X | x ∈ / dom(f )}. For such an x
¯ ¯ ¯
define f : dom(f ) ∪ { x0 } −→ Y by f (x) = f (x) if x ∈ dom(f ) and f (x0 ) = g(x0 , {f (x) | x < x0 }).
Then one would clearly have that f¯ is an attempt, but is not a subset of f . contradiction! Hence
f : X −→ Y as we want.

Now we shall see a stronger recursion theorem which deals with classes.

Definition. Let A and B be classes. Thus A × B = { (x, y) | x ∈ A & y ∈ B } is a class as well,


because if A = { x | φ(x, ā)} and B = {x | ψ(x, b̄)} for two formulas φ(x, ā) and ψ(x, b̄) in LTC,
then A × B = { z | z = {{x}, {x, y }} & φ(x, ā) & φ(y, b̄)}.

Let A be a class. < is a well-founded Relation (note the capital “R”) on A if < is a subclass do
A × A, ∀a ∈ A { b ∈ A | b < a} is a set, and any B with ∅ =
6 B ⊆ A has <-minimal elements.

Let A, B be classes. G : A −→ B is a Function (note the capital “F”) if G is a subclass of A × B

4
and for each x ∈ A there is a unique y ∈ B such that (x, y) ∈ G. If x ∈ A, y ∈ B and (x, y) ∈ G
we shall write (naturally) G(x) = y. (Note that to say that G is a (sub)class means that there is a
formula χ(z, c̄) in LTC such that x ∈ G if and only if χ(x, c̄) is true.)

Remember that sets are classes as well and if A and B are sets, then A × B is a set, < is a
well-founded relation and G is a function, respectively.

Strong recursion theorem. Let < be a well-founded Relation on a class A and G : A × V −→ V


a Function. Then there is a unique Function F : A −→ V such that for all x ∈ A we have that
F (x) = G(x, {F (y) | y < x}).

Proof. (Part 1.) The first part is just as in the weak recursion theorem. Define φ to be an attempt
if φ : B −→ V , where B is a set that is an initial segment of A and φ(x) = G(x, {φ(y) | y < x}).
Then any two attempts agree on the intersection of their initial segments.
S
(Part 2.) Let F = { φ | φ is an attempt } (that is (x, z) ∈ F if there is an attempt φ with φ(x) = z).
Note that the last time this was a set, but here we merely have that F ⊆ P (A × V ) and we do
not know that F is a set, since it will not be one if A is not. On the other hand we have that
F (x) = G(x, { F (y) | y < x}) for all x ∈ dom(F ). Suppose that dom(F ) 6= A, and choose a0 that is
<-minimal in the set A \ dom(F ).

Now we have that ∀b < a0 ∃φ (φ is an attempt and b ∈ dom(φ). By this we can apply the Ax-
iom of Collection which gives that ∃v ∀b < a0 ∃φ ∈ v (φ is an attempt and b ∈ dom(fS ). Hence
w = v ∩ { φ | φ is anattempt} is a set by the Axiom of Comprehension. Clearly f = w is an
attempt and we can consider f¯ = f ∪ {(a0 , G(a0 , {f (b) | b < a0 }))} which is an attempt but is not
a subset do f . Thus, as in the weak recursion theorem we have a contradiction! Hencedom(F ) = A.

Why are there differences in the proof from that of the weak recursion theory? Well, in order to
imitate that proof you would have to know that G(a0 , {F (a) | a < a0 }) makes sense before defining
F̄ = F ∪ { (a0 , G(a0 , { F (a) | a < a0 }))}. And in order to know this you would have to know that
{ F (a) | a < a0 } is a set, which is a consequence of applying Replacement to the set {a | a < a0 }.
Hence one sees that it is not possible to avoid the use of Collection or Replacement.

I ought to warn that one cannot avoid the use of Collection in the strong recursion theorem even
if A is a set if G is not one, and this is also so even if < is a well-order A and rather than just a
well-founded relation.

2.6 Comparison theorems.

Definition. A function f : (X, <X ) −→ (Y, <Y ) is an isomorphism which preserves order if f is a
bijetion between X and Y and ∀x, y ∈ X (x <X y ←→ f (x) <Y f (y)).

Note. If f : (X, <X ) −→ (Y, <Y ) is a function that preserves order f is injective, and so you only
need to know that f is also a surjection in order to have that f is an isomorphism.

Theorem. For any well-ordered set (X, <) there is a unique ordinal α for which there is an (unique)
isomorphism from (X, <) to α which preserves order.

Proof. Define, by the (weak) recursion theorem, a function f : X −→ V (On) which satisfies
f (x) = { f (y) | y < x}.

(i) ∀x ∈ X f (x) ∈ On. If not choose some x0 which is <-minimal in the set { x ∈ X | f (x) ∈/ On}.
Suppose that x ∈ X and for all y < x we have that f (y) ∈ On. Then f (x) ⊆ On by the definition
of f , and f (x) is well-ordered by ∈. But also, if z ∈ y ∈ f (x), we have that y = f (v) for some

5
v < x. Thus z ∈ {f (u) | u < v } and there is some u < v < x such that z = f (u). Consequently,
z ∈ f (x), and f (x) is transitive. Hence f (x) ∈ On. So, by the principle of indution on <, we have
that ∀x ∈ X f (x) ∈ On.

(ii) im(f ) is a set (by the axioms of collection and comprehension or by replacement), and (i) shows
that im(f ) ⊆ On, thus im(f ) is well-ordered by ∈. Suppose that z ∈ y ∈ im(f ), hence there is
some x ∈ X such that z ∈ y = f (x), and so there is some v ∈ X such that v < x and z = f (v).
This gives that z ∈ im(f ) and im(f ) ∈ On.

Finally if g : X −→ β is another isomorphism which preserves order, then f · g −1 would be an


isomorphism from β to α which preserves the order given by ∈. Thus β = α and f · g −1 is equal to
the identity function by (the first corollary to) trichotomy.

Comparison Theorem. Let (X, <X ) and (Y, <Y ) be two w.o.sets. Then there is an isomorphism
that preserves order between one of them and an initial segment of the other.

Proof. The previous theorem says that there are α, β ∈ On and isomorphisms f : (X, <X ) −→ α
and g : (Y, <Y ) −→ β which preserve order. Now we apply trichotomy. If α = β we have that g −1 ·f
is an order-preserving isomorphism between (X, <X ) and (Y, <Y ). If α ∈ β we have that g −1 · f is
an order-presrving isomorphism between (X, <X ) and a proper initial segment of (Y, <Y ) (of which
g −1 (α) is a successor). And if β ∈ α we have that f −1 · g is an isomorphism which preserves order
between (Y, <Y ) and a proper initial segment of (X, <X ) (of which f −1 (β) is a successor).

2.7. The Vα hierarchy.

Now we can rigorously define (from the axioms) the Vα hierarchy. Define, bySthe strong recursion
theorem, a Function V : On −→ V (the collection of all sets) such that Vα = { P (Vβ ) | β < α }.

Proposition. ∀α Vα is transitive.

Proof. If not choose α (<-)minimal such that Vα not transitive. We have already seen (in the first
proposition
S of §1.5) that P (X) is transitive if X is transitive. So ∀β < α P (Vβ ) is transitive. But
Vα = { P (Vβ ) | β < α } is a union of transitive sets and so is also transitive.

Proposition. If α ≤ β we have that Vα ⊆ Vβ .

Proof. If α = β it is trivial. If α < β, then Vα ⊆ P (Vα ), because Vα and, so, P (Vα ) are transitive,
and P (Vα ) ⊆ Vβ .

Corollary. If α is a successor ordinal, then Vs(α) = Vα+1 = P (Vα ).


S S
Proof. Vs(α) = { P (Vβ ) | β ≤ αS} = { P (Vβ ) | β ≤ α } ∪ P (Vα ). But Vβ ⊆ Vα if β < α, and so
P (Vβ ) ⊆ P (Vα ) if β < α. Hence { P (Vβ ) | β ≤ α } ⊆ P (Vα ).
S
Corollary. If λ is a limit ordinal then Vλ = { Vα | α < λ }.
S S S S
Proof. { Vα | α < λ} ⊆ Vλ = { P (Vα ) | α < λ} = {Vs(α) | α < λ} ⊆ {Vα | α < λ} because
s(α) < λ if α < λ.

Theorem. The axiom of foundation is equivalent to “∀x ∃α ∈ On x ∈ Vα .”

Proof. “=⇒”. If not let x0 be ∈-minimal such that ∀β ∈ On x ∈ / Vβ . So ∀x ∈ x0 ∃β x ∈ Vβ .


If we apply the axiom of Collection we have ∃v ∀x ∈ x0 ∃β ∈ v x ∈ Vβ . Let u = v ∩ On. Then
∀x ∈ x0 ∃β ≤ sup(u) x ∈ Vβ , and this gives that ∀x ∈ x0 x ∈ Vsup(u) . It follows that x0 ⊆ Vsup(u) ,

6
and so that x0 ∈ Vs(sup(u)) . contradiction!
S
“⇐=”. Let A 6= ∅ be a class with A ⊆ { Vα | α ∈ On}. Take α minimal such that A ∩ Vα 6= ∅.
Then any a ∈ A ∩ Vα is ∈-minimal in A.
S
Definition. Define a function rk : V −→ V (On) by rk(x) = { s(rk(y)) | y ∈ x}, using the
(strong) recursion theorem.

Proposition. (i) ∀x ∈ V rk(x) ∈ On. (ii) rk(x) = the minimal α such that x ⊆ Vα . (iii) rk(x)+1 =
the minimal α such that x ∈ Vα .

Proof. Exercise. (Use induction over (V, ∈).)

2.8. Transitive closures.

For each set define, by recursion over (ω, ≤), a function t(n, x) such that
[
t(0, x) = x and t(n + 1, x) = t(n, x) ∪ t(n, x).
S
At the end, define TC(x) = { t(n, x) | n ∈ ω }. TC(x) is the transitive closure of x

Proposition. For every x, TC(x) is the minimal transitive set z with x ⊆ z. (That is, if y is
transitive and x ⊆ y, then TC(x) ⊆ y.)

S Let u ∈ v ∈ TC(x). Then there is some n < ω such that u ∈ v ∈ t(n, x).
Proof. So
u ∈ t(n, x) ⊆ t(n + 1, x) ⊆ TC(x). Thus TC(x) is transitive.

Let y be transitive x ⊆ y. We shall show by induction on ω that each t(n, x) ⊆ y. This is clear
whenS n = 0. Suppose that t(n, x) ⊆ y. If z ∈ t(n + 1, x) we either have z ∈ t(n, x), when z ∈ y, or
z ∈ t(n, x). So there is some v ∈ t(n, x) such that z ∈ v. But if z ∈ v ∈ t(n,Sx) ⊆ y, we have that
z ∈ y by the transitivity of y. So we have t(n + 1, x) ⊆ y, and thus TC(x) = t(n, x) ⊆ y.

Proposition. The axiom of foundation for sets (each non-empty set has a ∈-minimal element)
implies the axiom of foundation for classes (each non-empty class has a ∈-minimal element).

Proof. Let A, 6= ∅, be a class. Let x ∈ A. Either x is ∈-minimal (when we are done) or x ∩ A 6= ∅.


Then TC(x) ∩ A 6= ∅. Let y be ∈-minimal in the set TC(x) ∩ A. (We know that it is a set by the
previous proposition.) We have that y ∈ A. Now suppose that z ∈ y. Then z ∈ / TC(x) ∩ A. But
z ∈ y ∈ TC(x) and TC(x) is transitive, so z ∈ TC(x). Thus z ∈ / A, and we have shown that y is
∈-minimal in the class A.

2.9. Ordinal arithmetic: addition of ordinals.

We will use recursion to define addition and mutlipication on On.

Definition. Define, for α fixed and β variable, α + β = α ∪ {α + γ | γ < β }

Proposition. Let α, β ∈ On. Then α + β ∈ On.

Proof. If not, let β0 be minimal with α + β0 ∈


/ On. Then for all γ < β0 we have that α + γ ∈ On,
so α + β0 = α ∪ {α + γ | γ < β0 } ⊆ On and, hence, is well-ordered by ∈.

Now we will show that α + β0 is transitive, and so is an element of On, giving a contradiction to
the supposition. Let z ∈ y ∈ α ∪ { α + γ | γ < β0 }. Then, either y ∈ α, when z ∈ α, because α is

7
an ordinal, or there is some γ < β such that y = α + γ ∈ On, hence, again, z ∈ { α + δ | δ < γ }. In
each case we have that z ∈ α + { α + γ | γ < β0 }, giving the desired contradiction. So α + β0 ∈ On.

Lemma. ∀α, β, γ, δ ∈ On: (i) β < γ =⇒ α + β < α + γ; (ii) α ≤ δ =⇒ α + β ≤ δ + β.

Proof. (i) If β < γ, then α + β ∈ α + γ.


(ii) Suppose that the Lemma is false for some pair α and δ, and let β0 be minimal such that
α + β 6≤ δ + β. Then ∀β < β0 we have that α + β ≤ δ + β and so either α + β = δ + β or
α + β < δ + β. In the latter case either there is some γ < β such that α + β = δ + γ, or α + β ∈ δ.
So α + β0 = α ∪ {α + β | β < β0 } ⊆ δ ∪ {δ + γ | γ < β0 } = δ + β0 .

Proposition.
S (i) α + 0 = α; (ii) α + s(β) = s(α + β); (iii) if λ is a limit ordinal, then
α + λ = { α + γ | γ < λ}.

Proof. (i) Trivial.


(ii) α + s(β) = α ∪ {α + γ | γ < s(β)} = α ∪ {α + γ | γ < s(β)} = α ∪ {α + γ | γ < β } ∪ {α + β } =
(α + β) ∪ {αS + β } = s(α + β).
(iii) if x ∈ { α + γ | γ < λ } then there is some
S γ <Sλ such that x ∈ α ∪ { α + β | β < γ }. Thus
x ∈ α∪{α+β | β < λ}. But we know that λ = λ = {γ | γ < λ}, hence if x ∈ α∪{α+β | β < λ}
S x ∈ α or x = α + β for some β < λ and there is some γ < λ such that β < γ. Hence
either
x ∈ { α + γ | γ < λ}.

Theorem. Let α, β ∈ On and let ≺ be the anti-lexicografic order on α × {0} ∪ β × {1 } defined by


(γ, i) ≺ (δ, j) if and only if either i < j or i = j and γ < δ. So this order is isomorphic to (α + β, ∈)

Proof. Define a function f : α × {0 } ∪ β × {1} −→ α + β by f (γ, 0) = γ and f (δ, 1) = α + δ.


It is clear that f is surjective and also that ≺ is a total order on dom(f ). We shall show that
(γ, i) ≺ (δ, j) implies f (γ, i) < f (δ, j).

If i < j then i = 0 and j = 1, f (γ, i) = γ and f (δ, j) = α + δ, and we have that γ < α ≤ α + δ.
If i = j = 0, then f (γ, i) = γ and f (δ, j) = δ and we have γ < δ. And if i = j = 1 we have that
α + γ < α + δ by the previous lemma.

Note. 1 + ω = ω, while ω + 1 = s(ω), so + is non-comutative in general.

INSERT Pictures of 1 + ω and ω + 1.

S S
Proposition. If x ⊆ On is a non-empty set then α + x= {α + β | β ∈ x}. (+ is continuous
in the second place/variable.)
S S S S
Proof. If β ∈ x then β ≤ x, and so ∀β ∈ x (α+β ≤ α+ x). Hence {α+β | β ∈ x} ⊆ α+ x.
S S S
Let ρ = { α + β | β ∈ x} If ρ ∈ α + x, then either ρ ∈ α or there is some γ ∈ x such S that
ρ = α + γ. If ρ ∈ α, then ∀β ∈ x α + β ≤ ρ < α, a contradiction. And ifSρ = α + γ with γ ∈ x,
then there is some β ∈ x such that
S γ < β and so ρ < α + β and S ρ < { α + β | β ∈ x} = ρ, a
contradiction again. So, ρ ∈
/ α + x and we have that ρ = α + x.

We can define subtraction as well, but because addition is not commutativity it is not as useful as
addition.

Definition. α − β = { γ | β + γ < α }. Alternatively one can define α − β by recursion: α − β = 0

8
if β > α and α − β = {α − γ | γ < β } if β ≤ α.

Proposition. Let α, β ∈ On and β ≤ α. Then β + (α − β) = α.

Proof. β + (α − β) = β ∪ { β + γ | γ < α − β } = β ∪ { β + γ | β + γ < α } ⊆ α. Suppose that


β + (α − β) < α. Then (α − β) ∈ { γ | β + γ < α } = α − β. A contradiction. So β + (α − β) = α.

Note. (α − β) + β 6= α in general. For example, ω − 1 = ω, hence (ω − 1) + 1 = s(ω) 6= ω.

2.10 Ordinal aritmetic: multiplication of ordinals.

By the recursion theorem define α.β = { α.γ + δ | γ < β & δ < α }.

Proposition. ∀α, β ∈ On (α.β ∈ On).

Proof. Suppose that α.γ ∈ On for each γ < β. So α.γ + δ ∈ On for each γ < β by the
proposition that ξ + ζ ∈ On if ξ, ζ ∈ On, and we have that α.β ⊆ On and hence is well-ordered
by ∈. Also, for each γ < β the function fγ : α −→ {α.γ + δ | δ < α } given by fγ (δ) = α.γ + δ has
fγ “α = { α.γ +δ | δ < α }, and hence { α.γ +δ | δ < α }, Aγ let’s call it, is a set by Replacement.
S Let g
S given by γ 7→ Aγ for all γ < β. Then g“β is again a set and so α.β = {Aγ | γ < β }
be the function
is the union g“β of a set and is also a set. Finally, if x ∈ y ∈ α.β, then there is some γ < β
and δ < α such that x ∈ y = α.γ + δ. Hence either x ∈ α.γ or there is some σ < δ such that
x = α.γ + σ. In the first case there are some  < γ and τ < α such that x = α. + τ . So in each
case we have that x ∈ α.β. Because we now have that ∀β (∀γ < β (α.γ ∈ On) −→ α.β ∈ On), we
have that ∀β ∈ On α.β ∈ On.

Lemma. ∀α ∈ On (i) 0.α = 0; (ii) 1.α = α; (iii) ∀β, γ ∈ On (β < γ) =⇒ α.β < α.γ; and (iv) ∀δ
β ∈ On, (α ≤ δ =⇒ α.β ≤ δ.β).

Proof. (i)–(iii) are obvious. (iv) Suppose that α, δ ∈ On, β ∈ On and for all γ < β we have that
α.γ ≤ δ.γ. Using the lemma about addition from §2.8, we have for all γ < β and all  < α that
α.γ +  ≤ δ.γ + . Hence either α.γ +  = δ.γ + , when α.γ +  ∈ δ.β, or α.γ +  ∈ δ.γ +  ∈ δ.β,
and α.γ +  ∈ δ.β, by the transitivity of δ.β. In each case we have that α.β ⊆ δ.β and so α.β ≤ δ.β.
But this shows that (∀γ < β α.β ≤ δ.γ) −→ α.β ≤ δ.β. Hence, because < is well-founded on the
ordinals, ∀β ∈ On α.β ≤ δ.β.

Proposition.
S (i) α.0 = 0; (ii) α.s(α) = α.β + α; and (iii) if λ ∈ On is a limit ordinal, then
α.λ = { α.γ | γ < λ}.

Proof. (i) Trivial.


(ii) α.s(β) = {α.γ + δ | γ ≤ β & δ < α } = { α.γ + δ | γ < β & δ < α } ∪ {α.β + δ | δ < α } = α.β + α.
(iii) If λ is a limit ordinal then
[
{ α.β | β < λ} = {α.γ + δ | (∃β < λ γ < β) & δ < α } =
[
{ α.γ + δ | γ ∈ λ & δ < α } = { α.γ + δ | γ < λ & δ < α, }

with this last step because λ is a limit ordinal.

Theorem. Let α, β ∈ On and let ≺ be the anti-lexicographic order on α × β, defined by


(δ0 , γ0 ) ≺ (δ1 , γ1 ) if γ0 < γ1 or if γ0 = γ1 and δ0 < δ1 . Hence (α × β, ≺) is isomorphic to
(α.β, ∈) via an order-preserving isomorphism.

Proof. Define f : α × β −→ α.β by f (δ, γ) = α.γ + δ. It is clear that f is a surjection. If


(δ0 , γ0 ) ≺ (δ1 , γ1 ) either γ0 < γ1 when α.γ0 + δ0 < α.s(γ0 ) ≤ α.γ1 ≤ α.γ1 + δ1 , or γ0 = γ1 and

9
δ0 < δ1 , when α.γ0 + δ0 < α.γ0 + δ1 by the lemma about addition. Hence, f preserves order, and
so is an isomorphism.

Note. 2.ω = ω, 3.ω = ω, . . . , but ω.ω 6= ω. Note also that (ω + 1).ω = ω.ω

Theorem. Let α, β ∈ On, β > 0. Then there are unique σ, τ with τ < β such that α = β.σ + τ .

Proof. Let σ = { γ | β.s(γ) ≤ α } and τ = α − β.σ, = {δ | β.σ + δ < α }. Hence α = β.σ + τ .


In order to see that τ < β, observe that if not either β = τ , when α = β.σ + β = β.s(σ) or
β ∈ {δ | β.σ + δ < α } and, so, β.σ + β = β.s(σ) < α. So in any case β.s(σ) ≤ α and σ ∈ σ, a
contradiction!
S S
Proposition. If x ⊆ On then α. x= { α.β | β ∈ x}. (Which means that . is continuous in the
second place/variable.)
S
Proof.
S α. x = {α.γ + δ | δ < α & (∃β ∈ x γ < β)} = { α.γ + δ | ∃β ∈ x (γ < β & δ < α)}
= { α.β | β ∈ x}.
S
Note. In the previous theorem σ = {γ | β.γ ≤ α }.

Ordinals arithmetic: 2.11 Exponentiation of ordinals.

Next we make another definition by recursion and define exponentiation.

Definition. Let α, β ∈ On. Then αβ = {0 } ∪ {αγ .δ +  | γ < β & δ < α &  < αγ }.

Proposition. Let α, β ∈ On. Then αβ ∈ On.

Lemma. ∀α, β, γ δ ∈ On we have (i) αβ .αγ = αβ+γ ; (ii) (αβ )γ = αβ.γ ; (iii) β < γ =⇒ αβ < αγ ;
and (iv) α ≤ δ =⇒ αβ ≤ δ β .

α ∈ On. (i) α0 = 1; (ii) αs(β) = αβ .α for each β ∈ On; and (iii) if λ is a limit
Proposition. Let S
ordinal, then α = {αγ | γ < λ}.
λ

The proofs are similar to the proofs of the equivalents for ‘.’. You should check these if you desire.
ω
Note. ∀n ∈ ω nω = ω, but ω ω 6= ω, when ω.ω ω = ω ω . And if we define 0 = { ω, ω ω , ω ω , . . . },
S
then ω 0 = 0 .

When you come back to this section later you should remember that all of these facts are for
exponentiations of ordinals, that is very different from the theory of cardinal exponentiation that
we will see in Chapter (4).

10

You might also like