![]() |
Intuitionistic Logic Explorer Theorem List (p. 74 of 156) | < Previous Next > |
Bad symbols? Try the
GIF version. |
||
Mirrors > Metamath Home Page > ILE Home Page > Theorem List Contents > Recent Proofs This page: Page List |
Type | Label | Description |
---|---|---|
Statement | ||
Theorem | onntri45 7301* | Double negated ordinal trichotomy. (Contributed by James E. Hanson and Jim Kingdon, 2-Aug-2024.) |
⊢ (∀𝑥 ∈ On ∀𝑦 ∈ On ¬ ¬ (𝑥 ⊆ 𝑦 ∨ 𝑦 ⊆ 𝑥) → ¬ ¬ EXMID) | ||
Theorem | onntri24 7302 | Double negated ordinal trichotomy. (Contributed by James E. Hanson and Jim Kingdon, 2-Aug-2024.) |
⊢ (¬ ¬ ∀𝑥 ∈ On ∀𝑦 ∈ On (𝑥 ⊆ 𝑦 ∨ 𝑦 ⊆ 𝑥) → ∀𝑥 ∈ On ∀𝑦 ∈ On ¬ ¬ (𝑥 ⊆ 𝑦 ∨ 𝑦 ⊆ 𝑥)) | ||
Theorem | exmidontri2or 7303* | Ordinal trichotomy is equivalent to excluded middle. (Contributed by Jim Kingdon, 26-Aug-2024.) |
⊢ (EXMID ↔ ∀𝑥 ∈ On ∀𝑦 ∈ On (𝑥 ⊆ 𝑦 ∨ 𝑦 ⊆ 𝑥)) | ||
Theorem | onntri52 7304* | Double negated ordinal trichotomy. (Contributed by James E. Hanson and Jim Kingdon, 2-Aug-2024.) |
⊢ (¬ ¬ EXMID → ¬ ¬ ∀𝑥 ∈ On ∀𝑦 ∈ On (𝑥 ⊆ 𝑦 ∨ 𝑦 ⊆ 𝑥)) | ||
Theorem | onntri3or 7305* | Double negated ordinal trichotomy. (Contributed by Jim Kingdon, 25-Aug-2024.) |
⊢ (¬ ¬ EXMID ↔ ∀𝑥 ∈ On ∀𝑦 ∈ On ¬ ¬ (𝑥 ∈ 𝑦 ∨ 𝑥 = 𝑦 ∨ 𝑦 ∈ 𝑥)) | ||
Theorem | onntri2or 7306* | Double negated ordinal trichotomy. (Contributed by Jim Kingdon, 25-Aug-2024.) |
⊢ (¬ ¬ EXMID ↔ ∀𝑥 ∈ On ∀𝑦 ∈ On ¬ ¬ (𝑥 ⊆ 𝑦 ∨ 𝑦 ⊆ 𝑥)) | ||
Syntax | wap 7307 | Apartness predicate symbol. |
wff 𝑅 Ap 𝐴 | ||
Definition | df-pap 7308* | Apartness predicate. A relation 𝑅 is an apartness if it is irreflexive, symmetric, and cotransitive. (Contributed by Jim Kingdon, 14-Feb-2025.) |
⊢ (𝑅 Ap 𝐴 ↔ ((𝑅 ⊆ (𝐴 × 𝐴) ∧ ∀𝑥 ∈ 𝐴 ¬ 𝑥𝑅𝑥) ∧ (∀𝑥 ∈ 𝐴 ∀𝑦 ∈ 𝐴 (𝑥𝑅𝑦 → 𝑦𝑅𝑥) ∧ ∀𝑥 ∈ 𝐴 ∀𝑦 ∈ 𝐴 ∀𝑧 ∈ 𝐴 (𝑥𝑅𝑦 → (𝑥𝑅𝑧 ∨ 𝑦𝑅𝑧))))) | ||
Syntax | wtap 7309 | Tight apartness predicate symbol. |
wff 𝑅 TAp 𝐴 | ||
Definition | df-tap 7310* | Tight apartness predicate. A relation 𝑅 is a tight apartness if it is irreflexive, symmetric, cotransitive, and tight. (Contributed by Jim Kingdon, 5-Feb-2025.) |
⊢ (𝑅 TAp 𝐴 ↔ (𝑅 Ap 𝐴 ∧ ∀𝑥 ∈ 𝐴 ∀𝑦 ∈ 𝐴 (¬ 𝑥𝑅𝑦 → 𝑥 = 𝑦))) | ||
Theorem | dftap2 7311* | Tight apartness with the apartness properties from df-pap 7308 expanded. (Contributed by Jim Kingdon, 21-Feb-2025.) |
⊢ (𝑅 TAp 𝐴 ↔ (𝑅 ⊆ (𝐴 × 𝐴) ∧ (∀𝑥 ∈ 𝐴 ¬ 𝑥𝑅𝑥 ∧ ∀𝑥 ∈ 𝐴 ∀𝑦 ∈ 𝐴 (𝑥𝑅𝑦 → 𝑦𝑅𝑥)) ∧ (∀𝑥 ∈ 𝐴 ∀𝑦 ∈ 𝐴 ∀𝑧 ∈ 𝐴 (𝑥𝑅𝑦 → (𝑥𝑅𝑧 ∨ 𝑦𝑅𝑧)) ∧ ∀𝑥 ∈ 𝐴 ∀𝑦 ∈ 𝐴 (¬ 𝑥𝑅𝑦 → 𝑥 = 𝑦)))) | ||
Theorem | tapeq1 7312 | Equality theorem for tight apartness predicate. (Contributed by Jim Kingdon, 8-Feb-2025.) |
⊢ (𝑅 = 𝑆 → (𝑅 TAp 𝐴 ↔ 𝑆 TAp 𝐴)) | ||
Theorem | tapeq2 7313 | Equality theorem for tight apartness predicate. (Contributed by Jim Kingdon, 15-Feb-2025.) |
⊢ (𝐴 = 𝐵 → (𝑅 TAp 𝐴 ↔ 𝑅 TAp 𝐵)) | ||
Theorem | netap 7314* | Negated equality on a set with decidable equality is a tight apartness. (Contributed by Jim Kingdon, 5-Feb-2025.) |
⊢ (∀𝑥 ∈ 𝐴 ∀𝑦 ∈ 𝐴 DECID 𝑥 = 𝑦 → {〈𝑢, 𝑣〉 ∣ ((𝑢 ∈ 𝐴 ∧ 𝑣 ∈ 𝐴) ∧ 𝑢 ≠ 𝑣)} TAp 𝐴) | ||
Theorem | 2onetap 7315* | Negated equality is a tight apartness on 2o. (Contributed by Jim Kingdon, 6-Feb-2025.) |
⊢ {〈𝑢, 𝑣〉 ∣ ((𝑢 ∈ 2o ∧ 𝑣 ∈ 2o) ∧ 𝑢 ≠ 𝑣)} TAp 2o | ||
Theorem | 2oneel 7316* | ∅ and 1o are two unequal elements of 2o. (Contributed by Jim Kingdon, 8-Feb-2025.) |
⊢ 〈∅, 1o〉 ∈ {〈𝑢, 𝑣〉 ∣ ((𝑢 ∈ 2o ∧ 𝑣 ∈ 2o) ∧ 𝑢 ≠ 𝑣)} | ||
Theorem | 2omotaplemap 7317* | Lemma for 2omotap 7319. (Contributed by Jim Kingdon, 6-Feb-2025.) |
⊢ (¬ ¬ 𝜑 → {〈𝑢, 𝑣〉 ∣ ((𝑢 ∈ 2o ∧ 𝑣 ∈ 2o) ∧ (𝜑 ∧ 𝑢 ≠ 𝑣))} TAp 2o) | ||
Theorem | 2omotaplemst 7318* | Lemma for 2omotap 7319. (Contributed by Jim Kingdon, 6-Feb-2025.) |
⊢ ((∃*𝑟 𝑟 TAp 2o ∧ ¬ ¬ 𝜑) → 𝜑) | ||
Theorem | 2omotap 7319 | If there is at most one tight apartness on 2o, excluded middle follows. Based on online discussions by Tom de Jong, Andrew W Swan, and Martin Escardo. (Contributed by Jim Kingdon, 6-Feb-2025.) |
⊢ (∃*𝑟 𝑟 TAp 2o → EXMID) | ||
Theorem | exmidapne 7320* | Excluded middle implies there is only one tight apartness on any class, namely negated equality. (Contributed by Jim Kingdon, 14-Feb-2025.) |
⊢ (EXMID → (𝑅 TAp 𝐴 ↔ 𝑅 = {〈𝑢, 𝑣〉 ∣ ((𝑢 ∈ 𝐴 ∧ 𝑣 ∈ 𝐴) ∧ 𝑢 ≠ 𝑣)})) | ||
Theorem | exmidmotap 7321* | The proposition that every class has at most one tight apartness is equivalent to excluded middle. (Contributed by Jim Kingdon, 14-Feb-2025.) |
⊢ (EXMID ↔ ∀𝑥∃*𝑟 𝑟 TAp 𝑥) | ||
We have already introduced the full Axiom of Choice df-ac 7266 but since it implies excluded middle as shown at exmidac 7269, it is not especially relevant to us. In this section we define countable choice and dependent choice, which are not as strong as thus often considered in mathematics which seeks to avoid full excluded middle. | ||
Syntax | wacc 7322 | Formula for an abbreviation of countable choice. |
wff CCHOICE | ||
Definition | df-cc 7323* | The expression CCHOICE will be used as a readable shorthand for any form of countable choice, analogous to df-ac 7266 for full choice. (Contributed by Jim Kingdon, 27-Nov-2023.) |
⊢ (CCHOICE ↔ ∀𝑥(dom 𝑥 ≈ ω → ∃𝑓(𝑓 ⊆ 𝑥 ∧ 𝑓 Fn dom 𝑥))) | ||
Theorem | ccfunen 7324* | Existence of a choice function for a countably infinite set. (Contributed by Jim Kingdon, 28-Nov-2023.) |
⊢ (𝜑 → CCHOICE) & ⊢ (𝜑 → 𝐴 ≈ ω) & ⊢ (𝜑 → ∀𝑥 ∈ 𝐴 ∃𝑤 𝑤 ∈ 𝑥) ⇒ ⊢ (𝜑 → ∃𝑓(𝑓 Fn 𝐴 ∧ ∀𝑥 ∈ 𝐴 (𝑓‘𝑥) ∈ 𝑥)) | ||
Theorem | cc1 7325* | Countable choice in terms of a choice function on a countably infinite set of inhabited sets. (Contributed by Jim Kingdon, 27-Apr-2024.) |
⊢ (CCHOICE → ∀𝑥((𝑥 ≈ ω ∧ ∀𝑧 ∈ 𝑥 ∃𝑤 𝑤 ∈ 𝑧) → ∃𝑓∀𝑧 ∈ 𝑥 (𝑓‘𝑧) ∈ 𝑧)) | ||
Theorem | cc2lem 7326* | Lemma for cc2 7327. (Contributed by Jim Kingdon, 27-Apr-2024.) |
⊢ (𝜑 → CCHOICE) & ⊢ (𝜑 → 𝐹 Fn ω) & ⊢ (𝜑 → ∀𝑥 ∈ ω ∃𝑤 𝑤 ∈ (𝐹‘𝑥)) & ⊢ 𝐴 = (𝑛 ∈ ω ↦ ({𝑛} × (𝐹‘𝑛))) & ⊢ 𝐺 = (𝑛 ∈ ω ↦ (2nd ‘(𝑓‘(𝐴‘𝑛)))) ⇒ ⊢ (𝜑 → ∃𝑔(𝑔 Fn ω ∧ ∀𝑛 ∈ ω (𝑔‘𝑛) ∈ (𝐹‘𝑛))) | ||
Theorem | cc2 7327* | Countable choice using sequences instead of countable sets. (Contributed by Jim Kingdon, 27-Apr-2024.) |
⊢ (𝜑 → CCHOICE) & ⊢ (𝜑 → 𝐹 Fn ω) & ⊢ (𝜑 → ∀𝑥 ∈ ω ∃𝑤 𝑤 ∈ (𝐹‘𝑥)) ⇒ ⊢ (𝜑 → ∃𝑔(𝑔 Fn ω ∧ ∀𝑛 ∈ ω (𝑔‘𝑛) ∈ (𝐹‘𝑛))) | ||
Theorem | cc3 7328* | Countable choice using a sequence F(n) . (Contributed by Mario Carneiro, 8-Feb-2013.) (Revised by Jim Kingdon, 29-Apr-2024.) |
⊢ (𝜑 → CCHOICE) & ⊢ (𝜑 → ∀𝑛 ∈ 𝑁 𝐹 ∈ V) & ⊢ (𝜑 → ∀𝑛 ∈ 𝑁 ∃𝑤 𝑤 ∈ 𝐹) & ⊢ (𝜑 → 𝑁 ≈ ω) ⇒ ⊢ (𝜑 → ∃𝑓(𝑓 Fn 𝑁 ∧ ∀𝑛 ∈ 𝑁 (𝑓‘𝑛) ∈ 𝐹)) | ||
Theorem | cc4f 7329* | Countable choice by showing the existence of a function 𝑓 which can choose a value at each index 𝑛 such that 𝜒 holds. (Contributed by Mario Carneiro, 7-Apr-2013.) (Revised by Jim Kingdon, 3-May-2024.) |
⊢ (𝜑 → CCHOICE) & ⊢ (𝜑 → 𝐴 ∈ 𝑉) & ⊢ Ⅎ𝑛𝐴 & ⊢ (𝜑 → 𝑁 ≈ ω) & ⊢ (𝑥 = (𝑓‘𝑛) → (𝜓 ↔ 𝜒)) & ⊢ (𝜑 → ∀𝑛 ∈ 𝑁 ∃𝑥 ∈ 𝐴 𝜓) ⇒ ⊢ (𝜑 → ∃𝑓(𝑓:𝑁⟶𝐴 ∧ ∀𝑛 ∈ 𝑁 𝜒)) | ||
Theorem | cc4 7330* | Countable choice by showing the existence of a function 𝑓 which can choose a value at each index 𝑛 such that 𝜒 holds. (Contributed by Mario Carneiro, 7-Apr-2013.) (Revised by Jim Kingdon, 1-May-2024.) |
⊢ (𝜑 → CCHOICE) & ⊢ (𝜑 → 𝐴 ∈ 𝑉) & ⊢ (𝜑 → 𝑁 ≈ ω) & ⊢ (𝑥 = (𝑓‘𝑛) → (𝜓 ↔ 𝜒)) & ⊢ (𝜑 → ∀𝑛 ∈ 𝑁 ∃𝑥 ∈ 𝐴 𝜓) ⇒ ⊢ (𝜑 → ∃𝑓(𝑓:𝑁⟶𝐴 ∧ ∀𝑛 ∈ 𝑁 𝜒)) | ||
Theorem | cc4n 7331* | Countable choice with a simpler restriction on how every set in the countable collection needs to be inhabited. That is, compared with cc4 7330, the hypotheses only require an A(n) for each value of 𝑛, not a single set 𝐴 which suffices for every 𝑛 ∈ ω. (Contributed by Mario Carneiro, 7-Apr-2013.) (Revised by Jim Kingdon, 3-May-2024.) |
⊢ (𝜑 → CCHOICE) & ⊢ (𝜑 → ∀𝑛 ∈ 𝑁 {𝑥 ∈ 𝐴 ∣ 𝜓} ∈ 𝑉) & ⊢ (𝜑 → 𝑁 ≈ ω) & ⊢ (𝑥 = (𝑓‘𝑛) → (𝜓 ↔ 𝜒)) & ⊢ (𝜑 → ∀𝑛 ∈ 𝑁 ∃𝑥 ∈ 𝐴 𝜓) ⇒ ⊢ (𝜑 → ∃𝑓(𝑓 Fn 𝑁 ∧ ∀𝑛 ∈ 𝑁 𝜒)) | ||
This section derives the basics of real and complex numbers. To construct the real numbers constructively, we follow two main sources. The first is Metamath Proof Explorer, which has the advantage of being already formalized in metamath. Its disadvantage, for our purposes, is that it assumes the law of the excluded middle throughout. Since we have already developed natural numbers ( for example, nna0 6527 and similar theorems ), going from there to positive integers (df-ni 7364) and then positive rational numbers (df-nqqs 7408) does not involve a major change in approach compared with the Metamath Proof Explorer. It is when we proceed to Dedekind cuts that we bring in more material from Section 11.2 of [HoTT], which focuses on the aspects of Dedekind cuts which are different without excluded middle or choice principles. With excluded middle, it is natural to define a cut as the lower set only (as Metamath Proof Explorer does), but here we define the cut as a pair of both the lower and upper sets, as [HoTT] does. There are also differences in how we handle order and replacing "not equal to zero" with "apart from zero". When working constructively, there are several possible definitions of real numbers. Here we adopt the most common definition, as two-sided Dedekind cuts with the properties described at df-inp 7526. The Cauchy reals (without countable choice) fail to satisfy ax-caucvg 7992 and the MacNeille reals fail to satisfy axltwlin 8087, and we do not develop them here. For more on differing definitions of the reals, see the introduction to Chapter 11 in [HoTT] or Section 1.2 of [BauerHanson]. | ||
Syntax | cnpi 7332 |
The set of positive integers, which is the set of natural numbers ω
with 0 removed.
Note: This is the start of the Dedekind-cut construction of real and complex numbers. |
class N | ||
Syntax | cpli 7333 | Positive integer addition. |
class +N | ||
Syntax | cmi 7334 | Positive integer multiplication. |
class ·N | ||
Syntax | clti 7335 | Positive integer ordering relation. |
class <N | ||
Syntax | cplpq 7336 | Positive pre-fraction addition. |
class +pQ | ||
Syntax | cmpq 7337 | Positive pre-fraction multiplication. |
class ·pQ | ||
Syntax | cltpq 7338 | Positive pre-fraction ordering relation. |
class <pQ | ||
Syntax | ceq 7339 | Equivalence class used to construct positive fractions. |
class ~Q | ||
Syntax | cnq 7340 | Set of positive fractions. |
class Q | ||
Syntax | c1q 7341 | The positive fraction constant 1. |
class 1Q | ||
Syntax | cplq 7342 | Positive fraction addition. |
class +Q | ||
Syntax | cmq 7343 | Positive fraction multiplication. |
class ·Q | ||
Syntax | crq 7344 | Positive fraction reciprocal operation. |
class *Q | ||
Syntax | cltq 7345 | Positive fraction ordering relation. |
class <Q | ||
Syntax | ceq0 7346 | Equivalence class used to construct nonnegative fractions. |
class ~Q0 | ||
Syntax | cnq0 7347 | Set of nonnegative fractions. |
class Q0 | ||
Syntax | c0q0 7348 | The nonnegative fraction constant 0. |
class 0Q0 | ||
Syntax | cplq0 7349 | Nonnegative fraction addition. |
class +Q0 | ||
Syntax | cmq0 7350 | Nonnegative fraction multiplication. |
class ·Q0 | ||
Syntax | cnp 7351 | Set of positive reals. |
class P | ||
Syntax | c1p 7352 | Positive real constant 1. |
class 1P | ||
Syntax | cpp 7353 | Positive real addition. |
class +P | ||
Syntax | cmp 7354 | Positive real multiplication. |
class ·P | ||
Syntax | cltp 7355 | Positive real ordering relation. |
class <P | ||
Syntax | cer 7356 | Equivalence class used to construct signed reals. |
class ~R | ||
Syntax | cnr 7357 | Set of signed reals. |
class R | ||
Syntax | c0r 7358 | The signed real constant 0. |
class 0R | ||
Syntax | c1r 7359 | The signed real constant 1. |
class 1R | ||
Syntax | cm1r 7360 | The signed real constant -1. |
class -1R | ||
Syntax | cplr 7361 | Signed real addition. |
class +R | ||
Syntax | cmr 7362 | Signed real multiplication. |
class ·R | ||
Syntax | cltr 7363 | Signed real ordering relation. |
class <R | ||
Definition | df-ni 7364 | Define the class of positive integers. This is a "temporary" set used in the construction of complex numbers, and is intended to be used only by the construction. (Contributed by NM, 15-Aug-1995.) |
⊢ N = (ω ∖ {∅}) | ||
Definition | df-pli 7365 | Define addition on positive integers. This is a "temporary" set used in the construction of complex numbers, and is intended to be used only by the construction. (Contributed by NM, 26-Aug-1995.) |
⊢ +N = ( +o ↾ (N × N)) | ||
Definition | df-mi 7366 | Define multiplication on positive integers. This is a "temporary" set used in the construction of complex numbers and is intended to be used only by the construction. (Contributed by NM, 26-Aug-1995.) |
⊢ ·N = ( ·o ↾ (N × N)) | ||
Definition | df-lti 7367 | Define 'less than' on positive integers. This is a "temporary" set used in the construction of complex numbers, and is intended to be used only by the construction. (Contributed by NM, 6-Feb-1996.) |
⊢ <N = ( E ∩ (N × N)) | ||
Theorem | elni 7368 | Membership in the class of positive integers. (Contributed by NM, 15-Aug-1995.) |
⊢ (𝐴 ∈ N ↔ (𝐴 ∈ ω ∧ 𝐴 ≠ ∅)) | ||
Theorem | pinn 7369 | A positive integer is a natural number. (Contributed by NM, 15-Aug-1995.) |
⊢ (𝐴 ∈ N → 𝐴 ∈ ω) | ||
Theorem | pion 7370 | A positive integer is an ordinal number. (Contributed by NM, 23-Mar-1996.) |
⊢ (𝐴 ∈ N → 𝐴 ∈ On) | ||
Theorem | piord 7371 | A positive integer is ordinal. (Contributed by NM, 29-Jan-1996.) |
⊢ (𝐴 ∈ N → Ord 𝐴) | ||
Theorem | niex 7372 | The class of positive integers is a set. (Contributed by NM, 15-Aug-1995.) |
⊢ N ∈ V | ||
Theorem | 0npi 7373 | The empty set is not a positive integer. (Contributed by NM, 26-Aug-1995.) |
⊢ ¬ ∅ ∈ N | ||
Theorem | elni2 7374 | Membership in the class of positive integers. (Contributed by NM, 27-Nov-1995.) |
⊢ (𝐴 ∈ N ↔ (𝐴 ∈ ω ∧ ∅ ∈ 𝐴)) | ||
Theorem | 1pi 7375 | Ordinal 'one' is a positive integer. (Contributed by NM, 29-Oct-1995.) |
⊢ 1o ∈ N | ||
Theorem | addpiord 7376 | Positive integer addition in terms of ordinal addition. (Contributed by NM, 27-Aug-1995.) |
⊢ ((𝐴 ∈ N ∧ 𝐵 ∈ N) → (𝐴 +N 𝐵) = (𝐴 +o 𝐵)) | ||
Theorem | mulpiord 7377 | Positive integer multiplication in terms of ordinal multiplication. (Contributed by NM, 27-Aug-1995.) |
⊢ ((𝐴 ∈ N ∧ 𝐵 ∈ N) → (𝐴 ·N 𝐵) = (𝐴 ·o 𝐵)) | ||
Theorem | mulidpi 7378 | 1 is an identity element for multiplication on positive integers. (Contributed by NM, 4-Mar-1996.) (Revised by Mario Carneiro, 17-Nov-2014.) |
⊢ (𝐴 ∈ N → (𝐴 ·N 1o) = 𝐴) | ||
Theorem | ltpiord 7379 | Positive integer 'less than' in terms of ordinal membership. (Contributed by NM, 6-Feb-1996.) (Revised by Mario Carneiro, 28-Apr-2015.) |
⊢ ((𝐴 ∈ N ∧ 𝐵 ∈ N) → (𝐴 <N 𝐵 ↔ 𝐴 ∈ 𝐵)) | ||
Theorem | ltsopi 7380 | Positive integer 'less than' is a strict ordering. (Contributed by NM, 8-Feb-1996.) (Proof shortened by Mario Carneiro, 10-Jul-2014.) |
⊢ <N Or N | ||
Theorem | pitric 7381 | Trichotomy for positive integers. (Contributed by Jim Kingdon, 21-Sep-2019.) |
⊢ ((𝐴 ∈ N ∧ 𝐵 ∈ N) → (𝐴 <N 𝐵 ↔ ¬ (𝐴 = 𝐵 ∨ 𝐵 <N 𝐴))) | ||
Theorem | pitri3or 7382 | Trichotomy for positive integers. (Contributed by Jim Kingdon, 21-Sep-2019.) |
⊢ ((𝐴 ∈ N ∧ 𝐵 ∈ N) → (𝐴 <N 𝐵 ∨ 𝐴 = 𝐵 ∨ 𝐵 <N 𝐴)) | ||
Theorem | ltdcpi 7383 | Less-than for positive integers is decidable. (Contributed by Jim Kingdon, 12-Dec-2019.) |
⊢ ((𝐴 ∈ N ∧ 𝐵 ∈ N) → DECID 𝐴 <N 𝐵) | ||
Theorem | ltrelpi 7384 | Positive integer 'less than' is a relation on positive integers. (Contributed by NM, 8-Feb-1996.) |
⊢ <N ⊆ (N × N) | ||
Theorem | dmaddpi 7385 | Domain of addition on positive integers. (Contributed by NM, 26-Aug-1995.) |
⊢ dom +N = (N × N) | ||
Theorem | dmmulpi 7386 | Domain of multiplication on positive integers. (Contributed by NM, 26-Aug-1995.) |
⊢ dom ·N = (N × N) | ||
Theorem | addclpi 7387 | Closure of addition of positive integers. (Contributed by NM, 18-Oct-1995.) |
⊢ ((𝐴 ∈ N ∧ 𝐵 ∈ N) → (𝐴 +N 𝐵) ∈ N) | ||
Theorem | mulclpi 7388 | Closure of multiplication of positive integers. (Contributed by NM, 18-Oct-1995.) |
⊢ ((𝐴 ∈ N ∧ 𝐵 ∈ N) → (𝐴 ·N 𝐵) ∈ N) | ||
Theorem | addcompig 7389 | Addition of positive integers is commutative. (Contributed by Jim Kingdon, 26-Aug-2019.) |
⊢ ((𝐴 ∈ N ∧ 𝐵 ∈ N) → (𝐴 +N 𝐵) = (𝐵 +N 𝐴)) | ||
Theorem | addasspig 7390 | Addition of positive integers is associative. (Contributed by Jim Kingdon, 26-Aug-2019.) |
⊢ ((𝐴 ∈ N ∧ 𝐵 ∈ N ∧ 𝐶 ∈ N) → ((𝐴 +N 𝐵) +N 𝐶) = (𝐴 +N (𝐵 +N 𝐶))) | ||
Theorem | mulcompig 7391 | Multiplication of positive integers is commutative. (Contributed by Jim Kingdon, 26-Aug-2019.) |
⊢ ((𝐴 ∈ N ∧ 𝐵 ∈ N) → (𝐴 ·N 𝐵) = (𝐵 ·N 𝐴)) | ||
Theorem | mulasspig 7392 | Multiplication of positive integers is associative. (Contributed by Jim Kingdon, 26-Aug-2019.) |
⊢ ((𝐴 ∈ N ∧ 𝐵 ∈ N ∧ 𝐶 ∈ N) → ((𝐴 ·N 𝐵) ·N 𝐶) = (𝐴 ·N (𝐵 ·N 𝐶))) | ||
Theorem | distrpig 7393 | Multiplication of positive integers is distributive. (Contributed by Jim Kingdon, 26-Aug-2019.) |
⊢ ((𝐴 ∈ N ∧ 𝐵 ∈ N ∧ 𝐶 ∈ N) → (𝐴 ·N (𝐵 +N 𝐶)) = ((𝐴 ·N 𝐵) +N (𝐴 ·N 𝐶))) | ||
Theorem | addcanpig 7394 | Addition cancellation law for positive integers. (Contributed by Jim Kingdon, 27-Aug-2019.) |
⊢ ((𝐴 ∈ N ∧ 𝐵 ∈ N ∧ 𝐶 ∈ N) → ((𝐴 +N 𝐵) = (𝐴 +N 𝐶) ↔ 𝐵 = 𝐶)) | ||
Theorem | mulcanpig 7395 | Multiplication cancellation law for positive integers. (Contributed by Jim Kingdon, 29-Aug-2019.) |
⊢ ((𝐴 ∈ N ∧ 𝐵 ∈ N ∧ 𝐶 ∈ N) → ((𝐴 ·N 𝐵) = (𝐴 ·N 𝐶) ↔ 𝐵 = 𝐶)) | ||
Theorem | addnidpig 7396 | There is no identity element for addition on positive integers. (Contributed by NM, 28-Nov-1995.) |
⊢ ((𝐴 ∈ N ∧ 𝐵 ∈ N) → ¬ (𝐴 +N 𝐵) = 𝐴) | ||
Theorem | ltexpi 7397* | Ordering on positive integers in terms of existence of sum. (Contributed by NM, 15-Mar-1996.) (Revised by Mario Carneiro, 14-Jun-2013.) |
⊢ ((𝐴 ∈ N ∧ 𝐵 ∈ N) → (𝐴 <N 𝐵 ↔ ∃𝑥 ∈ N (𝐴 +N 𝑥) = 𝐵)) | ||
Theorem | ltapig 7398 | Ordering property of addition for positive integers. (Contributed by Jim Kingdon, 31-Aug-2019.) |
⊢ ((𝐴 ∈ N ∧ 𝐵 ∈ N ∧ 𝐶 ∈ N) → (𝐴 <N 𝐵 ↔ (𝐶 +N 𝐴) <N (𝐶 +N 𝐵))) | ||
Theorem | ltmpig 7399 | Ordering property of multiplication for positive integers. (Contributed by Jim Kingdon, 31-Aug-2019.) |
⊢ ((𝐴 ∈ N ∧ 𝐵 ∈ N ∧ 𝐶 ∈ N) → (𝐴 <N 𝐵 ↔ (𝐶 ·N 𝐴) <N (𝐶 ·N 𝐵))) | ||
Theorem | 1lt2pi 7400 | One is less than two (one plus one). (Contributed by NM, 13-Mar-1996.) |
⊢ 1o <N (1o +N 1o) |
< Previous Next > |
Copyright terms: Public domain | < Previous Next > |