Arithmetic on families of ordinals #
Main definitions and results #
- sup,- lsub: the supremum / least strict upper bound of an indexed family of ordinals in- Type u, as an ordinal in- Type u.
- bsup,- blsub: the supremum / least strict upper bound of a set of ordinals indexed by ordinals less than a given ordinal- o.
Various other basic arithmetic results are given in Principal.lean instead.
Families of ordinals #
There are two kinds of indexed families that naturally arise when dealing with ordinals: those indexed by some type in the appropriate universe, and those indexed by ordinals less than another. The following API allows one to convert from one kind of family to the other.
In many cases, this makes it easy to prove claims about one kind of family via the corresponding claim on the other.
Converts a family indexed by a Type u to one indexed by an Ordinal.{u} using a specified
well-ordering.
Equations
- Ordinal.bfamilyOfFamily' r f a ha = f ((Ordinal.enum r) ⟨a, ha⟩)
Instances For
Converts a family indexed by a Type u to one indexed by an Ordinal.{u} using a well-ordering
given by the axiom of choice.
Instances For
Converts a family indexed by an Ordinal.{u} to one indexed by a Type u using a specified
well-ordering.
Equations
- Ordinal.familyOfBFamily' r ho f i = f ((Ordinal.typein r).toRelEmbedding i) ⋯
Instances For
Converts a family indexed by an Ordinal.{u} to one indexed by a Type u using a well-ordering
given by the axiom of choice.
Equations
- o.familyOfBFamily f = Ordinal.familyOfBFamily' (fun (x1 x2 : o.toType) => x1 < x2) ⋯ f
Instances For
The range of a family indexed by ordinals.
Instances For
Supremum of a family of ordinals #
The range of an indexed ordinal function, whose outputs live in a higher universe than the
inputs, is always bounded above. See Ordinal.lsub for an explicit bound.
le_ciSup whenever the input type is small in the output universe. This lemma sometimes
fails to infer f in simple cases and needs it to be given explicitly.
ciSup_le_iff' whenever the input type is small in the output universe.
An alias of ciSup_le' for discoverability.
lt_ciSup_iff' whenever the input type is small in the output universe.
Alias of iSup_succ.
Alias of Ordinal.IsNormal.apply_of_isSuccLimit.
The supremum of a family of ordinals indexed by the set of ordinals less than some
o : Ordinal.{u}. This is a special case of iSup over the family provided by
familyOfBFamily.
Equations
- o.bsup f = iSup (o.familyOfBFamily f)
Instances For
Alias of Ordinal.iSup_eq_iSup.
Alias of Ordinal.iSup'_eq_bsup.
Alias of Ordinal.iSup_eq_bsup.
Alias of Ordinal.bsup'_eq_iSup.
Alias of Ordinal.bsup_eq_iSup.
The least strict upper bound of a family of ordinals.
Equations
- Ordinal.lsub f = iSup (Order.succ ∘ f)
Instances For
Alias of Ordinal.lsub_notMem_range.
Alias of Ordinal.iSup_eq_lsub.
Alias of Ordinal.iSup_le_lsub.
Alias of Ordinal.lsub_le_succ_iSup.
Alias of Ordinal.succ_iSup_le_lsub_iff.
Alias of Ordinal.succ_iSup_eq_lsub_iff.
Alias of Ordinal.iSup_eq_lsub_iff.
Alias of Ordinal.iSup_eq_lsub_iff_lt_iSup.
Alias of Ordinal.iSup_typein_limit.
Alias of Ordinal.iSup_typein_succ.
The least strict upper bound of a family of ordinals indexed by the set of ordinals less than
some o : Ordinal.{u}.
This is to lsub as bsup is to sup.
Equations
- o.blsub f = o.bsup fun (a : Ordinal.{?u.22}) (ha : a < o) => Order.succ (f a ha)
Instances For
Results about injectivity and surjectivity #
Alias of not_surjective_of_ordinal.
Alias of not_injective_of_ordinal.
The type of ordinals in universe u is not Small.{u}. This is the type-theoretic analog of
the Burali-Forti paradox.