Home | Metamath
Proof Explorer Theorem List (p. 123 of 466) | < 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: | Metamath Proof Explorer
(1-29289) |
Hilbert Space Explorer
(29290-30812) |
Users' Mathboxes
(30813-46532) |
Type | Label | Description |
---|---|---|
Statement | ||
Theorem | 1mhlfehlf 12201 | Prove that 1 - 1/2 = 1/2. (Contributed by David A. Wheeler, 4-Jan-2017.) |
⊢ (1 − (1 / 2)) = (1 / 2) | ||
Theorem | 8th4div3 12202 | An eighth of four thirds is a sixth. (Contributed by Paul Chapman, 24-Nov-2007.) |
⊢ ((1 / 8) · (4 / 3)) = (1 / 6) | ||
Theorem | halfpm6th 12203 | One half plus or minus one sixth. (Contributed by Paul Chapman, 17-Jan-2008.) |
⊢ (((1 / 2) − (1 / 6)) = (1 / 3) ∧ ((1 / 2) + (1 / 6)) = (2 / 3)) | ||
Theorem | it0e0 12204 | i times 0 equals 0. (Contributed by David A. Wheeler, 8-Dec-2018.) |
⊢ (i · 0) = 0 | ||
Theorem | 2mulicn 12205 | (2 · i) ∈ ℂ. (Contributed by David A. Wheeler, 8-Dec-2018.) |
⊢ (2 · i) ∈ ℂ | ||
Theorem | 2muline0 12206 | (2 · i) ≠ 0. (Contributed by David A. Wheeler, 8-Dec-2018.) |
⊢ (2 · i) ≠ 0 | ||
Theorem | halfcl 12207 | Closure of half of a number. (Contributed by NM, 1-Jan-2006.) |
⊢ (𝐴 ∈ ℂ → (𝐴 / 2) ∈ ℂ) | ||
Theorem | rehalfcl 12208 | Real closure of half. (Contributed by NM, 1-Jan-2006.) |
⊢ (𝐴 ∈ ℝ → (𝐴 / 2) ∈ ℝ) | ||
Theorem | half0 12209 | Half of a number is zero iff the number is zero. (Contributed by NM, 20-Apr-2006.) |
⊢ (𝐴 ∈ ℂ → ((𝐴 / 2) = 0 ↔ 𝐴 = 0)) | ||
Theorem | 2halves 12210 | Two halves make a whole. (Contributed by NM, 11-Apr-2005.) |
⊢ (𝐴 ∈ ℂ → ((𝐴 / 2) + (𝐴 / 2)) = 𝐴) | ||
Theorem | halfpos2 12211 | A number is positive iff its half is positive. (Contributed by NM, 10-Apr-2005.) |
⊢ (𝐴 ∈ ℝ → (0 < 𝐴 ↔ 0 < (𝐴 / 2))) | ||
Theorem | halfpos 12212 | A positive number is greater than its half. (Contributed by NM, 28-Oct-2004.) (Proof shortened by Mario Carneiro, 27-May-2016.) |
⊢ (𝐴 ∈ ℝ → (0 < 𝐴 ↔ (𝐴 / 2) < 𝐴)) | ||
Theorem | halfnneg2 12213 | A number is nonnegative iff its half is nonnegative. (Contributed by NM, 9-Dec-2005.) |
⊢ (𝐴 ∈ ℝ → (0 ≤ 𝐴 ↔ 0 ≤ (𝐴 / 2))) | ||
Theorem | halfaddsubcl 12214 | Closure of half-sum and half-difference. (Contributed by Paul Chapman, 12-Oct-2007.) |
⊢ ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ) → (((𝐴 + 𝐵) / 2) ∈ ℂ ∧ ((𝐴 − 𝐵) / 2) ∈ ℂ)) | ||
Theorem | halfaddsub 12215 | Sum and difference of half-sum and half-difference. (Contributed by Paul Chapman, 12-Oct-2007.) |
⊢ ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ) → ((((𝐴 + 𝐵) / 2) + ((𝐴 − 𝐵) / 2)) = 𝐴 ∧ (((𝐴 + 𝐵) / 2) − ((𝐴 − 𝐵) / 2)) = 𝐵)) | ||
Theorem | subhalfhalf 12216 | Subtracting the half of a number from the number yields the half of the number. (Contributed by AV, 28-Jun-2021.) |
⊢ (𝐴 ∈ ℂ → (𝐴 − (𝐴 / 2)) = (𝐴 / 2)) | ||
Theorem | lt2halves 12217 | A sum is less than the whole if each term is less than half. (Contributed by NM, 13-Dec-2006.) |
⊢ ((𝐴 ∈ ℝ ∧ 𝐵 ∈ ℝ ∧ 𝐶 ∈ ℝ) → ((𝐴 < (𝐶 / 2) ∧ 𝐵 < (𝐶 / 2)) → (𝐴 + 𝐵) < 𝐶)) | ||
Theorem | addltmul 12218 | Sum is less than product for numbers greater than 2. (Contributed by Stefan Allan, 24-Sep-2010.) |
⊢ (((𝐴 ∈ ℝ ∧ 𝐵 ∈ ℝ) ∧ (2 < 𝐴 ∧ 2 < 𝐵)) → (𝐴 + 𝐵) < (𝐴 · 𝐵)) | ||
Theorem | nominpos 12219* | There is no smallest positive real number. (Contributed by NM, 28-Oct-2004.) |
⊢ ¬ ∃𝑥 ∈ ℝ (0 < 𝑥 ∧ ¬ ∃𝑦 ∈ ℝ (0 < 𝑦 ∧ 𝑦 < 𝑥)) | ||
Theorem | avglt1 12220 | Ordering property for average. (Contributed by Mario Carneiro, 28-May-2014.) |
⊢ ((𝐴 ∈ ℝ ∧ 𝐵 ∈ ℝ) → (𝐴 < 𝐵 ↔ 𝐴 < ((𝐴 + 𝐵) / 2))) | ||
Theorem | avglt2 12221 | Ordering property for average. (Contributed by Mario Carneiro, 28-May-2014.) |
⊢ ((𝐴 ∈ ℝ ∧ 𝐵 ∈ ℝ) → (𝐴 < 𝐵 ↔ ((𝐴 + 𝐵) / 2) < 𝐵)) | ||
Theorem | avgle1 12222 | Ordering property for average. (Contributed by Mario Carneiro, 28-May-2014.) |
⊢ ((𝐴 ∈ ℝ ∧ 𝐵 ∈ ℝ) → (𝐴 ≤ 𝐵 ↔ 𝐴 ≤ ((𝐴 + 𝐵) / 2))) | ||
Theorem | avgle2 12223 | Ordering property for average. (Contributed by Jeff Hankins, 15-Sep-2013.) (Revised by Mario Carneiro, 28-May-2014.) |
⊢ ((𝐴 ∈ ℝ ∧ 𝐵 ∈ ℝ) → (𝐴 ≤ 𝐵 ↔ ((𝐴 + 𝐵) / 2) ≤ 𝐵)) | ||
Theorem | avgle 12224 | The average of two numbers is less than or equal to at least one of them. (Contributed by NM, 9-Dec-2005.) (Revised by Mario Carneiro, 28-May-2014.) |
⊢ ((𝐴 ∈ ℝ ∧ 𝐵 ∈ ℝ) → (((𝐴 + 𝐵) / 2) ≤ 𝐴 ∨ ((𝐴 + 𝐵) / 2) ≤ 𝐵)) | ||
Theorem | 2timesd 12225 | Two times a number. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℂ) ⇒ ⊢ (𝜑 → (2 · 𝐴) = (𝐴 + 𝐴)) | ||
Theorem | times2d 12226 | A number times 2. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℂ) ⇒ ⊢ (𝜑 → (𝐴 · 2) = (𝐴 + 𝐴)) | ||
Theorem | halfcld 12227 | Closure of half of a number (frequently used special case). (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℂ) ⇒ ⊢ (𝜑 → (𝐴 / 2) ∈ ℂ) | ||
Theorem | 2halvesd 12228 | Two halves make a whole. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℂ) ⇒ ⊢ (𝜑 → ((𝐴 / 2) + (𝐴 / 2)) = 𝐴) | ||
Theorem | rehalfcld 12229 | Real closure of half. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) ⇒ ⊢ (𝜑 → (𝐴 / 2) ∈ ℝ) | ||
Theorem | lt2halvesd 12230 | A sum is less than the whole if each term is less than half. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) & ⊢ (𝜑 → 𝐶 ∈ ℝ) & ⊢ (𝜑 → 𝐴 < (𝐶 / 2)) & ⊢ (𝜑 → 𝐵 < (𝐶 / 2)) ⇒ ⊢ (𝜑 → (𝐴 + 𝐵) < 𝐶) | ||
Theorem | rehalfcli 12231 | Half a real number is real. Inference form. (Contributed by David Moews, 28-Feb-2017.) |
⊢ 𝐴 ∈ ℝ ⇒ ⊢ (𝐴 / 2) ∈ ℝ | ||
Theorem | lt2addmuld 12232 | If two real numbers are less than a third real number, the sum of the two real numbers is less than twice the third real number. (Contributed by Glauco Siliprandi, 11-Dec-2019.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) & ⊢ (𝜑 → 𝐶 ∈ ℝ) & ⊢ (𝜑 → 𝐴 < 𝐶) & ⊢ (𝜑 → 𝐵 < 𝐶) ⇒ ⊢ (𝜑 → (𝐴 + 𝐵) < (2 · 𝐶)) | ||
Theorem | add1p1 12233 | Adding two times 1 to a number. (Contributed by AV, 22-Sep-2018.) |
⊢ (𝑁 ∈ ℂ → ((𝑁 + 1) + 1) = (𝑁 + 2)) | ||
Theorem | sub1m1 12234 | Subtracting two times 1 from a number. (Contributed by AV, 23-Oct-2018.) |
⊢ (𝑁 ∈ ℂ → ((𝑁 − 1) − 1) = (𝑁 − 2)) | ||
Theorem | cnm2m1cnm3 12235 | Subtracting 2 and afterwards 1 from a number results in the difference between the number and 3. (Contributed by Alexander van der Vekens, 16-Sep-2018.) |
⊢ (𝐴 ∈ ℂ → ((𝐴 − 2) − 1) = (𝐴 − 3)) | ||
Theorem | xp1d2m1eqxm1d2 12236 | A complex number increased by 1, then divided by 2, then decreased by 1 equals the complex number decreased by 1 and then divided by 2. (Contributed by AV, 24-May-2020.) |
⊢ (𝑋 ∈ ℂ → (((𝑋 + 1) / 2) − 1) = ((𝑋 − 1) / 2)) | ||
Theorem | div4p1lem1div2 12237 | An integer greater than 5, divided by 4 and increased by 1, is less than or equal to the half of the integer minus 1. (Contributed by AV, 8-Jul-2021.) |
⊢ ((𝑁 ∈ ℝ ∧ 6 ≤ 𝑁) → ((𝑁 / 4) + 1) ≤ ((𝑁 − 1) / 2)) | ||
Theorem | nnunb 12238* | The set of positive integers is unbounded above. Theorem I.28 of [Apostol] p. 26. (Contributed by NM, 21-Jan-1997.) |
⊢ ¬ ∃𝑥 ∈ ℝ ∀𝑦 ∈ ℕ (𝑦 < 𝑥 ∨ 𝑦 = 𝑥) | ||
Theorem | arch 12239* | Archimedean property of real numbers. For any real number, there is an integer greater than it. Theorem I.29 of [Apostol] p. 26. (Contributed by NM, 21-Jan-1997.) |
⊢ (𝐴 ∈ ℝ → ∃𝑛 ∈ ℕ 𝐴 < 𝑛) | ||
Theorem | nnrecl 12240* | There exists a positive integer whose reciprocal is less than a given positive real. Exercise 3 of [Apostol] p. 28. (Contributed by NM, 8-Nov-2004.) |
⊢ ((𝐴 ∈ ℝ ∧ 0 < 𝐴) → ∃𝑛 ∈ ℕ (1 / 𝑛) < 𝐴) | ||
Theorem | bndndx 12241* | A bounded real sequence 𝐴(𝑘) is less than or equal to at least one of its indices. (Contributed by NM, 18-Jan-2008.) |
⊢ (∃𝑥 ∈ ℝ ∀𝑘 ∈ ℕ (𝐴 ∈ ℝ ∧ 𝐴 ≤ 𝑥) → ∃𝑘 ∈ ℕ 𝐴 ≤ 𝑘) | ||
Syntax | cn0 12242 | Extend class notation to include the class of nonnegative integers. |
class ℕ0 | ||
Definition | df-n0 12243 | Define the set of nonnegative integers. (Contributed by Raph Levien, 10-Dec-2002.) |
⊢ ℕ0 = (ℕ ∪ {0}) | ||
Theorem | elnn0 12244 | Nonnegative integers expressed in terms of naturals and zero. (Contributed by Raph Levien, 10-Dec-2002.) |
⊢ (𝐴 ∈ ℕ0 ↔ (𝐴 ∈ ℕ ∨ 𝐴 = 0)) | ||
Theorem | nnssnn0 12245 | Positive naturals are a subset of nonnegative integers. (Contributed by Raph Levien, 10-Dec-2002.) |
⊢ ℕ ⊆ ℕ0 | ||
Theorem | nn0ssre 12246 | Nonnegative integers are a subset of the reals. (Contributed by Raph Levien, 10-Dec-2002.) |
⊢ ℕ0 ⊆ ℝ | ||
Theorem | nn0sscn 12247 | Nonnegative integers are a subset of the complex numbers. (Contributed by NM, 9-May-2004.) Reduce dependencies on axioms. (Revised by Steven Nguyen, 8-Oct-2022.) |
⊢ ℕ0 ⊆ ℂ | ||
Theorem | nn0ex 12248 | The set of nonnegative integers exists. (Contributed by NM, 18-Jul-2004.) |
⊢ ℕ0 ∈ V | ||
Theorem | nnnn0 12249 | A positive integer is a nonnegative integer. (Contributed by NM, 9-May-2004.) |
⊢ (𝐴 ∈ ℕ → 𝐴 ∈ ℕ0) | ||
Theorem | nnnn0i 12250 | A positive integer is a nonnegative integer. (Contributed by NM, 20-Jun-2005.) |
⊢ 𝑁 ∈ ℕ ⇒ ⊢ 𝑁 ∈ ℕ0 | ||
Theorem | nn0re 12251 | A nonnegative integer is a real number. (Contributed by NM, 9-May-2004.) |
⊢ (𝐴 ∈ ℕ0 → 𝐴 ∈ ℝ) | ||
Theorem | nn0cn 12252 | A nonnegative integer is a complex number. (Contributed by NM, 9-May-2004.) |
⊢ (𝐴 ∈ ℕ0 → 𝐴 ∈ ℂ) | ||
Theorem | nn0rei 12253 | A nonnegative integer is a real number. (Contributed by NM, 14-May-2003.) |
⊢ 𝐴 ∈ ℕ0 ⇒ ⊢ 𝐴 ∈ ℝ | ||
Theorem | nn0cni 12254 | A nonnegative integer is a complex number. (Contributed by NM, 14-May-2003.) Reduce dependencies on axioms. (Revised by Steven Nguyen, 8-Oct-2022.) |
⊢ 𝐴 ∈ ℕ0 ⇒ ⊢ 𝐴 ∈ ℂ | ||
Theorem | dfn2 12255 | The set of positive integers defined in terms of nonnegative integers. (Contributed by NM, 23-Sep-2007.) (Proof shortened by Mario Carneiro, 13-Feb-2013.) |
⊢ ℕ = (ℕ0 ∖ {0}) | ||
Theorem | elnnne0 12256 | The positive integer property expressed in terms of difference from zero. (Contributed by Stefan O'Rear, 12-Sep-2015.) |
⊢ (𝑁 ∈ ℕ ↔ (𝑁 ∈ ℕ0 ∧ 𝑁 ≠ 0)) | ||
Theorem | 0nn0 12257 | 0 is a nonnegative integer. (Contributed by Raph Levien, 10-Dec-2002.) |
⊢ 0 ∈ ℕ0 | ||
Theorem | 1nn0 12258 | 1 is a nonnegative integer. (Contributed by Raph Levien, 10-Dec-2002.) |
⊢ 1 ∈ ℕ0 | ||
Theorem | 2nn0 12259 | 2 is a nonnegative integer. (Contributed by Raph Levien, 10-Dec-2002.) |
⊢ 2 ∈ ℕ0 | ||
Theorem | 3nn0 12260 | 3 is a nonnegative integer. (Contributed by Mario Carneiro, 18-Feb-2014.) |
⊢ 3 ∈ ℕ0 | ||
Theorem | 4nn0 12261 | 4 is a nonnegative integer. (Contributed by Mario Carneiro, 18-Feb-2014.) |
⊢ 4 ∈ ℕ0 | ||
Theorem | 5nn0 12262 | 5 is a nonnegative integer. (Contributed by Mario Carneiro, 19-Apr-2015.) |
⊢ 5 ∈ ℕ0 | ||
Theorem | 6nn0 12263 | 6 is a nonnegative integer. (Contributed by Mario Carneiro, 19-Apr-2015.) |
⊢ 6 ∈ ℕ0 | ||
Theorem | 7nn0 12264 | 7 is a nonnegative integer. (Contributed by Mario Carneiro, 19-Apr-2015.) |
⊢ 7 ∈ ℕ0 | ||
Theorem | 8nn0 12265 | 8 is a nonnegative integer. (Contributed by Mario Carneiro, 19-Apr-2015.) |
⊢ 8 ∈ ℕ0 | ||
Theorem | 9nn0 12266 | 9 is a nonnegative integer. (Contributed by Mario Carneiro, 19-Apr-2015.) |
⊢ 9 ∈ ℕ0 | ||
Theorem | nn0ge0 12267 | A nonnegative integer is greater than or equal to zero. (Contributed by NM, 9-May-2004.) (Revised by Mario Carneiro, 16-May-2014.) |
⊢ (𝑁 ∈ ℕ0 → 0 ≤ 𝑁) | ||
Theorem | nn0nlt0 12268 | A nonnegative integer is not less than zero. (Contributed by NM, 9-May-2004.) (Revised by Mario Carneiro, 27-May-2016.) |
⊢ (𝐴 ∈ ℕ0 → ¬ 𝐴 < 0) | ||
Theorem | nn0ge0i 12269 | Nonnegative integers are nonnegative. (Contributed by Raph Levien, 10-Dec-2002.) |
⊢ 𝑁 ∈ ℕ0 ⇒ ⊢ 0 ≤ 𝑁 | ||
Theorem | nn0le0eq0 12270 | A nonnegative integer is less than or equal to zero iff it is equal to zero. (Contributed by NM, 9-Dec-2005.) |
⊢ (𝑁 ∈ ℕ0 → (𝑁 ≤ 0 ↔ 𝑁 = 0)) | ||
Theorem | nn0p1gt0 12271 | A nonnegative integer increased by 1 is greater than 0. (Contributed by Alexander van der Vekens, 3-Oct-2018.) |
⊢ (𝑁 ∈ ℕ0 → 0 < (𝑁 + 1)) | ||
Theorem | nnnn0addcl 12272 | A positive integer plus a nonnegative integer is a positive integer. (Contributed by NM, 20-Apr-2005.) (Proof shortened by Mario Carneiro, 16-May-2014.) |
⊢ ((𝑀 ∈ ℕ ∧ 𝑁 ∈ ℕ0) → (𝑀 + 𝑁) ∈ ℕ) | ||
Theorem | nn0nnaddcl 12273 | A nonnegative integer plus a positive integer is a positive integer. (Contributed by NM, 22-Dec-2005.) |
⊢ ((𝑀 ∈ ℕ0 ∧ 𝑁 ∈ ℕ) → (𝑀 + 𝑁) ∈ ℕ) | ||
Theorem | 0mnnnnn0 12274 | The result of subtracting a positive integer from 0 is not a nonnegative integer. (Contributed by Alexander van der Vekens, 19-Mar-2018.) |
⊢ (𝑁 ∈ ℕ → (0 − 𝑁) ∉ ℕ0) | ||
Theorem | un0addcl 12275 | If 𝑆 is closed under addition, then so is 𝑆 ∪ {0}. (Contributed by Mario Carneiro, 17-Jul-2014.) |
⊢ (𝜑 → 𝑆 ⊆ ℂ) & ⊢ 𝑇 = (𝑆 ∪ {0}) & ⊢ ((𝜑 ∧ (𝑀 ∈ 𝑆 ∧ 𝑁 ∈ 𝑆)) → (𝑀 + 𝑁) ∈ 𝑆) ⇒ ⊢ ((𝜑 ∧ (𝑀 ∈ 𝑇 ∧ 𝑁 ∈ 𝑇)) → (𝑀 + 𝑁) ∈ 𝑇) | ||
Theorem | un0mulcl 12276 | If 𝑆 is closed under multiplication, then so is 𝑆 ∪ {0}. (Contributed by Mario Carneiro, 17-Jul-2014.) |
⊢ (𝜑 → 𝑆 ⊆ ℂ) & ⊢ 𝑇 = (𝑆 ∪ {0}) & ⊢ ((𝜑 ∧ (𝑀 ∈ 𝑆 ∧ 𝑁 ∈ 𝑆)) → (𝑀 · 𝑁) ∈ 𝑆) ⇒ ⊢ ((𝜑 ∧ (𝑀 ∈ 𝑇 ∧ 𝑁 ∈ 𝑇)) → (𝑀 · 𝑁) ∈ 𝑇) | ||
Theorem | nn0addcl 12277 | Closure of addition of nonnegative integers. (Contributed by Raph Levien, 10-Dec-2002.) (Proof shortened by Mario Carneiro, 17-Jul-2014.) |
⊢ ((𝑀 ∈ ℕ0 ∧ 𝑁 ∈ ℕ0) → (𝑀 + 𝑁) ∈ ℕ0) | ||
Theorem | nn0mulcl 12278 | Closure of multiplication of nonnegative integers. (Contributed by NM, 22-Jul-2004.) (Proof shortened by Mario Carneiro, 17-Jul-2014.) |
⊢ ((𝑀 ∈ ℕ0 ∧ 𝑁 ∈ ℕ0) → (𝑀 · 𝑁) ∈ ℕ0) | ||
Theorem | nn0addcli 12279 | Closure of addition of nonnegative integers, inference form. (Contributed by Raph Levien, 10-Dec-2002.) |
⊢ 𝑀 ∈ ℕ0 & ⊢ 𝑁 ∈ ℕ0 ⇒ ⊢ (𝑀 + 𝑁) ∈ ℕ0 | ||
Theorem | nn0mulcli 12280 | Closure of multiplication of nonnegative integers, inference form. (Contributed by Raph Levien, 10-Dec-2002.) |
⊢ 𝑀 ∈ ℕ0 & ⊢ 𝑁 ∈ ℕ0 ⇒ ⊢ (𝑀 · 𝑁) ∈ ℕ0 | ||
Theorem | nn0p1nn 12281 | A nonnegative integer plus 1 is a positive integer. Strengthening of peano2nn 11994. (Contributed by Raph Levien, 30-Jun-2006.) (Revised by Mario Carneiro, 16-May-2014.) |
⊢ (𝑁 ∈ ℕ0 → (𝑁 + 1) ∈ ℕ) | ||
Theorem | peano2nn0 12282 | Second Peano postulate for nonnegative integers. (Contributed by NM, 9-May-2004.) |
⊢ (𝑁 ∈ ℕ0 → (𝑁 + 1) ∈ ℕ0) | ||
Theorem | nnm1nn0 12283 | A positive integer minus 1 is a nonnegative integer. (Contributed by Jason Orendorff, 24-Jan-2007.) (Revised by Mario Carneiro, 16-May-2014.) |
⊢ (𝑁 ∈ ℕ → (𝑁 − 1) ∈ ℕ0) | ||
Theorem | elnn0nn 12284 | The nonnegative integer property expressed in terms of positive integers. (Contributed by NM, 10-May-2004.) (Proof shortened by Mario Carneiro, 16-May-2014.) |
⊢ (𝑁 ∈ ℕ0 ↔ (𝑁 ∈ ℂ ∧ (𝑁 + 1) ∈ ℕ)) | ||
Theorem | elnnnn0 12285 | The positive integer property expressed in terms of nonnegative integers. (Contributed by NM, 10-May-2004.) |
⊢ (𝑁 ∈ ℕ ↔ (𝑁 ∈ ℂ ∧ (𝑁 − 1) ∈ ℕ0)) | ||
Theorem | elnnnn0b 12286 | The positive integer property expressed in terms of nonnegative integers. (Contributed by NM, 1-Sep-2005.) |
⊢ (𝑁 ∈ ℕ ↔ (𝑁 ∈ ℕ0 ∧ 0 < 𝑁)) | ||
Theorem | elnnnn0c 12287 | The positive integer property expressed in terms of nonnegative integers. (Contributed by NM, 10-Jan-2006.) |
⊢ (𝑁 ∈ ℕ ↔ (𝑁 ∈ ℕ0 ∧ 1 ≤ 𝑁)) | ||
Theorem | nn0addge1 12288 | A number is less than or equal to itself plus a nonnegative integer. (Contributed by NM, 10-Mar-2005.) |
⊢ ((𝐴 ∈ ℝ ∧ 𝑁 ∈ ℕ0) → 𝐴 ≤ (𝐴 + 𝑁)) | ||
Theorem | nn0addge2 12289 | A number is less than or equal to itself plus a nonnegative integer. (Contributed by NM, 10-Mar-2005.) |
⊢ ((𝐴 ∈ ℝ ∧ 𝑁 ∈ ℕ0) → 𝐴 ≤ (𝑁 + 𝐴)) | ||
Theorem | nn0addge1i 12290 | A number is less than or equal to itself plus a nonnegative integer. (Contributed by NM, 10-Mar-2005.) |
⊢ 𝐴 ∈ ℝ & ⊢ 𝑁 ∈ ℕ0 ⇒ ⊢ 𝐴 ≤ (𝐴 + 𝑁) | ||
Theorem | nn0addge2i 12291 | A number is less than or equal to itself plus a nonnegative integer. (Contributed by NM, 10-Mar-2005.) |
⊢ 𝐴 ∈ ℝ & ⊢ 𝑁 ∈ ℕ0 ⇒ ⊢ 𝐴 ≤ (𝑁 + 𝐴) | ||
Theorem | nn0sub 12292 | Subtraction of nonnegative integers. (Contributed by NM, 9-May-2004.) (Proof shortened by Mario Carneiro, 16-May-2014.) |
⊢ ((𝑀 ∈ ℕ0 ∧ 𝑁 ∈ ℕ0) → (𝑀 ≤ 𝑁 ↔ (𝑁 − 𝑀) ∈ ℕ0)) | ||
Theorem | ltsubnn0 12293 | Subtracting a nonnegative integer from a nonnegative integer which is greater than the first one results in a nonnegative integer. (Contributed by Alexander van der Vekens, 6-Apr-2018.) |
⊢ ((𝐴 ∈ ℕ0 ∧ 𝐵 ∈ ℕ0) → (𝐵 < 𝐴 → (𝐴 − 𝐵) ∈ ℕ0)) | ||
Theorem | nn0negleid 12294 | A nonnegative integer is greater than or equal to its negative. (Contributed by AV, 13-Aug-2021.) |
⊢ (𝐴 ∈ ℕ0 → -𝐴 ≤ 𝐴) | ||
Theorem | difgtsumgt 12295 | If the difference of a real number and a nonnegative integer is greater than another real number, the sum of the real number and the nonnegative integer is also greater than the other real number. (Contributed by AV, 13-Aug-2021.) |
⊢ ((𝐴 ∈ ℝ ∧ 𝐵 ∈ ℕ0 ∧ 𝐶 ∈ ℝ) → (𝐶 < (𝐴 − 𝐵) → 𝐶 < (𝐴 + 𝐵))) | ||
Theorem | nn0le2xi 12296 | A nonnegative integer is less than or equal to twice itself. (Contributed by Raph Levien, 10-Dec-2002.) |
⊢ 𝑁 ∈ ℕ0 ⇒ ⊢ 𝑁 ≤ (2 · 𝑁) | ||
Theorem | nn0lele2xi 12297 | 'Less than or equal to' implies 'less than or equal to twice' for nonnegative integers. (Contributed by Raph Levien, 10-Dec-2002.) |
⊢ 𝑀 ∈ ℕ0 & ⊢ 𝑁 ∈ ℕ0 ⇒ ⊢ (𝑁 ≤ 𝑀 → 𝑁 ≤ (2 · 𝑀)) | ||
Theorem | frnnn0supp 12298 | Two ways to write the support of a function on ℕ0. (Contributed by Mario Carneiro, 29-Dec-2014.) (Revised by AV, 7-Jul-2019.) |
⊢ ((𝐼 ∈ 𝑉 ∧ 𝐹:𝐼⟶ℕ0) → (𝐹 supp 0) = (◡𝐹 “ ℕ)) | ||
Theorem | frnnn0fsupp 12299 | A function on ℕ0 is finitely supported iff its support is finite. (Contributed by AV, 8-Jul-2019.) |
⊢ ((𝐼 ∈ 𝑉 ∧ 𝐹:𝐼⟶ℕ0) → (𝐹 finSupp 0 ↔ (◡𝐹 “ ℕ) ∈ Fin)) | ||
Theorem | frnnn0suppg 12300 | Version of frnnn0supp 12298 avoiding ax-rep 5210 by assuming 𝐹 is a set rather than its domain 𝐼. (Contributed by SN, 5-Aug-2024.) |
⊢ ((𝐹 ∈ 𝑉 ∧ 𝐹:𝐼⟶ℕ0) → (𝐹 supp 0) = (◡𝐹 “ ℕ)) |
< Previous Next > |
Copyright terms: Public domain | < Previous Next > |