Skip to content

Commit

Permalink
fix(Cardinal): fix theorem names (#10465)
Browse files Browse the repository at this point in the history
Remove unnecessary `of_lt_aleph_0` from 2 theorem names. Also fix typos in the comments of 2 other files.



Co-authored-by: damiano <adomani@gmail.com>
  • Loading branch information
YnirPaz and adomani committed Feb 12, 2024
1 parent a694837 commit a6f1457
Show file tree
Hide file tree
Showing 3 changed files with 12 additions and 6 deletions.
2 changes: 1 addition & 1 deletion Mathlib/SetTheory/Cardinal/Basic.lean
Expand Up @@ -61,7 +61,7 @@ We define cardinal numbers as a quotient of types under the equivalence relation
`Cardinal.{u} : Type (u + 1)` is the quotient of types in `Type u`.
The operation `Cardinal.lift` lifts cardinal numbers to a higher level.
* Cardinal arithmetic specifically for infinite cardinals (like `κ * κ = κ`) is in the file
`SetTheory/CardinalOrdinal.lean`.
`SetTheory/Cardinal/Ordinal.lean`.
* There is an instance `Pow Cardinal`, but this will only fire if Lean already knows that both
the base and the exponent live in the same universe. As a workaround, you can add
```
Expand Down
14 changes: 10 additions & 4 deletions Mathlib/SetTheory/Cardinal/Ordinal.lean
Expand Up @@ -944,14 +944,20 @@ theorem add_le_add_iff_of_lt_aleph0 {α β γ : Cardinal} (γ₀ : γ < Cardinal
#align cardinal.add_le_add_iff_of_lt_aleph_0 Cardinal.add_le_add_iff_of_lt_aleph0

@[simp]
theorem add_nat_le_add_nat_iff_of_lt_aleph_0 {α β : Cardinal} (n : ℕ) : α + n ≤ β + n ↔ α ≤ β :=
theorem add_nat_le_add_nat_iff {α β : Cardinal} (n : ℕ) : α + n ≤ β + n ↔ α ≤ β :=
add_le_add_iff_of_lt_aleph0 (nat_lt_aleph0 n)
#align cardinal.add_nat_le_add_nat_iff_of_lt_aleph_0 Cardinal.add_nat_le_add_nat_iff_of_lt_aleph_0
#align cardinal.add_nat_le_add_nat_iff_of_lt_aleph_0 Cardinal.add_nat_le_add_nat_iff

@[deprecated]
alias add_nat_le_add_nat_iff_of_lt_aleph_0 := add_nat_le_add_nat_iff -- deprecated on 2024-02-12

@[simp]
theorem add_one_le_add_one_iff_of_lt_aleph_0 {α β : Cardinal} : α + 1 ≤ β + 1 ↔ α ≤ β :=
theorem add_one_le_add_one_iff {α β : Cardinal} : α + 1 ≤ β + 1 ↔ α ≤ β :=
add_le_add_iff_of_lt_aleph0 one_lt_aleph0
#align cardinal.add_one_le_add_one_iff_of_lt_aleph_0 Cardinal.add_one_le_add_one_iff_of_lt_aleph_0
#align cardinal.add_one_le_add_one_iff_of_lt_aleph_0 Cardinal.add_one_le_add_one_iff

@[deprecated]
alias add_one_le_add_one_iff_of_lt_aleph_0 := add_one_le_add_one_iff -- deprecated on 2024-02-12

/-! ### Properties about power -/

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/SetTheory/Ordinal/Basic.lean
Expand Up @@ -38,7 +38,7 @@ initial segment (or, equivalently, in any way). This total order is well founded
* `o₁ + o₂` is the order on the disjoint union of `o₁` and `o₂` obtained by declaring that
every element of `o₁` is smaller than every element of `o₂`. The main properties of addition
(and the other operations on ordinals) are stated and proved in `OrdinalArithmetic.lean`. Here,
(and the other operations on ordinals) are stated and proved in `Ordinal/Arithmetic.lean`. Here,
we only introduce it and prove its basic properties to deduce the fact that the order on ordinals
is total (and well founded).
* `succ o` is the successor of the ordinal `o`.
Expand Down

0 comments on commit a6f1457

Please sign in to comment.