| Metamath
Proof Explorer Theorem List (p. 131 of 497) | < 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-30845) |
(30846-32368) |
(32369-49617) |
| Type | Label | Description |
|---|---|---|
| Statement | ||
| Theorem | xrex 13001 | The set of extended reals exists. (Contributed by NM, 24-Dec-2006.) |
| ⊢ ℝ* ∈ V | ||
| Theorem | mpoaddex 13002* | The addition operation is a set. Version of addex 13003 using maps-to notation , which does not require ax-addf 11206. (Contributed by GG, 31-Mar-2025.) |
| ⊢ (𝑥 ∈ ℂ, 𝑦 ∈ ℂ ↦ (𝑥 + 𝑦)) ∈ V | ||
| Theorem | addex 13003 | The addition operation is a set. (Contributed by NM, 19-Oct-2004.) (Revised by Mario Carneiro, 17-Nov-2014.) |
| ⊢ + ∈ V | ||
| Theorem | mpomulex 13004* | The multiplication operation is a set. Version of mulex 13005 using maps-to notation , which does not require ax-mulf 11207. (Contributed by GG, 16-Mar-2025.) |
| ⊢ (𝑥 ∈ ℂ, 𝑦 ∈ ℂ ↦ (𝑥 · 𝑦)) ∈ V | ||
| Theorem | mulex 13005 | The multiplication operation is a set. (Contributed by NM, 19-Oct-2004.) (Revised by Mario Carneiro, 17-Nov-2014.) |
| ⊢ · ∈ V | ||
| Syntax | crp 13006 | Extend class notation to include the class of positive reals. |
| class ℝ+ | ||
| Definition | df-rp 13007 | Define the set of positive reals. Definition of positive numbers in [Apostol] p. 20. (Contributed by NM, 27-Oct-2007.) |
| ⊢ ℝ+ = {𝑥 ∈ ℝ ∣ 0 < 𝑥} | ||
| Theorem | elrp 13008 | Membership in the set of positive reals. (Contributed by NM, 27-Oct-2007.) |
| ⊢ (𝐴 ∈ ℝ+ ↔ (𝐴 ∈ ℝ ∧ 0 < 𝐴)) | ||
| Theorem | elrpii 13009 | Membership in the set of positive reals. (Contributed by NM, 23-Feb-2008.) |
| ⊢ 𝐴 ∈ ℝ & ⊢ 0 < 𝐴 ⇒ ⊢ 𝐴 ∈ ℝ+ | ||
| Theorem | 1rp 13010 | 1 is a positive real. (Contributed by Jeff Hankins, 23-Nov-2008.) |
| ⊢ 1 ∈ ℝ+ | ||
| Theorem | 2rp 13011 | 2 is a positive real. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ 2 ∈ ℝ+ | ||
| Theorem | 3rp 13012 | 3 is a positive real. (Contributed by Glauco Siliprandi, 11-Dec-2019.) |
| ⊢ 3 ∈ ℝ+ | ||
| Theorem | 5rp 13013 | 5 is a positive real. (Contributed by SN, 26-Aug-2025.) |
| ⊢ 5 ∈ ℝ+ | ||
| Theorem | rpssre 13014 | The positive reals are a subset of the reals. (Contributed by NM, 24-Feb-2008.) |
| ⊢ ℝ+ ⊆ ℝ | ||
| Theorem | rpre 13015 | A positive real is a real. (Contributed by NM, 27-Oct-2007.) (Proof shortened by Steven Nguyen, 8-Oct-2022.) |
| ⊢ (𝐴 ∈ ℝ+ → 𝐴 ∈ ℝ) | ||
| Theorem | rpxr 13016 | A positive real is an extended real. (Contributed by Mario Carneiro, 21-Aug-2015.) |
| ⊢ (𝐴 ∈ ℝ+ → 𝐴 ∈ ℝ*) | ||
| Theorem | rpcn 13017 | A positive real is a complex number. (Contributed by NM, 11-Nov-2008.) |
| ⊢ (𝐴 ∈ ℝ+ → 𝐴 ∈ ℂ) | ||
| Theorem | nnrp 13018 | A positive integer is a positive real. (Contributed by NM, 28-Nov-2008.) |
| ⊢ (𝐴 ∈ ℕ → 𝐴 ∈ ℝ+) | ||
| Theorem | rpgt0 13019 | A positive real is greater than zero. (Contributed by FL, 27-Dec-2007.) |
| ⊢ (𝐴 ∈ ℝ+ → 0 < 𝐴) | ||
| Theorem | rpge0 13020 | A positive real is greater than or equal to zero. (Contributed by NM, 22-Feb-2008.) |
| ⊢ (𝐴 ∈ ℝ+ → 0 ≤ 𝐴) | ||
| Theorem | rpregt0 13021 | A positive real is a positive real number. (Contributed by NM, 11-Nov-2008.) (Revised by Mario Carneiro, 31-Jan-2014.) |
| ⊢ (𝐴 ∈ ℝ+ → (𝐴 ∈ ℝ ∧ 0 < 𝐴)) | ||
| Theorem | rprege0 13022 | A positive real is a nonnegative real number. (Contributed by Mario Carneiro, 31-Jan-2014.) |
| ⊢ (𝐴 ∈ ℝ+ → (𝐴 ∈ ℝ ∧ 0 ≤ 𝐴)) | ||
| Theorem | rpne0 13023 | A positive real is nonzero. (Contributed by NM, 18-Jul-2008.) |
| ⊢ (𝐴 ∈ ℝ+ → 𝐴 ≠ 0) | ||
| Theorem | rprene0 13024 | A positive real is a nonzero real number. (Contributed by NM, 11-Nov-2008.) |
| ⊢ (𝐴 ∈ ℝ+ → (𝐴 ∈ ℝ ∧ 𝐴 ≠ 0)) | ||
| Theorem | rpcnne0 13025 | A positive real is a nonzero complex number. (Contributed by NM, 11-Nov-2008.) |
| ⊢ (𝐴 ∈ ℝ+ → (𝐴 ∈ ℂ ∧ 𝐴 ≠ 0)) | ||
| Theorem | rpcndif0 13026 | A positive real number is a complex number not being 0. (Contributed by AV, 29-May-2020.) |
| ⊢ (𝐴 ∈ ℝ+ → 𝐴 ∈ (ℂ ∖ {0})) | ||
| Theorem | ralrp 13027 | Quantification over positive reals. (Contributed by NM, 12-Feb-2008.) |
| ⊢ (∀𝑥 ∈ ℝ+ 𝜑 ↔ ∀𝑥 ∈ ℝ (0 < 𝑥 → 𝜑)) | ||
| Theorem | rexrp 13028 | Quantification over positive reals. (Contributed by Mario Carneiro, 21-May-2014.) |
| ⊢ (∃𝑥 ∈ ℝ+ 𝜑 ↔ ∃𝑥 ∈ ℝ (0 < 𝑥 ∧ 𝜑)) | ||
| Theorem | rpaddcl 13029 | Closure law for addition of positive reals. Part of Axiom 7 of [Apostol] p. 20. (Contributed by NM, 27-Oct-2007.) |
| ⊢ ((𝐴 ∈ ℝ+ ∧ 𝐵 ∈ ℝ+) → (𝐴 + 𝐵) ∈ ℝ+) | ||
| Theorem | rpmulcl 13030 | Closure law for multiplication of positive reals. Part of Axiom 7 of [Apostol] p. 20. (Contributed by NM, 27-Oct-2007.) |
| ⊢ ((𝐴 ∈ ℝ+ ∧ 𝐵 ∈ ℝ+) → (𝐴 · 𝐵) ∈ ℝ+) | ||
| Theorem | rpmtmip 13031 | "Minus times minus is plus", see also nnmtmip 12264, holds for positive reals, too (formalized to "The product of two negative reals is a positive real"). "The reason for this" in this case is that (-𝐴 · -𝐵) = (𝐴 · 𝐵) for all complex numbers 𝐴 and 𝐵 because of mul2neg 11674, 𝐴 and 𝐵 are complex numbers because of rpcn 13017, and (𝐴 · 𝐵) ∈ ℝ+ because of rpmulcl 13030. Note that the opposites -𝐴 and -𝐵 of the positive reals 𝐴 and 𝐵 are negative reals. (Contributed by AV, 23-Dec-2022.) |
| ⊢ ((𝐴 ∈ ℝ+ ∧ 𝐵 ∈ ℝ+) → (-𝐴 · -𝐵) ∈ ℝ+) | ||
| Theorem | rpdivcl 13032 | Closure law for division of positive reals. (Contributed by FL, 27-Dec-2007.) |
| ⊢ ((𝐴 ∈ ℝ+ ∧ 𝐵 ∈ ℝ+) → (𝐴 / 𝐵) ∈ ℝ+) | ||
| Theorem | rpreccl 13033 | Closure law for reciprocation of positive reals. (Contributed by Jeff Hankins, 23-Nov-2008.) |
| ⊢ (𝐴 ∈ ℝ+ → (1 / 𝐴) ∈ ℝ+) | ||
| Theorem | rphalfcl 13034 | Closure law for half of a positive real. (Contributed by Mario Carneiro, 31-Jan-2014.) |
| ⊢ (𝐴 ∈ ℝ+ → (𝐴 / 2) ∈ ℝ+) | ||
| Theorem | rpgecl 13035 | A number greater than or equal to a positive real is positive real. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ ((𝐴 ∈ ℝ+ ∧ 𝐵 ∈ ℝ ∧ 𝐴 ≤ 𝐵) → 𝐵 ∈ ℝ+) | ||
| Theorem | rphalflt 13036 | Half of a positive real is less than the original number. (Contributed by Mario Carneiro, 21-May-2014.) |
| ⊢ (𝐴 ∈ ℝ+ → (𝐴 / 2) < 𝐴) | ||
| Theorem | rerpdivcl 13037 | Closure law for division of a real by a positive real. (Contributed by NM, 10-Nov-2008.) |
| ⊢ ((𝐴 ∈ ℝ ∧ 𝐵 ∈ ℝ+) → (𝐴 / 𝐵) ∈ ℝ) | ||
| Theorem | ge0p1rp 13038 | A nonnegative number plus one is a positive number. (Contributed by Mario Carneiro, 5-Oct-2015.) |
| ⊢ ((𝐴 ∈ ℝ ∧ 0 ≤ 𝐴) → (𝐴 + 1) ∈ ℝ+) | ||
| Theorem | rpneg 13039 | Either a nonzero real or its negation is a positive real, but not both. Axiom 8 of [Apostol] p. 20. (Contributed by NM, 7-Nov-2008.) |
| ⊢ ((𝐴 ∈ ℝ ∧ 𝐴 ≠ 0) → (𝐴 ∈ ℝ+ ↔ ¬ -𝐴 ∈ ℝ+)) | ||
| Theorem | negelrp 13040 | Elementhood of a negation in the positive real numbers. (Contributed by Thierry Arnoux, 19-Sep-2018.) |
| ⊢ (𝐴 ∈ ℝ → (-𝐴 ∈ ℝ+ ↔ 𝐴 < 0)) | ||
| Theorem | negelrpd 13041 | The negation of a negative number is in the positive real numbers. (Contributed by Glauco Siliprandi, 26-Jun-2021.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐴 < 0) ⇒ ⊢ (𝜑 → -𝐴 ∈ ℝ+) | ||
| Theorem | 0nrp 13042 | Zero is not a positive real. Axiom 9 of [Apostol] p. 20. (Contributed by NM, 27-Oct-2007.) |
| ⊢ ¬ 0 ∈ ℝ+ | ||
| Theorem | ltsubrp 13043 | Subtracting a positive real from another number decreases it. (Contributed by FL, 27-Dec-2007.) |
| ⊢ ((𝐴 ∈ ℝ ∧ 𝐵 ∈ ℝ+) → (𝐴 − 𝐵) < 𝐴) | ||
| Theorem | ltaddrp 13044 | Adding a positive number to another number increases it. (Contributed by FL, 27-Dec-2007.) |
| ⊢ ((𝐴 ∈ ℝ ∧ 𝐵 ∈ ℝ+) → 𝐴 < (𝐴 + 𝐵)) | ||
| Theorem | difrp 13045 | Two ways to say one number is less than another. (Contributed by Mario Carneiro, 21-May-2014.) |
| ⊢ ((𝐴 ∈ ℝ ∧ 𝐵 ∈ ℝ) → (𝐴 < 𝐵 ↔ (𝐵 − 𝐴) ∈ ℝ+)) | ||
| Theorem | elrpd 13046 | Membership in the set of positive reals. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 0 < 𝐴) ⇒ ⊢ (𝜑 → 𝐴 ∈ ℝ+) | ||
| Theorem | nnrpd 13047 | A positive integer is a positive real. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℕ) ⇒ ⊢ (𝜑 → 𝐴 ∈ ℝ+) | ||
| Theorem | zgt1rpn0n1 13048 | An integer greater than 1 is a positive real number not equal to 0 or 1. Useful for working with integer logarithm bases (which is a common case, e.g., base 2, base 3, or base 10). (Contributed by Thierry Arnoux, 26-Sep-2017.) (Proof shortened by AV, 9-Jul-2022.) |
| ⊢ (𝐵 ∈ (ℤ≥‘2) → (𝐵 ∈ ℝ+ ∧ 𝐵 ≠ 0 ∧ 𝐵 ≠ 1)) | ||
| Theorem | rpred 13049 | A positive real is a real. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ+) ⇒ ⊢ (𝜑 → 𝐴 ∈ ℝ) | ||
| Theorem | rpxrd 13050 | A positive real is an extended real. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ+) ⇒ ⊢ (𝜑 → 𝐴 ∈ ℝ*) | ||
| Theorem | rpcnd 13051 | A positive real is a complex number. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ+) ⇒ ⊢ (𝜑 → 𝐴 ∈ ℂ) | ||
| Theorem | rpgt0d 13052 | A positive real is greater than zero. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ+) ⇒ ⊢ (𝜑 → 0 < 𝐴) | ||
| Theorem | rpge0d 13053 | A positive real is greater than or equal to zero. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ+) ⇒ ⊢ (𝜑 → 0 ≤ 𝐴) | ||
| Theorem | rpne0d 13054 | A positive real is nonzero. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ+) ⇒ ⊢ (𝜑 → 𝐴 ≠ 0) | ||
| Theorem | rpregt0d 13055 | A positive real is real and greater than zero. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ+) ⇒ ⊢ (𝜑 → (𝐴 ∈ ℝ ∧ 0 < 𝐴)) | ||
| Theorem | rprege0d 13056 | A positive real is real and greater than or equal to zero. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ+) ⇒ ⊢ (𝜑 → (𝐴 ∈ ℝ ∧ 0 ≤ 𝐴)) | ||
| Theorem | rprene0d 13057 | A positive real is a nonzero real number. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ+) ⇒ ⊢ (𝜑 → (𝐴 ∈ ℝ ∧ 𝐴 ≠ 0)) | ||
| Theorem | rpcnne0d 13058 | A positive real is a nonzero complex number. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ+) ⇒ ⊢ (𝜑 → (𝐴 ∈ ℂ ∧ 𝐴 ≠ 0)) | ||
| Theorem | rpreccld 13059 | Closure law for reciprocation of positive reals. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ+) ⇒ ⊢ (𝜑 → (1 / 𝐴) ∈ ℝ+) | ||
| Theorem | rprecred 13060 | Closure law for reciprocation of positive reals. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ+) ⇒ ⊢ (𝜑 → (1 / 𝐴) ∈ ℝ) | ||
| Theorem | rphalfcld 13061 | Closure law for half of a positive real. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ+) ⇒ ⊢ (𝜑 → (𝐴 / 2) ∈ ℝ+) | ||
| Theorem | reclt1d 13062 | The reciprocal of a positive number less than 1 is greater than 1. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ+) ⇒ ⊢ (𝜑 → (𝐴 < 1 ↔ 1 < (1 / 𝐴))) | ||
| Theorem | recgt1d 13063 | The reciprocal of a positive number greater than 1 is less than 1. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ+) ⇒ ⊢ (𝜑 → (1 < 𝐴 ↔ (1 / 𝐴) < 1)) | ||
| Theorem | rpaddcld 13064 | Closure law for addition of positive reals. Part of Axiom 7 of [Apostol] p. 20. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ+) & ⊢ (𝜑 → 𝐵 ∈ ℝ+) ⇒ ⊢ (𝜑 → (𝐴 + 𝐵) ∈ ℝ+) | ||
| Theorem | rpmulcld 13065 | Closure law for multiplication of positive reals. Part of Axiom 7 of [Apostol] p. 20. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ+) & ⊢ (𝜑 → 𝐵 ∈ ℝ+) ⇒ ⊢ (𝜑 → (𝐴 · 𝐵) ∈ ℝ+) | ||
| Theorem | rpdivcld 13066 | Closure law for division of positive reals. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ+) & ⊢ (𝜑 → 𝐵 ∈ ℝ+) ⇒ ⊢ (𝜑 → (𝐴 / 𝐵) ∈ ℝ+) | ||
| Theorem | ltrecd 13067 | The reciprocal of both sides of 'less than'. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ+) & ⊢ (𝜑 → 𝐵 ∈ ℝ+) ⇒ ⊢ (𝜑 → (𝐴 < 𝐵 ↔ (1 / 𝐵) < (1 / 𝐴))) | ||
| Theorem | lerecd 13068 | The reciprocal of both sides of 'less than or equal to'. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ+) & ⊢ (𝜑 → 𝐵 ∈ ℝ+) ⇒ ⊢ (𝜑 → (𝐴 ≤ 𝐵 ↔ (1 / 𝐵) ≤ (1 / 𝐴))) | ||
| Theorem | ltrec1d 13069 | Reciprocal swap in a 'less than' relation. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ+) & ⊢ (𝜑 → 𝐵 ∈ ℝ+) & ⊢ (𝜑 → (1 / 𝐴) < 𝐵) ⇒ ⊢ (𝜑 → (1 / 𝐵) < 𝐴) | ||
| Theorem | lerec2d 13070 | Reciprocal swap in a 'less than or equal to' relation. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ+) & ⊢ (𝜑 → 𝐵 ∈ ℝ+) & ⊢ (𝜑 → 𝐴 ≤ (1 / 𝐵)) ⇒ ⊢ (𝜑 → 𝐵 ≤ (1 / 𝐴)) | ||
| Theorem | lediv2ad 13071 | Division of both sides of 'less than or equal to' into a nonnegative number. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ+) & ⊢ (𝜑 → 𝐵 ∈ ℝ+) & ⊢ (𝜑 → 𝐶 ∈ ℝ) & ⊢ (𝜑 → 0 ≤ 𝐶) & ⊢ (𝜑 → 𝐴 ≤ 𝐵) ⇒ ⊢ (𝜑 → (𝐶 / 𝐵) ≤ (𝐶 / 𝐴)) | ||
| Theorem | ltdiv2d 13072 | Division of a positive number by both sides of 'less than'. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ+) & ⊢ (𝜑 → 𝐵 ∈ ℝ+) & ⊢ (𝜑 → 𝐶 ∈ ℝ+) ⇒ ⊢ (𝜑 → (𝐴 < 𝐵 ↔ (𝐶 / 𝐵) < (𝐶 / 𝐴))) | ||
| Theorem | lediv2d 13073 | Division of a positive number by both sides of 'less than or equal to'. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ+) & ⊢ (𝜑 → 𝐵 ∈ ℝ+) & ⊢ (𝜑 → 𝐶 ∈ ℝ+) ⇒ ⊢ (𝜑 → (𝐴 ≤ 𝐵 ↔ (𝐶 / 𝐵) ≤ (𝐶 / 𝐴))) | ||
| Theorem | ledivdivd 13074 | Invert ratios of positive numbers and swap their ordering. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ+) & ⊢ (𝜑 → 𝐵 ∈ ℝ+) & ⊢ (𝜑 → 𝐶 ∈ ℝ+) & ⊢ (𝜑 → 𝐷 ∈ ℝ+) & ⊢ (𝜑 → (𝐴 / 𝐵) ≤ (𝐶 / 𝐷)) ⇒ ⊢ (𝜑 → (𝐷 / 𝐶) ≤ (𝐵 / 𝐴)) | ||
| Theorem | divge1 13075 | The ratio of a number over a smaller positive number is larger than 1. (Contributed by Glauco Siliprandi, 5-Apr-2020.) |
| ⊢ ((𝐴 ∈ ℝ+ ∧ 𝐵 ∈ ℝ ∧ 𝐴 ≤ 𝐵) → 1 ≤ (𝐵 / 𝐴)) | ||
| Theorem | divlt1lt 13076 | A real number divided by a positive real number is less than 1 iff the real number is less than the positive real number. (Contributed by AV, 25-May-2020.) |
| ⊢ ((𝐴 ∈ ℝ ∧ 𝐵 ∈ ℝ+) → ((𝐴 / 𝐵) < 1 ↔ 𝐴 < 𝐵)) | ||
| Theorem | divle1le 13077 | A real number divided by a positive real number is less than or equal to 1 iff the real number is less than or equal to the positive real number. (Contributed by AV, 29-Jun-2021.) |
| ⊢ ((𝐴 ∈ ℝ ∧ 𝐵 ∈ ℝ+) → ((𝐴 / 𝐵) ≤ 1 ↔ 𝐴 ≤ 𝐵)) | ||
| Theorem | ledivge1le 13078 | If a number is less than or equal to another number, the number divided by a positive number greater than or equal to one is less than or equal to the other number. (Contributed by AV, 29-Jun-2021.) |
| ⊢ ((𝐴 ∈ ℝ ∧ 𝐵 ∈ ℝ+ ∧ (𝐶 ∈ ℝ+ ∧ 1 ≤ 𝐶)) → (𝐴 ≤ 𝐵 → (𝐴 / 𝐶) ≤ 𝐵)) | ||
| Theorem | ge0p1rpd 13079 | A nonnegative number plus one is a positive number. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 0 ≤ 𝐴) ⇒ ⊢ (𝜑 → (𝐴 + 1) ∈ ℝ+) | ||
| Theorem | rerpdivcld 13080 | Closure law for division of a real by a positive real. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ+) ⇒ ⊢ (𝜑 → (𝐴 / 𝐵) ∈ ℝ) | ||
| Theorem | ltsubrpd 13081 | Subtracting a positive real from another number decreases it. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ+) ⇒ ⊢ (𝜑 → (𝐴 − 𝐵) < 𝐴) | ||
| Theorem | ltaddrpd 13082 | Adding a positive number to another number increases it. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ+) ⇒ ⊢ (𝜑 → 𝐴 < (𝐴 + 𝐵)) | ||
| Theorem | ltaddrp2d 13083 | Adding a positive number to another number increases it. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ+) ⇒ ⊢ (𝜑 → 𝐴 < (𝐵 + 𝐴)) | ||
| Theorem | ltmulgt11d 13084 | Multiplication by a number greater than 1. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ+) ⇒ ⊢ (𝜑 → (1 < 𝐴 ↔ 𝐵 < (𝐵 · 𝐴))) | ||
| Theorem | ltmulgt12d 13085 | Multiplication by a number greater than 1. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ+) ⇒ ⊢ (𝜑 → (1 < 𝐴 ↔ 𝐵 < (𝐴 · 𝐵))) | ||
| Theorem | gt0divd 13086 | Division of a positive number by a positive number. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ+) ⇒ ⊢ (𝜑 → (0 < 𝐴 ↔ 0 < (𝐴 / 𝐵))) | ||
| Theorem | ge0divd 13087 | Division of a nonnegative number by a positive number. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ+) ⇒ ⊢ (𝜑 → (0 ≤ 𝐴 ↔ 0 ≤ (𝐴 / 𝐵))) | ||
| Theorem | rpgecld 13088 | A number greater than or equal to a positive real is positive real. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ+) & ⊢ (𝜑 → 𝐵 ≤ 𝐴) ⇒ ⊢ (𝜑 → 𝐴 ∈ ℝ+) | ||
| Theorem | divge0d 13089 | The ratio of nonnegative and positive numbers is nonnegative. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ+) & ⊢ (𝜑 → 0 ≤ 𝐴) ⇒ ⊢ (𝜑 → 0 ≤ (𝐴 / 𝐵)) | ||
| Theorem | ltmul1d 13090 | The ratio of nonnegative and positive numbers is nonnegative. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) & ⊢ (𝜑 → 𝐶 ∈ ℝ+) ⇒ ⊢ (𝜑 → (𝐴 < 𝐵 ↔ (𝐴 · 𝐶) < (𝐵 · 𝐶))) | ||
| Theorem | ltmul2d 13091 | Multiplication of both sides of 'less than' by a positive number. Theorem I.19 of [Apostol] p. 20. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) & ⊢ (𝜑 → 𝐶 ∈ ℝ+) ⇒ ⊢ (𝜑 → (𝐴 < 𝐵 ↔ (𝐶 · 𝐴) < (𝐶 · 𝐵))) | ||
| Theorem | lemul1d 13092 | Multiplication of both sides of 'less than or equal to' by a positive number. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) & ⊢ (𝜑 → 𝐶 ∈ ℝ+) ⇒ ⊢ (𝜑 → (𝐴 ≤ 𝐵 ↔ (𝐴 · 𝐶) ≤ (𝐵 · 𝐶))) | ||
| Theorem | lemul2d 13093 | Multiplication of both sides of 'less than or equal to' by a positive number. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) & ⊢ (𝜑 → 𝐶 ∈ ℝ+) ⇒ ⊢ (𝜑 → (𝐴 ≤ 𝐵 ↔ (𝐶 · 𝐴) ≤ (𝐶 · 𝐵))) | ||
| Theorem | ltdiv1d 13094 | Division of both sides of 'less than' by a positive number. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) & ⊢ (𝜑 → 𝐶 ∈ ℝ+) ⇒ ⊢ (𝜑 → (𝐴 < 𝐵 ↔ (𝐴 / 𝐶) < (𝐵 / 𝐶))) | ||
| Theorem | lediv1d 13095 | Division of both sides of a less than or equal to relation by a positive number. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) & ⊢ (𝜑 → 𝐶 ∈ ℝ+) ⇒ ⊢ (𝜑 → (𝐴 ≤ 𝐵 ↔ (𝐴 / 𝐶) ≤ (𝐵 / 𝐶))) | ||
| Theorem | ltmuldivd 13096 | 'Less than' relationship between division and multiplication. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) & ⊢ (𝜑 → 𝐶 ∈ ℝ+) ⇒ ⊢ (𝜑 → ((𝐴 · 𝐶) < 𝐵 ↔ 𝐴 < (𝐵 / 𝐶))) | ||
| Theorem | ltmuldiv2d 13097 | 'Less than' relationship between division and multiplication. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) & ⊢ (𝜑 → 𝐶 ∈ ℝ+) ⇒ ⊢ (𝜑 → ((𝐶 · 𝐴) < 𝐵 ↔ 𝐴 < (𝐵 / 𝐶))) | ||
| Theorem | lemuldivd 13098 | 'Less than or equal to' relationship between division and multiplication. (Contributed by Mario Carneiro, 30-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) & ⊢ (𝜑 → 𝐶 ∈ ℝ+) ⇒ ⊢ (𝜑 → ((𝐴 · 𝐶) ≤ 𝐵 ↔ 𝐴 ≤ (𝐵 / 𝐶))) | ||
| Theorem | lemuldiv2d 13099 | 'Less than or equal to' relationship between division and multiplication. (Contributed by Mario Carneiro, 30-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) & ⊢ (𝜑 → 𝐶 ∈ ℝ+) ⇒ ⊢ (𝜑 → ((𝐶 · 𝐴) ≤ 𝐵 ↔ 𝐴 ≤ (𝐵 / 𝐶))) | ||
| Theorem | ltdivmuld 13100 | 'Less than' relationship between division and multiplication. (Contributed by Mario Carneiro, 28-May-2016.) |
| ⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) & ⊢ (𝜑 → 𝐶 ∈ ℝ+) ⇒ ⊢ (𝜑 → ((𝐴 / 𝐶) < 𝐵 ↔ 𝐴 < (𝐶 · 𝐵))) | ||
| < Previous Next > |
| Copyright terms: Public domain | < Previous Next > |