| Metamath
Proof Explorer Theorem List (p. 86 of 494) | < Previous Next > | |
| Bad symbols? Try the
GIF version. |
||
|
Mirrors > Metamath Home Page > MPE Home Page > Theorem List Contents > Recent Proofs This page: Page List |
||
| Color key: | (1-30937) |
(30938-32460) |
(32461-49324) |
| Type | Label | Description |
|---|---|---|
| Statement | ||
| Syntax | c3o 8501 | Extend the definition of a class to include the ordinal number 3. |
| class 3o | ||
| Syntax | c4o 8502 | Extend the definition of a class to include the ordinal number 4. |
| class 4o | ||
| Syntax | coa 8503 | Extend the definition of a class to include the ordinal addition operation. |
| class +o | ||
| Syntax | comu 8504 | Extend the definition of a class to include the ordinal multiplication operation. |
| class ·o | ||
| Syntax | coe 8505 | Extend the definition of a class to include the ordinal exponentiation operation. |
| class ↑o | ||
| Definition | df-1o 8506 | Define the ordinal number 1. Definition 2.1 of [Schloeder] p. 4. (Contributed by NM, 29-Oct-1995.) |
| ⊢ 1o = suc ∅ | ||
| Definition | df-2o 8507 | Define the ordinal number 2. Lemma 3.17 of [Schloeder] p. 10. (Contributed by NM, 18-Feb-2004.) |
| ⊢ 2o = suc 1o | ||
| Definition | df-3o 8508 | Define the ordinal number 3. (Contributed by Mario Carneiro, 14-Jul-2013.) |
| ⊢ 3o = suc 2o | ||
| Definition | df-4o 8509 | Define the ordinal number 4. (Contributed by Mario Carneiro, 14-Jul-2013.) |
| ⊢ 4o = suc 3o | ||
| Definition | df-oadd 8510* | Define the ordinal addition operation. (Contributed by NM, 3-May-1995.) |
| ⊢ +o = (𝑥 ∈ On, 𝑦 ∈ On ↦ (rec((𝑧 ∈ V ↦ suc 𝑧), 𝑥)‘𝑦)) | ||
| Definition | df-omul 8511* | Define the ordinal multiplication operation. (Contributed by NM, 26-Aug-1995.) |
| ⊢ ·o = (𝑥 ∈ On, 𝑦 ∈ On ↦ (rec((𝑧 ∈ V ↦ (𝑧 +o 𝑥)), ∅)‘𝑦)) | ||
| Definition | df-oexp 8512* | Define the ordinal exponentiation operation. (Contributed by NM, 30-Dec-2004.) |
| ⊢ ↑o = (𝑥 ∈ On, 𝑦 ∈ On ↦ if(𝑥 = ∅, (1o ∖ 𝑦), (rec((𝑧 ∈ V ↦ (𝑧 ·o 𝑥)), 1o)‘𝑦))) | ||
| Theorem | df1o2 8513 | Expanded value of the ordinal number 1. Definition 2.1 of [Schloeder] p. 4. (Contributed by NM, 4-Nov-2002.) |
| ⊢ 1o = {∅} | ||
| Theorem | df2o3 8514 | Expanded value of the ordinal number 2. (Contributed by Mario Carneiro, 14-Aug-2015.) |
| ⊢ 2o = {∅, 1o} | ||
| Theorem | df2o2 8515 | Expanded value of the ordinal number 2. (Contributed by NM, 29-Jan-2004.) |
| ⊢ 2o = {∅, {∅}} | ||
| Theorem | 1oex 8516 | Ordinal 1 is a set. (Contributed by BJ, 6-Apr-2019.) (Proof shortened by AV, 1-Jul-2022.) Remove dependency on ax-10 2141, ax-11 2157, ax-12 2177, ax-un 7755. (Revised by Zhi Wang, 19-Sep-2024.) |
| ⊢ 1o ∈ V | ||
| Theorem | 2oex 8517 | 2o is a set. (Contributed by BJ, 6-Apr-2019.) Remove dependency on ax-10 2141, ax-11 2157, ax-12 2177, ax-un 7755. (Proof shortened by Zhi Wang, 19-Sep-2024.) |
| ⊢ 2o ∈ V | ||
| Theorem | 1on 8518 | Ordinal 1 is an ordinal number. (Contributed by NM, 29-Oct-1995.) Avoid ax-un 7755. (Revised by BTernaryTau, 30-Nov-2024.) |
| ⊢ 1o ∈ On | ||
| Theorem | 1onOLD 8519 | Obsolete version of 1on 8518 as of 30-Nov-2024. (Contributed by NM, 29-Oct-1995.) (Proof modification is discouraged.) (New usage is discouraged.) |
| ⊢ 1o ∈ On | ||
| Theorem | 2on 8520 | Ordinal 2 is an ordinal number. (Contributed by NM, 18-Feb-2004.) (Proof shortened by Andrew Salmon, 12-Aug-2011.) Avoid ax-un 7755. (Revised by BTernaryTau, 30-Nov-2024.) |
| ⊢ 2o ∈ On | ||
| Theorem | 2onOLD 8521 | Obsolete version of 2on 8520 as of 30-Nov-2024. (Contributed by NM, 18-Feb-2004.) (Proof shortened by Andrew Salmon, 12-Aug-2011.) (Proof modification is discouraged.) (New usage is discouraged.) |
| ⊢ 2o ∈ On | ||
| Theorem | 2on0 8522 | Ordinal two is not zero. (Contributed by Scott Fenton, 17-Jun-2011.) |
| ⊢ 2o ≠ ∅ | ||
| Theorem | ord3 8523 | Ordinal 3 is an ordinal class. (Contributed by BTernaryTau, 6-Jan-2025.) |
| ⊢ Ord 3o | ||
| Theorem | 3on 8524 | Ordinal 3 is an ordinal number. (Contributed by Mario Carneiro, 5-Jan-2016.) |
| ⊢ 3o ∈ On | ||
| Theorem | 4on 8525 | Ordinal 4 is an ordinal number. (Contributed by Mario Carneiro, 5-Jan-2016.) |
| ⊢ 4o ∈ On | ||
| Theorem | 1n0 8526 | Ordinal one is not equal to ordinal zero. (Contributed by NM, 26-Dec-2004.) |
| ⊢ 1o ≠ ∅ | ||
| Theorem | nlim1 8527 | 1 is not a limit ordinal. (Contributed by BTernaryTau, 1-Dec-2024.) |
| ⊢ ¬ Lim 1o | ||
| Theorem | nlim2 8528 | 2 is not a limit ordinal. (Contributed by BTernaryTau, 1-Dec-2024.) |
| ⊢ ¬ Lim 2o | ||
| Theorem | xp01disj 8529 | Cartesian products with the singletons of ordinals 0 and 1 are disjoint. (Contributed by NM, 2-Jun-2007.) |
| ⊢ ((𝐴 × {∅}) ∩ (𝐶 × {1o})) = ∅ | ||
| Theorem | xp01disjl 8530 | Cartesian products with the singletons of ordinals 0 and 1 are disjoint. (Contributed by Jim Kingdon, 11-Jul-2023.) |
| ⊢ (({∅} × 𝐴) ∩ ({1o} × 𝐶)) = ∅ | ||
| Theorem | ordgt0ge1 8531 | Two ways to express that an ordinal class is positive. (Contributed by NM, 21-Dec-2004.) |
| ⊢ (Ord 𝐴 → (∅ ∈ 𝐴 ↔ 1o ⊆ 𝐴)) | ||
| Theorem | ordge1n0 8532 | An ordinal greater than or equal to 1 is nonzero. (Contributed by NM, 21-Dec-2004.) |
| ⊢ (Ord 𝐴 → (1o ⊆ 𝐴 ↔ 𝐴 ≠ ∅)) | ||
| Theorem | el1o 8533 | Membership in ordinal one. (Contributed by NM, 5-Jan-2005.) |
| ⊢ (𝐴 ∈ 1o ↔ 𝐴 = ∅) | ||
| Theorem | ord1eln01 8534 | An ordinal that is not 0 or 1 contains 1. (Contributed by BTernaryTau, 1-Dec-2024.) |
| ⊢ (Ord 𝐴 → (1o ∈ 𝐴 ↔ (𝐴 ≠ ∅ ∧ 𝐴 ≠ 1o))) | ||
| Theorem | ord2eln012 8535 | An ordinal that is not 0, 1, or 2 contains 2. (Contributed by BTernaryTau, 1-Dec-2024.) |
| ⊢ (Ord 𝐴 → (2o ∈ 𝐴 ↔ (𝐴 ≠ ∅ ∧ 𝐴 ≠ 1o ∧ 𝐴 ≠ 2o))) | ||
| Theorem | 1ellim 8536 | A limit ordinal contains 1. (Contributed by BTernaryTau, 1-Dec-2024.) |
| ⊢ (Lim 𝐴 → 1o ∈ 𝐴) | ||
| Theorem | 2ellim 8537 | A limit ordinal contains 2. (Contributed by BTernaryTau, 1-Dec-2024.) |
| ⊢ (Lim 𝐴 → 2o ∈ 𝐴) | ||
| Theorem | dif1o 8538 | Two ways to say that 𝐴 is a nonzero number of the set 𝐵. (Contributed by Mario Carneiro, 21-May-2015.) |
| ⊢ (𝐴 ∈ (𝐵 ∖ 1o) ↔ (𝐴 ∈ 𝐵 ∧ 𝐴 ≠ ∅)) | ||
| Theorem | ondif1 8539 | Two ways to say that 𝐴 is a nonzero ordinal number. Lemma 1.10 of [Schloeder] p. 2. (Contributed by Mario Carneiro, 21-May-2015.) |
| ⊢ (𝐴 ∈ (On ∖ 1o) ↔ (𝐴 ∈ On ∧ ∅ ∈ 𝐴)) | ||
| Theorem | ondif2 8540 | Two ways to say that 𝐴 is an ordinal greater than one. (Contributed by Mario Carneiro, 21-May-2015.) |
| ⊢ (𝐴 ∈ (On ∖ 2o) ↔ (𝐴 ∈ On ∧ 1o ∈ 𝐴)) | ||
| Theorem | 2oconcl 8541 | Closure of the pair swapping function on 2o. (Contributed by Mario Carneiro, 27-Sep-2015.) |
| ⊢ (𝐴 ∈ 2o → (1o ∖ 𝐴) ∈ 2o) | ||
| Theorem | 0lt1o 8542 | Ordinal zero is less than ordinal one. (Contributed by NM, 5-Jan-2005.) |
| ⊢ ∅ ∈ 1o | ||
| Theorem | dif20el 8543 | An ordinal greater than one is greater than zero. (Contributed by Mario Carneiro, 25-May-2015.) |
| ⊢ (𝐴 ∈ (On ∖ 2o) → ∅ ∈ 𝐴) | ||
| Theorem | 0we1 8544 | The empty set is a well-ordering of ordinal one. (Contributed by Mario Carneiro, 9-Feb-2015.) |
| ⊢ ∅ We 1o | ||
| Theorem | brwitnlem 8545 | Lemma for relations which assert the existence of a witness in a two-parameter set. (Contributed by Stefan O'Rear, 25-Jan-2015.) (Revised by Mario Carneiro, 23-Aug-2015.) |
| ⊢ 𝑅 = (◡𝑂 “ (V ∖ 1o)) & ⊢ 𝑂 Fn 𝑋 ⇒ ⊢ (𝐴𝑅𝐵 ↔ (𝐴𝑂𝐵) ≠ ∅) | ||
| Theorem | fnoa 8546 | Functionality and domain of ordinal addition. (Contributed by NM, 26-Aug-1995.) (Revised by Mario Carneiro, 8-Sep-2013.) |
| ⊢ +o Fn (On × On) | ||
| Theorem | fnom 8547 | Functionality and domain of ordinal multiplication. (Contributed by NM, 26-Aug-1995.) (Revised by Mario Carneiro, 8-Sep-2013.) |
| ⊢ ·o Fn (On × On) | ||
| Theorem | fnoe 8548 | Functionality and domain of ordinal exponentiation. (Contributed by Mario Carneiro, 29-May-2015.) |
| ⊢ ↑o Fn (On × On) | ||
| Theorem | oav 8549* | Value of ordinal addition. (Contributed by NM, 3-May-1995.) (Revised by Mario Carneiro, 8-Sep-2013.) |
| ⊢ ((𝐴 ∈ On ∧ 𝐵 ∈ On) → (𝐴 +o 𝐵) = (rec((𝑥 ∈ V ↦ suc 𝑥), 𝐴)‘𝐵)) | ||
| Theorem | omv 8550* | Value of ordinal multiplication. (Contributed by NM, 17-Sep-1995.) (Revised by Mario Carneiro, 23-Aug-2014.) |
| ⊢ ((𝐴 ∈ On ∧ 𝐵 ∈ On) → (𝐴 ·o 𝐵) = (rec((𝑥 ∈ V ↦ (𝑥 +o 𝐴)), ∅)‘𝐵)) | ||
| Theorem | oe0lem 8551 | A helper lemma for oe0 8560 and others. (Contributed by NM, 6-Jan-2005.) |
| ⊢ ((𝜑 ∧ 𝐴 = ∅) → 𝜓) & ⊢ (((𝐴 ∈ On ∧ 𝜑) ∧ ∅ ∈ 𝐴) → 𝜓) ⇒ ⊢ ((𝐴 ∈ On ∧ 𝜑) → 𝜓) | ||
| Theorem | oev 8552* | Value of ordinal exponentiation. (Contributed by NM, 30-Dec-2004.) (Revised by Mario Carneiro, 23-Aug-2014.) |
| ⊢ ((𝐴 ∈ On ∧ 𝐵 ∈ On) → (𝐴 ↑o 𝐵) = if(𝐴 = ∅, (1o ∖ 𝐵), (rec((𝑥 ∈ V ↦ (𝑥 ·o 𝐴)), 1o)‘𝐵))) | ||
| Theorem | oevn0 8553* | Value of ordinal exponentiation at a nonzero base. (Contributed by NM, 31-Dec-2004.) (Revised by Mario Carneiro, 8-Sep-2013.) |
| ⊢ (((𝐴 ∈ On ∧ 𝐵 ∈ On) ∧ ∅ ∈ 𝐴) → (𝐴 ↑o 𝐵) = (rec((𝑥 ∈ V ↦ (𝑥 ·o 𝐴)), 1o)‘𝐵)) | ||
| Theorem | oa0 8554 | Addition with zero. Proposition 8.3 of [TakeutiZaring] p. 57. Definition 2.3 of [Schloeder] p. 4. (Contributed by NM, 3-May-1995.) (Revised by Mario Carneiro, 8-Sep-2013.) |
| ⊢ (𝐴 ∈ On → (𝐴 +o ∅) = 𝐴) | ||
| Theorem | om0 8555 | Ordinal multiplication with zero. Definition 8.15(a) of [TakeutiZaring] p. 62. Definition 2.5 of [Schloeder] p. 4. See om0x 8557 for a way to remove the antecedent 𝐴 ∈ On. (Contributed by NM, 17-Sep-1995.) (Revised by Mario Carneiro, 8-Sep-2013.) |
| ⊢ (𝐴 ∈ On → (𝐴 ·o ∅) = ∅) | ||
| Theorem | oe0m 8556 | Value of zero raised to an ordinal. (Contributed by NM, 31-Dec-2004.) (Revised by Mario Carneiro, 8-Sep-2013.) |
| ⊢ (𝐴 ∈ On → (∅ ↑o 𝐴) = (1o ∖ 𝐴)) | ||
| Theorem | om0x 8557 | Ordinal multiplication with zero. Definition 8.15 of [TakeutiZaring] p. 62. Unlike om0 8555, this version works whether or not 𝐴 is an ordinal. However, since it is an artifact of our particular function value definition outside the domain, we will not use it in order to be conventional and present it only as a curiosity. (Contributed by NM, 1-Feb-1996.) (New usage is discouraged.) |
| ⊢ (𝐴 ·o ∅) = ∅ | ||
| Theorem | oe0m0 8558 | Ordinal exponentiation with zero base and zero exponent. Proposition 8.31 of [TakeutiZaring] p. 67. (Contributed by NM, 31-Dec-2004.) |
| ⊢ (∅ ↑o ∅) = 1o | ||
| Theorem | oe0m1 8559 | Ordinal exponentiation with zero base and nonzero exponent. Proposition 8.31(2) of [TakeutiZaring] p. 67 and its converse. Definition 2.6 of [Schloeder] p. 4. (Contributed by NM, 5-Jan-2005.) |
| ⊢ (𝐴 ∈ On → (∅ ∈ 𝐴 ↔ (∅ ↑o 𝐴) = ∅)) | ||
| Theorem | oe0 8560 | Ordinal exponentiation with zero exponent. Definition 8.30 of [TakeutiZaring] p. 67. Definition 2.6 of [Schloeder] p. 4. (Contributed by NM, 31-Dec-2004.) (Revised by Mario Carneiro, 8-Sep-2013.) |
| ⊢ (𝐴 ∈ On → (𝐴 ↑o ∅) = 1o) | ||
| Theorem | oev2 8561* | Alternate value of ordinal exponentiation. Compare oev 8552. (Contributed by NM, 2-Jan-2004.) (Revised by Mario Carneiro, 8-Sep-2013.) |
| ⊢ ((𝐴 ∈ On ∧ 𝐵 ∈ On) → (𝐴 ↑o 𝐵) = ((rec((𝑥 ∈ V ↦ (𝑥 ·o 𝐴)), 1o)‘𝐵) ∩ ((V ∖ ∩ 𝐴) ∪ ∩ 𝐵))) | ||
| Theorem | oasuc 8562 | Addition with successor. Definition 8.1 of [TakeutiZaring] p. 56. Definition 2.3 of [Schloeder] p. 4. (Contributed by NM, 3-May-1995.) (Revised by Mario Carneiro, 8-Sep-2013.) |
| ⊢ ((𝐴 ∈ On ∧ 𝐵 ∈ On) → (𝐴 +o suc 𝐵) = suc (𝐴 +o 𝐵)) | ||
| Theorem | oesuclem 8563* | Lemma for oesuc 8565. (Contributed by NM, 31-Dec-2004.) (Revised by Mario Carneiro, 15-Nov-2014.) |
| ⊢ Lim 𝑋 & ⊢ (𝐵 ∈ 𝑋 → (rec((𝑥 ∈ V ↦ (𝑥 ·o 𝐴)), 1o)‘suc 𝐵) = ((𝑥 ∈ V ↦ (𝑥 ·o 𝐴))‘(rec((𝑥 ∈ V ↦ (𝑥 ·o 𝐴)), 1o)‘𝐵))) ⇒ ⊢ ((𝐴 ∈ On ∧ 𝐵 ∈ 𝑋) → (𝐴 ↑o suc 𝐵) = ((𝐴 ↑o 𝐵) ·o 𝐴)) | ||
| Theorem | omsuc 8564 | Multiplication with successor. Definition 8.15 of [TakeutiZaring] p. 62. Definition 2.5 of [Schloeder] p. 4. (Contributed by NM, 17-Sep-1995.) (Revised by Mario Carneiro, 8-Sep-2013.) |
| ⊢ ((𝐴 ∈ On ∧ 𝐵 ∈ On) → (𝐴 ·o suc 𝐵) = ((𝐴 ·o 𝐵) +o 𝐴)) | ||
| Theorem | oesuc 8565 | Ordinal exponentiation with a successor exponent. Definition 8.30 of [TakeutiZaring] p. 67. Definition 2.6 of [Schloeder] p. 4. (Contributed by NM, 31-Dec-2004.) (Revised by Mario Carneiro, 8-Sep-2013.) |
| ⊢ ((𝐴 ∈ On ∧ 𝐵 ∈ On) → (𝐴 ↑o suc 𝐵) = ((𝐴 ↑o 𝐵) ·o 𝐴)) | ||
| Theorem | onasuc 8566 | Addition with successor. Theorem 4I(A2) of [Enderton] p. 79. (Note that this version of oasuc 8562 does not need Replacement.) (Contributed by Mario Carneiro, 16-Nov-2014.) |
| ⊢ ((𝐴 ∈ On ∧ 𝐵 ∈ ω) → (𝐴 +o suc 𝐵) = suc (𝐴 +o 𝐵)) | ||
| Theorem | onmsuc 8567 | Multiplication with successor. Theorem 4J(A2) of [Enderton] p. 80. (Contributed by NM, 20-Sep-1995.) (Revised by Mario Carneiro, 14-Nov-2014.) |
| ⊢ ((𝐴 ∈ On ∧ 𝐵 ∈ ω) → (𝐴 ·o suc 𝐵) = ((𝐴 ·o 𝐵) +o 𝐴)) | ||
| Theorem | onesuc 8568 | Exponentiation with a successor exponent. Definition 8.30 of [TakeutiZaring] p. 67. (Contributed by Mario Carneiro, 14-Nov-2014.) |
| ⊢ ((𝐴 ∈ On ∧ 𝐵 ∈ ω) → (𝐴 ↑o suc 𝐵) = ((𝐴 ↑o 𝐵) ·o 𝐴)) | ||
| Theorem | oa1suc 8569 | Addition with 1 is same as successor. Proposition 4.34(a) of [Mendelson] p. 266. Remark 2.4 of [Schloeder] p. 4. (Contributed by NM, 29-Oct-1995.) (Revised by Mario Carneiro, 16-Nov-2014.) |
| ⊢ (𝐴 ∈ On → (𝐴 +o 1o) = suc 𝐴) | ||
| Theorem | oalim 8570* | Ordinal addition with a limit ordinal. Definition 8.1 of [TakeutiZaring] p. 56. Definition 2.3 of [Schloeder] p. 4. (Contributed by NM, 3-Aug-2004.) (Revised by Mario Carneiro, 8-Sep-2013.) |
| ⊢ ((𝐴 ∈ On ∧ (𝐵 ∈ 𝐶 ∧ Lim 𝐵)) → (𝐴 +o 𝐵) = ∪ 𝑥 ∈ 𝐵 (𝐴 +o 𝑥)) | ||
| Theorem | omlim 8571* | Ordinal multiplication with a limit ordinal. Definition 8.15 of [TakeutiZaring] p. 62. Definition 2.5 of [Schloeder] p. 4. (Contributed by NM, 3-Aug-2004.) (Revised by Mario Carneiro, 8-Sep-2013.) |
| ⊢ ((𝐴 ∈ On ∧ (𝐵 ∈ 𝐶 ∧ Lim 𝐵)) → (𝐴 ·o 𝐵) = ∪ 𝑥 ∈ 𝐵 (𝐴 ·o 𝑥)) | ||
| Theorem | oelim 8572* | Ordinal exponentiation with a limit exponent and nonzero base. Definition 8.30 of [TakeutiZaring] p. 67. Definition 2.6 of [Schloeder] p. 4. (Contributed by NM, 1-Jan-2005.) (Revised by Mario Carneiro, 8-Sep-2013.) |
| ⊢ (((𝐴 ∈ On ∧ (𝐵 ∈ 𝐶 ∧ Lim 𝐵)) ∧ ∅ ∈ 𝐴) → (𝐴 ↑o 𝐵) = ∪ 𝑥 ∈ 𝐵 (𝐴 ↑o 𝑥)) | ||
| Theorem | oacl 8573 | Closure law for ordinal addition. Proposition 8.2 of [TakeutiZaring] p. 57. Remark 2.8 of [Schloeder] p. 5. (Contributed by NM, 5-May-1995.) |
| ⊢ ((𝐴 ∈ On ∧ 𝐵 ∈ On) → (𝐴 +o 𝐵) ∈ On) | ||
| Theorem | omcl 8574 | Closure law for ordinal multiplication. Proposition 8.16 of [TakeutiZaring] p. 57. Remark 2.8 of [Schloeder] p. 5. (Contributed by NM, 3-Aug-2004.) (Proof shortened by Andrew Salmon, 22-Oct-2011.) |
| ⊢ ((𝐴 ∈ On ∧ 𝐵 ∈ On) → (𝐴 ·o 𝐵) ∈ On) | ||
| Theorem | oecl 8575 | Closure law for ordinal exponentiation. Remark 2.8 of [Schloeder] p. 5. (Contributed by NM, 1-Jan-2005.) (Proof shortened by Andrew Salmon, 22-Oct-2011.) |
| ⊢ ((𝐴 ∈ On ∧ 𝐵 ∈ On) → (𝐴 ↑o 𝐵) ∈ On) | ||
| Theorem | oa0r 8576 | Ordinal addition with zero. Proposition 8.3 of [TakeutiZaring] p. 57. Lemma 2.14 of [Schloeder] p. 5. (Contributed by NM, 5-May-1995.) |
| ⊢ (𝐴 ∈ On → (∅ +o 𝐴) = 𝐴) | ||
| Theorem | om0r 8577 | Ordinal multiplication with zero. Proposition 8.18(1) of [TakeutiZaring] p. 63. (Contributed by NM, 3-Aug-2004.) |
| ⊢ (𝐴 ∈ On → (∅ ·o 𝐴) = ∅) | ||
| Theorem | o1p1e2 8578 | 1 + 1 = 2 for ordinal numbers. (Contributed by NM, 18-Feb-2004.) |
| ⊢ (1o +o 1o) = 2o | ||
| Theorem | o2p2e4 8579 | 2 + 2 = 4 for ordinal numbers. Ordinal numbers are modeled as Von Neumann ordinals; see df-suc 6390. For the usual proof using complex numbers, see 2p2e4 12401. (Contributed by NM, 18-Aug-2021.) Avoid ax-rep 5279, from a comment by Sophie. (Revised by SN, 23-Mar-2024.) |
| ⊢ (2o +o 2o) = 4o | ||
| Theorem | om1 8580 | Ordinal multiplication with 1. Proposition 8.18(2) of [TakeutiZaring] p. 63. Lemma 2.15 of [Schloeder] p. 5. (Contributed by NM, 29-Oct-1995.) |
| ⊢ (𝐴 ∈ On → (𝐴 ·o 1o) = 𝐴) | ||
| Theorem | om1r 8581 | Ordinal multiplication with 1. Proposition 8.18(2) of [TakeutiZaring] p. 63. Lemma 2.15 of [Schloeder] p. 5. (Contributed by NM, 3-Aug-2004.) |
| ⊢ (𝐴 ∈ On → (1o ·o 𝐴) = 𝐴) | ||
| Theorem | oe1 8582 | Ordinal exponentiation with an exponent of 1. Lemma 2.16 of [Schloeder] p. 6. (Contributed by NM, 2-Jan-2005.) |
| ⊢ (𝐴 ∈ On → (𝐴 ↑o 1o) = 𝐴) | ||
| Theorem | oe1m 8583 | Ordinal exponentiation with a base of 1. Proposition 8.31(3) of [TakeutiZaring] p. 67. Lemma 2.17 of [Schloeder] p. 6. (Contributed by NM, 2-Jan-2005.) |
| ⊢ (𝐴 ∈ On → (1o ↑o 𝐴) = 1o) | ||
| Theorem | oaordi 8584 | Ordering property of ordinal addition. Proposition 8.4 of [TakeutiZaring] p. 58. (Contributed by NM, 5-Dec-2004.) |
| ⊢ ((𝐵 ∈ On ∧ 𝐶 ∈ On) → (𝐴 ∈ 𝐵 → (𝐶 +o 𝐴) ∈ (𝐶 +o 𝐵))) | ||
| Theorem | oaord 8585 | Ordering property of ordinal addition. Proposition 8.4 of [TakeutiZaring] p. 58 and its converse. (Contributed by NM, 5-Dec-2004.) |
| ⊢ ((𝐴 ∈ On ∧ 𝐵 ∈ On ∧ 𝐶 ∈ On) → (𝐴 ∈ 𝐵 ↔ (𝐶 +o 𝐴) ∈ (𝐶 +o 𝐵))) | ||
| Theorem | oacan 8586 | Left cancellation law for ordinal addition. Corollary 8.5 of [TakeutiZaring] p. 58. (Contributed by NM, 5-Dec-2004.) |
| ⊢ ((𝐴 ∈ On ∧ 𝐵 ∈ On ∧ 𝐶 ∈ On) → ((𝐴 +o 𝐵) = (𝐴 +o 𝐶) ↔ 𝐵 = 𝐶)) | ||
| Theorem | oaword 8587 | Weak ordering property of ordinal addition. (Contributed by NM, 6-Dec-2004.) (Proof shortened by Andrew Salmon, 22-Oct-2011.) |
| ⊢ ((𝐴 ∈ On ∧ 𝐵 ∈ On ∧ 𝐶 ∈ On) → (𝐴 ⊆ 𝐵 ↔ (𝐶 +o 𝐴) ⊆ (𝐶 +o 𝐵))) | ||
| Theorem | oawordri 8588 | Weak ordering property of ordinal addition. Proposition 8.7 of [TakeutiZaring] p. 59. (Contributed by NM, 7-Dec-2004.) |
| ⊢ ((𝐴 ∈ On ∧ 𝐵 ∈ On ∧ 𝐶 ∈ On) → (𝐴 ⊆ 𝐵 → (𝐴 +o 𝐶) ⊆ (𝐵 +o 𝐶))) | ||
| Theorem | oaord1 8589 | An ordinal is less than its sum with a nonzero ordinal. Theorem 18 of [Suppes] p. 209 and its converse. (Contributed by NM, 6-Dec-2004.) |
| ⊢ ((𝐴 ∈ On ∧ 𝐵 ∈ On) → (∅ ∈ 𝐵 ↔ 𝐴 ∈ (𝐴 +o 𝐵))) | ||
| Theorem | oaword1 8590 | An ordinal is less than or equal to its sum with another. Part of Exercise 5 of [TakeutiZaring] p. 62. Lemma 3.2 of [Schloeder] p. 7. (For the other part see oaord1 8589.) (Contributed by NM, 6-Dec-2004.) |
| ⊢ ((𝐴 ∈ On ∧ 𝐵 ∈ On) → 𝐴 ⊆ (𝐴 +o 𝐵)) | ||
| Theorem | oaword2 8591 | An ordinal is less than or equal to its sum with another. Theorem 21 of [Suppes] p. 209. Lemma 3.3 of [Schloeder] p. 7. (Contributed by NM, 7-Dec-2004.) |
| ⊢ ((𝐴 ∈ On ∧ 𝐵 ∈ On) → 𝐴 ⊆ (𝐵 +o 𝐴)) | ||
| Theorem | oawordeulem 8592* | Lemma for oawordex 8595. (Contributed by NM, 11-Dec-2004.) |
| ⊢ 𝐴 ∈ On & ⊢ 𝐵 ∈ On & ⊢ 𝑆 = {𝑦 ∈ On ∣ 𝐵 ⊆ (𝐴 +o 𝑦)} ⇒ ⊢ (𝐴 ⊆ 𝐵 → ∃!𝑥 ∈ On (𝐴 +o 𝑥) = 𝐵) | ||
| Theorem | oawordeu 8593* | Existence theorem for weak ordering of ordinal sum. Proposition 8.8 of [TakeutiZaring] p. 59. (Contributed by NM, 11-Dec-2004.) |
| ⊢ (((𝐴 ∈ On ∧ 𝐵 ∈ On) ∧ 𝐴 ⊆ 𝐵) → ∃!𝑥 ∈ On (𝐴 +o 𝑥) = 𝐵) | ||
| Theorem | oawordexr 8594* | Existence theorem for weak ordering of ordinal sum. (Contributed by NM, 12-Dec-2004.) |
| ⊢ ((𝐴 ∈ On ∧ ∃𝑥 ∈ On (𝐴 +o 𝑥) = 𝐵) → 𝐴 ⊆ 𝐵) | ||
| Theorem | oawordex 8595* | Existence theorem for weak ordering of ordinal sum. Proposition 8.8 of [TakeutiZaring] p. 59 and its converse. See oawordeu 8593 for uniqueness. (Contributed by NM, 12-Dec-2004.) |
| ⊢ ((𝐴 ∈ On ∧ 𝐵 ∈ On) → (𝐴 ⊆ 𝐵 ↔ ∃𝑥 ∈ On (𝐴 +o 𝑥) = 𝐵)) | ||
| Theorem | oaordex 8596* | Existence theorem for ordering of ordinal sum. Similar to Proposition 4.34(f) of [Mendelson] p. 266 and its converse. (Contributed by NM, 12-Dec-2004.) |
| ⊢ ((𝐴 ∈ On ∧ 𝐵 ∈ On) → (𝐴 ∈ 𝐵 ↔ ∃𝑥 ∈ On (∅ ∈ 𝑥 ∧ (𝐴 +o 𝑥) = 𝐵))) | ||
| Theorem | oa00 8597 | An ordinal sum is zero iff both of its arguments are zero. Lemma 3.10 of [Schloeder] p. 8. (Contributed by NM, 6-Dec-2004.) |
| ⊢ ((𝐴 ∈ On ∧ 𝐵 ∈ On) → ((𝐴 +o 𝐵) = ∅ ↔ (𝐴 = ∅ ∧ 𝐵 = ∅))) | ||
| Theorem | oalimcl 8598 | The ordinal sum with a limit ordinal is a limit ordinal. Proposition 8.11 of [TakeutiZaring] p. 60. Lemma 3.4 of [Schloeder] p. 7. (Contributed by NM, 8-Dec-2004.) |
| ⊢ ((𝐴 ∈ On ∧ (𝐵 ∈ 𝐶 ∧ Lim 𝐵)) → Lim (𝐴 +o 𝐵)) | ||
| Theorem | oaass 8599 | Ordinal addition is associative. Theorem 25 of [Suppes] p. 211. Theorem 4.2 of [Schloeder] p. 11. (Contributed by NM, 10-Dec-2004.) |
| ⊢ ((𝐴 ∈ On ∧ 𝐵 ∈ On ∧ 𝐶 ∈ On) → ((𝐴 +o 𝐵) +o 𝐶) = (𝐴 +o (𝐵 +o 𝐶))) | ||
| Theorem | oarec 8600* | Recursive definition of ordinal addition. Exercise 25 of [Enderton] p. 240. (Contributed by NM, 26-Dec-2004.) (Revised by Mario Carneiro, 30-May-2015.) |
| ⊢ ((𝐴 ∈ On ∧ 𝐵 ∈ On) → (𝐴 +o 𝐵) = (𝐴 ∪ ran (𝑥 ∈ 𝐵 ↦ (𝐴 +o 𝑥)))) | ||
| < Previous Next > |
| Copyright terms: Public domain | < Previous Next > |