Skip to content

Commit 13c52d6

Browse files
committed
chore(SetTheory/Cardinal/Ordinal): split file (#16990)
We split this file into two: - `Cardinal/Aleph`: contains the definitions for the aleph and beth functions (and soon, the omega function). - `Cardinal/Arithmetic`: any results on cardinal arithmetic that depend on `c * c = c` (which requires some basic properties of ordinals to be proven) These files are otherwise unchanged, with the exception of tweaking some section headers.
1 parent eab6727 commit 13c52d6

File tree

15 files changed

+478
-457
lines changed

15 files changed

+478
-457
lines changed

Mathlib.lean

Lines changed: 2 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -4141,6 +4141,8 @@ import Mathlib.RingTheory.WittVector.Truncated
41414141
import Mathlib.RingTheory.WittVector.Verschiebung
41424142
import Mathlib.RingTheory.WittVector.WittPolynomial
41434143
import Mathlib.RingTheory.ZMod
4144+
import Mathlib.SetTheory.Cardinal.Aleph
4145+
import Mathlib.SetTheory.Cardinal.Arithmetic
41444146
import Mathlib.SetTheory.Cardinal.Basic
41454147
import Mathlib.SetTheory.Cardinal.Cofinality
41464148
import Mathlib.SetTheory.Cardinal.Continuum
@@ -4149,7 +4151,6 @@ import Mathlib.SetTheory.Cardinal.Divisibility
41494151
import Mathlib.SetTheory.Cardinal.ENat
41504152
import Mathlib.SetTheory.Cardinal.Finite
41514153
import Mathlib.SetTheory.Cardinal.Finsupp
4152-
import Mathlib.SetTheory.Cardinal.Ordinal
41534154
import Mathlib.SetTheory.Cardinal.PartENat
41544155
import Mathlib.SetTheory.Cardinal.SchroederBernstein
41554156
import Mathlib.SetTheory.Cardinal.Subfield

Mathlib/Algebra/Quaternion.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -7,7 +7,7 @@ import Mathlib.Algebra.Algebra.Equiv
77
import Mathlib.LinearAlgebra.Dimension.StrongRankCondition
88
import Mathlib.LinearAlgebra.FreeModule.Basic
99
import Mathlib.LinearAlgebra.FreeModule.Finite.Basic
10-
import Mathlib.SetTheory.Cardinal.Ordinal
10+
import Mathlib.SetTheory.Cardinal.Arithmetic
1111

1212
/-!
1313
# Quaternions

Mathlib/Data/W/Cardinal.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Chris Hughes
55
-/
66
import Mathlib.Data.W.Basic
7-
import Mathlib.SetTheory.Cardinal.Ordinal
7+
import Mathlib.SetTheory.Cardinal.Arithmetic
88

99
/-!
1010
# Cardinality of W-types

Mathlib/ModelTheory/Encoding.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -6,7 +6,7 @@ Authors: Aaron Anderson
66
import Mathlib.Computability.Encoding
77
import Mathlib.Logic.Small.List
88
import Mathlib.ModelTheory.Syntax
9-
import Mathlib.SetTheory.Cardinal.Ordinal
9+
import Mathlib.SetTheory.Cardinal.Arithmetic
1010

1111
/-!
1212
# Encodings and Cardinality of First-Order Syntax

Mathlib/Order/Filter/CardinalInter.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -5,7 +5,7 @@ Authors: Josha Dekker
55
-/
66
import Mathlib.Order.Filter.Basic
77
import Mathlib.Order.Filter.CountableInter
8-
import Mathlib.SetTheory.Cardinal.Ordinal
8+
import Mathlib.SetTheory.Cardinal.Arithmetic
99
import Mathlib.SetTheory.Cardinal.Cofinality
1010

1111
/-!

Mathlib/Order/Filter/Cocardinal.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -6,7 +6,7 @@ Authors: Josha Dekker
66
import Mathlib.Order.Filter.Cofinite
77
import Mathlib.Order.Filter.CountableInter
88
import Mathlib.Order.Filter.CardinalInter
9-
import Mathlib.SetTheory.Cardinal.Ordinal
9+
import Mathlib.SetTheory.Cardinal.Arithmetic
1010
import Mathlib.SetTheory.Cardinal.Cofinality
1111
import Mathlib.Order.Filter.Bases
1212

Mathlib/RingTheory/Localization/Cardinality.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -3,7 +3,7 @@ Copyright (c) 2022 Eric Rodriguez. All rights reserved.
33
Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Eric Rodriguez
55
-/
6-
import Mathlib.SetTheory.Cardinal.Ordinal
6+
import Mathlib.SetTheory.Cardinal.Arithmetic
77
import Mathlib.RingTheory.Artinian
88

99
/-!

0 commit comments

Comments
 (0)