Von Neumann ordinals #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
This file works towards the development of von Neumann ordinals, i.e. transitive sets, well-ordered
under ∈
. We currently only have an initial development of transitive sets.
Further development can be found on the branch von_neumann_v2
.
Definitions #
Set.is_transitive
means that every element of a set is a subset.
Todo #
- Define von Neumann ordinals.
- Define the basic arithmetic operations on ordinals from a purely set-theoretic perspective.
- Prove the equivalences between these definitions and those provided in
set_theory/ordinal/arithmetic.lean
.
A transitive set is one where every element is a subset.
Alias of the forward direction of Set.is_transitive_iff_mem_trans
.
@[protected]
theorem
Set.is_transitive.inter
{x y : Set}
(hx : x.is_transitive)
(hy : y.is_transitive) :
(x ∩ y).is_transitive
@[protected]
theorem
Set.is_transitive.sUnion'
{x : Set}
(H : ∀ (y : Set), y ∈ x → y.is_transitive) :
(⋃₀ x).is_transitive
@[protected]
theorem
Set.is_transitive.union
{x y : Set}
(hx : x.is_transitive)
(hy : y.is_transitive) :
(x ∪ y).is_transitive
@[protected]
Alias of the forward direction of Set.is_transitive_iff_sUnion_subset
.
Alias of the forward direction of Set.is_transitive_iff_subset_powerset
.