![]() |
Metamath
Proof Explorer Theorem List (p. 108 of 431) | < 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-28055) |
![]() (28056-29580) |
![]() (29581-43033) |
Type | Label | Description |
---|---|---|
Statement | ||
Theorem | addge01 10701 | A number is less than or equal to itself plus a nonnegative number. (Contributed by NM, 21-Feb-2005.) |
⊢ ((𝐴 ∈ ℝ ∧ 𝐵 ∈ ℝ) → (0 ≤ 𝐵 ↔ 𝐴 ≤ (𝐴 + 𝐵))) | ||
Theorem | addge02 10702 | A number is less than or equal to itself plus a nonnegative number. (Contributed by NM, 27-Jul-2005.) |
⊢ ((𝐴 ∈ ℝ ∧ 𝐵 ∈ ℝ) → (0 ≤ 𝐵 ↔ 𝐴 ≤ (𝐵 + 𝐴))) | ||
Theorem | add20 10703 | Two nonnegative numbers are zero iff their sum is zero. (Contributed by Jeff Madsen, 2-Sep-2009.) (Proof shortened by Mario Carneiro, 27-May-2016.) |
⊢ (((𝐴 ∈ ℝ ∧ 0 ≤ 𝐴) ∧ (𝐵 ∈ ℝ ∧ 0 ≤ 𝐵)) → ((𝐴 + 𝐵) = 0 ↔ (𝐴 = 0 ∧ 𝐵 = 0))) | ||
Theorem | subge0 10704 | Nonnegative subtraction. (Contributed by NM, 14-Mar-2005.) (Proof shortened by Mario Carneiro, 27-May-2016.) |
⊢ ((𝐴 ∈ ℝ ∧ 𝐵 ∈ ℝ) → (0 ≤ (𝐴 − 𝐵) ↔ 𝐵 ≤ 𝐴)) | ||
Theorem | suble0 10705 | Nonpositive subtraction. (Contributed by NM, 20-Mar-2008.) (Proof shortened by Mario Carneiro, 27-May-2016.) |
⊢ ((𝐴 ∈ ℝ ∧ 𝐵 ∈ ℝ) → ((𝐴 − 𝐵) ≤ 0 ↔ 𝐴 ≤ 𝐵)) | ||
Theorem | leaddle0 10706 | The sum of a real number and a second real number is less than the real number iff the second real number is negative. (Contributed by Alexander van der Vekens, 30-May-2018.) |
⊢ ((𝐴 ∈ ℝ ∧ 𝐵 ∈ ℝ) → ((𝐴 + 𝐵) ≤ 𝐴 ↔ 𝐵 ≤ 0)) | ||
Theorem | subge02 10707 | Nonnegative subtraction. (Contributed by NM, 27-Jul-2005.) |
⊢ ((𝐴 ∈ ℝ ∧ 𝐵 ∈ ℝ) → (0 ≤ 𝐵 ↔ (𝐴 − 𝐵) ≤ 𝐴)) | ||
Theorem | lesub0 10708 | Lemma to show a nonnegative number is zero. (Contributed by NM, 8-Oct-1999.) (Proof shortened by Mario Carneiro, 27-May-2016.) |
⊢ ((𝐴 ∈ ℝ ∧ 𝐵 ∈ ℝ) → ((0 ≤ 𝐴 ∧ 𝐵 ≤ (𝐵 − 𝐴)) ↔ 𝐴 = 0)) | ||
Theorem | mulge0 10709 | The product of two nonnegative numbers is nonnegative. (Contributed by NM, 8-Oct-1999.) (Revised by Mario Carneiro, 27-May-2016.) |
⊢ (((𝐴 ∈ ℝ ∧ 0 ≤ 𝐴) ∧ (𝐵 ∈ ℝ ∧ 0 ≤ 𝐵)) → 0 ≤ (𝐴 · 𝐵)) | ||
Theorem | mullt0 10710 | The product of two negative numbers is positive. (Contributed by Jeff Hankins, 8-Jun-2009.) |
⊢ (((𝐴 ∈ ℝ ∧ 𝐴 < 0) ∧ (𝐵 ∈ ℝ ∧ 𝐵 < 0)) → 0 < (𝐴 · 𝐵)) | ||
Theorem | msqgt0 10711 | A nonzero square is positive. Theorem I.20 of [Apostol] p. 20. (Contributed by NM, 6-May-1999.) (Proof shortened by Mario Carneiro, 27-May-2016.) |
⊢ ((𝐴 ∈ ℝ ∧ 𝐴 ≠ 0) → 0 < (𝐴 · 𝐴)) | ||
Theorem | msqge0 10712 | A square is nonnegative. (Contributed by NM, 23-May-2007.) (Revised by Mario Carneiro, 27-May-2016.) |
⊢ (𝐴 ∈ ℝ → 0 ≤ (𝐴 · 𝐴)) | ||
Theorem | 0lt1 10713 | 0 is less than 1. Theorem I.21 of [Apostol] p. 20. (Contributed by NM, 17-Jan-1997.) |
⊢ 0 < 1 | ||
Theorem | 0le1 10714 | 0 is less than or equal to 1. (Contributed by Mario Carneiro, 29-Apr-2015.) |
⊢ 0 ≤ 1 | ||
Theorem | relin01 10715 | An interval law for less than or equal. (Contributed by Scott Fenton, 27-Jun-2013.) |
⊢ (𝐴 ∈ ℝ → (𝐴 ≤ 0 ∨ (0 ≤ 𝐴 ∧ 𝐴 ≤ 1) ∨ 1 ≤ 𝐴)) | ||
Theorem | ltordlem 10716* | Lemma for ltord1 10717. (Contributed by Mario Carneiro, 14-Jun-2014.) |
⊢ (𝑥 = 𝑦 → 𝐴 = 𝐵) & ⊢ (𝑥 = 𝐶 → 𝐴 = 𝑀) & ⊢ (𝑥 = 𝐷 → 𝐴 = 𝑁) & ⊢ 𝑆 ⊆ ℝ & ⊢ ((𝜑 ∧ 𝑥 ∈ 𝑆) → 𝐴 ∈ ℝ) & ⊢ ((𝜑 ∧ (𝑥 ∈ 𝑆 ∧ 𝑦 ∈ 𝑆)) → (𝑥 < 𝑦 → 𝐴 < 𝐵)) ⇒ ⊢ ((𝜑 ∧ (𝐶 ∈ 𝑆 ∧ 𝐷 ∈ 𝑆)) → (𝐶 < 𝐷 → 𝑀 < 𝑁)) | ||
Theorem | ltord1 10717* | Infer an ordering relation from a proof in only one direction. (Contributed by Mario Carneiro, 14-Jun-2014.) |
⊢ (𝑥 = 𝑦 → 𝐴 = 𝐵) & ⊢ (𝑥 = 𝐶 → 𝐴 = 𝑀) & ⊢ (𝑥 = 𝐷 → 𝐴 = 𝑁) & ⊢ 𝑆 ⊆ ℝ & ⊢ ((𝜑 ∧ 𝑥 ∈ 𝑆) → 𝐴 ∈ ℝ) & ⊢ ((𝜑 ∧ (𝑥 ∈ 𝑆 ∧ 𝑦 ∈ 𝑆)) → (𝑥 < 𝑦 → 𝐴 < 𝐵)) ⇒ ⊢ ((𝜑 ∧ (𝐶 ∈ 𝑆 ∧ 𝐷 ∈ 𝑆)) → (𝐶 < 𝐷 ↔ 𝑀 < 𝑁)) | ||
Theorem | leord1 10718* | Infer an ordering relation from a proof in only one direction. (Contributed by Mario Carneiro, 14-Jun-2014.) |
⊢ (𝑥 = 𝑦 → 𝐴 = 𝐵) & ⊢ (𝑥 = 𝐶 → 𝐴 = 𝑀) & ⊢ (𝑥 = 𝐷 → 𝐴 = 𝑁) & ⊢ 𝑆 ⊆ ℝ & ⊢ ((𝜑 ∧ 𝑥 ∈ 𝑆) → 𝐴 ∈ ℝ) & ⊢ ((𝜑 ∧ (𝑥 ∈ 𝑆 ∧ 𝑦 ∈ 𝑆)) → (𝑥 < 𝑦 → 𝐴 < 𝐵)) ⇒ ⊢ ((𝜑 ∧ (𝐶 ∈ 𝑆 ∧ 𝐷 ∈ 𝑆)) → (𝐶 ≤ 𝐷 ↔ 𝑀 ≤ 𝑁)) | ||
Theorem | eqord1 10719* | Infer an ordering relation from a proof in only one direction. (Contributed by Mario Carneiro, 14-Jun-2014.) |
⊢ (𝑥 = 𝑦 → 𝐴 = 𝐵) & ⊢ (𝑥 = 𝐶 → 𝐴 = 𝑀) & ⊢ (𝑥 = 𝐷 → 𝐴 = 𝑁) & ⊢ 𝑆 ⊆ ℝ & ⊢ ((𝜑 ∧ 𝑥 ∈ 𝑆) → 𝐴 ∈ ℝ) & ⊢ ((𝜑 ∧ (𝑥 ∈ 𝑆 ∧ 𝑦 ∈ 𝑆)) → (𝑥 < 𝑦 → 𝐴 < 𝐵)) ⇒ ⊢ ((𝜑 ∧ (𝐶 ∈ 𝑆 ∧ 𝐷 ∈ 𝑆)) → (𝐶 = 𝐷 ↔ 𝑀 = 𝑁)) | ||
Theorem | ltord2 10720* | Infer an ordering relation from a proof in only one direction. (Contributed by Mario Carneiro, 14-Jun-2014.) |
⊢ (𝑥 = 𝑦 → 𝐴 = 𝐵) & ⊢ (𝑥 = 𝐶 → 𝐴 = 𝑀) & ⊢ (𝑥 = 𝐷 → 𝐴 = 𝑁) & ⊢ 𝑆 ⊆ ℝ & ⊢ ((𝜑 ∧ 𝑥 ∈ 𝑆) → 𝐴 ∈ ℝ) & ⊢ ((𝜑 ∧ (𝑥 ∈ 𝑆 ∧ 𝑦 ∈ 𝑆)) → (𝑥 < 𝑦 → 𝐵 < 𝐴)) ⇒ ⊢ ((𝜑 ∧ (𝐶 ∈ 𝑆 ∧ 𝐷 ∈ 𝑆)) → (𝐶 < 𝐷 ↔ 𝑁 < 𝑀)) | ||
Theorem | leord2 10721* | Infer an ordering relation from a proof in only one direction. (Contributed by Mario Carneiro, 14-Jun-2014.) |
⊢ (𝑥 = 𝑦 → 𝐴 = 𝐵) & ⊢ (𝑥 = 𝐶 → 𝐴 = 𝑀) & ⊢ (𝑥 = 𝐷 → 𝐴 = 𝑁) & ⊢ 𝑆 ⊆ ℝ & ⊢ ((𝜑 ∧ 𝑥 ∈ 𝑆) → 𝐴 ∈ ℝ) & ⊢ ((𝜑 ∧ (𝑥 ∈ 𝑆 ∧ 𝑦 ∈ 𝑆)) → (𝑥 < 𝑦 → 𝐵 < 𝐴)) ⇒ ⊢ ((𝜑 ∧ (𝐶 ∈ 𝑆 ∧ 𝐷 ∈ 𝑆)) → (𝐶 ≤ 𝐷 ↔ 𝑁 ≤ 𝑀)) | ||
Theorem | eqord2 10722* | Infer an ordering relation from a proof in only one direction. (Contributed by Mario Carneiro, 14-Jun-2014.) |
⊢ (𝑥 = 𝑦 → 𝐴 = 𝐵) & ⊢ (𝑥 = 𝐶 → 𝐴 = 𝑀) & ⊢ (𝑥 = 𝐷 → 𝐴 = 𝑁) & ⊢ 𝑆 ⊆ ℝ & ⊢ ((𝜑 ∧ 𝑥 ∈ 𝑆) → 𝐴 ∈ ℝ) & ⊢ ((𝜑 ∧ (𝑥 ∈ 𝑆 ∧ 𝑦 ∈ 𝑆)) → (𝑥 < 𝑦 → 𝐵 < 𝐴)) ⇒ ⊢ ((𝜑 ∧ (𝐶 ∈ 𝑆 ∧ 𝐷 ∈ 𝑆)) → (𝐶 = 𝐷 ↔ 𝑀 = 𝑁)) | ||
Theorem | wloglei 10723* | Form of wlogle 10724 where both sides of the equivalence are proven rather than showing that they are equivalent to each other. (Contributed by Mario Carneiro, 9-Mar-2015.) |
⊢ ((𝑧 = 𝑥 ∧ 𝑤 = 𝑦) → (𝜓 ↔ 𝜒)) & ⊢ ((𝑧 = 𝑦 ∧ 𝑤 = 𝑥) → (𝜓 ↔ 𝜃)) & ⊢ (𝜑 → 𝑆 ⊆ ℝ) & ⊢ ((𝜑 ∧ (𝑥 ∈ 𝑆 ∧ 𝑦 ∈ 𝑆 ∧ 𝑥 ≤ 𝑦)) → 𝜃) & ⊢ ((𝜑 ∧ (𝑥 ∈ 𝑆 ∧ 𝑦 ∈ 𝑆 ∧ 𝑥 ≤ 𝑦)) → 𝜒) ⇒ ⊢ ((𝜑 ∧ (𝑥 ∈ 𝑆 ∧ 𝑦 ∈ 𝑆)) → 𝜒) | ||
Theorem | wlogle 10724* | If the predicate 𝜒(𝑥, 𝑦) is symmetric under interchange of 𝑥, 𝑦, then "without loss of generality" we can assume that 𝑥 ≤ 𝑦. (Contributed by Mario Carneiro, 18-Aug-2014.) (Revised by Mario Carneiro, 11-Sep-2014.) |
⊢ ((𝑧 = 𝑥 ∧ 𝑤 = 𝑦) → (𝜓 ↔ 𝜒)) & ⊢ ((𝑧 = 𝑦 ∧ 𝑤 = 𝑥) → (𝜓 ↔ 𝜃)) & ⊢ (𝜑 → 𝑆 ⊆ ℝ) & ⊢ ((𝜑 ∧ (𝑥 ∈ 𝑆 ∧ 𝑦 ∈ 𝑆)) → (𝜒 ↔ 𝜃)) & ⊢ ((𝜑 ∧ (𝑥 ∈ 𝑆 ∧ 𝑦 ∈ 𝑆 ∧ 𝑥 ≤ 𝑦)) → 𝜒) ⇒ ⊢ ((𝜑 ∧ (𝑥 ∈ 𝑆 ∧ 𝑦 ∈ 𝑆)) → 𝜒) | ||
Theorem | leidi 10725 | 'Less than or equal to' is reflexive. (Contributed by NM, 18-Aug-1999.) |
⊢ 𝐴 ∈ ℝ ⇒ ⊢ 𝐴 ≤ 𝐴 | ||
Theorem | gt0ne0i 10726 | Positive means nonzero (useful for ordering theorems involving division). (Contributed by NM, 16-Sep-1999.) |
⊢ 𝐴 ∈ ℝ ⇒ ⊢ (0 < 𝐴 → 𝐴 ≠ 0) | ||
Theorem | gt0ne0ii 10727 | Positive implies nonzero. (Contributed by NM, 15-May-1999.) |
⊢ 𝐴 ∈ ℝ & ⊢ 0 < 𝐴 ⇒ ⊢ 𝐴 ≠ 0 | ||
Theorem | msqgt0i 10728 | A nonzero square is positive. Theorem I.20 of [Apostol] p. 20. (Contributed by NM, 17-Jan-1997.) (Revised by Mario Carneiro, 27-May-2016.) |
⊢ 𝐴 ∈ ℝ ⇒ ⊢ (𝐴 ≠ 0 → 0 < (𝐴 · 𝐴)) | ||
Theorem | msqge0i 10729 | A square is nonnegative. (Contributed by NM, 14-May-1999.) (Proof shortened by Andrew Salmon, 19-Nov-2011.) |
⊢ 𝐴 ∈ ℝ ⇒ ⊢ 0 ≤ (𝐴 · 𝐴) | ||
Theorem | addgt0i 10730 | Addition of 2 positive numbers is positive. (Contributed by NM, 16-May-1999.) (Proof shortened by Andrew Salmon, 19-Nov-2011.) |
⊢ 𝐴 ∈ ℝ & ⊢ 𝐵 ∈ ℝ ⇒ ⊢ ((0 < 𝐴 ∧ 0 < 𝐵) → 0 < (𝐴 + 𝐵)) | ||
Theorem | addge0i 10731 | Addition of 2 nonnegative numbers is nonnegative. (Contributed by NM, 28-May-1999.) (Proof shortened by Andrew Salmon, 19-Nov-2011.) |
⊢ 𝐴 ∈ ℝ & ⊢ 𝐵 ∈ ℝ ⇒ ⊢ ((0 ≤ 𝐴 ∧ 0 ≤ 𝐵) → 0 ≤ (𝐴 + 𝐵)) | ||
Theorem | addgegt0i 10732 | Addition of nonnegative and positive numbers is positive. (Contributed by NM, 25-Sep-1999.) (Revised by Mario Carneiro, 27-May-2016.) |
⊢ 𝐴 ∈ ℝ & ⊢ 𝐵 ∈ ℝ ⇒ ⊢ ((0 ≤ 𝐴 ∧ 0 < 𝐵) → 0 < (𝐴 + 𝐵)) | ||
Theorem | addgt0ii 10733 | Addition of 2 positive numbers is positive. (Contributed by NM, 18-May-1999.) |
⊢ 𝐴 ∈ ℝ & ⊢ 𝐵 ∈ ℝ & ⊢ 0 < 𝐴 & ⊢ 0 < 𝐵 ⇒ ⊢ 0 < (𝐴 + 𝐵) | ||
Theorem | add20i 10734 | Two nonnegative numbers are zero iff their sum is zero. (Contributed by NM, 28-Jul-1999.) |
⊢ 𝐴 ∈ ℝ & ⊢ 𝐵 ∈ ℝ ⇒ ⊢ ((0 ≤ 𝐴 ∧ 0 ≤ 𝐵) → ((𝐴 + 𝐵) = 0 ↔ (𝐴 = 0 ∧ 𝐵 = 0))) | ||
Theorem | ltnegi 10735 | Negative of both sides of 'less than'. Theorem I.23 of [Apostol] p. 20. (Contributed by NM, 21-Jan-1997.) |
⊢ 𝐴 ∈ ℝ & ⊢ 𝐵 ∈ ℝ ⇒ ⊢ (𝐴 < 𝐵 ↔ -𝐵 < -𝐴) | ||
Theorem | lenegi 10736 | Negative of both sides of 'less than or equal to'. (Contributed by NM, 1-Aug-1999.) |
⊢ 𝐴 ∈ ℝ & ⊢ 𝐵 ∈ ℝ ⇒ ⊢ (𝐴 ≤ 𝐵 ↔ -𝐵 ≤ -𝐴) | ||
Theorem | ltnegcon2i 10737 | Contraposition of negative in 'less than'. (Contributed by NM, 14-May-1999.) |
⊢ 𝐴 ∈ ℝ & ⊢ 𝐵 ∈ ℝ ⇒ ⊢ (𝐴 < -𝐵 ↔ 𝐵 < -𝐴) | ||
Theorem | mulge0i 10738 | The product of two nonnegative numbers is nonnegative. (Contributed by NM, 30-Jul-1999.) |
⊢ 𝐴 ∈ ℝ & ⊢ 𝐵 ∈ ℝ ⇒ ⊢ ((0 ≤ 𝐴 ∧ 0 ≤ 𝐵) → 0 ≤ (𝐴 · 𝐵)) | ||
Theorem | lesub0i 10739 | Lemma to show a nonnegative number is zero. (Contributed by NM, 8-Oct-1999.) (Proof shortened by Andrew Salmon, 19-Nov-2011.) |
⊢ 𝐴 ∈ ℝ & ⊢ 𝐵 ∈ ℝ ⇒ ⊢ ((0 ≤ 𝐴 ∧ 𝐵 ≤ (𝐵 − 𝐴)) ↔ 𝐴 = 0) | ||
Theorem | ltaddposi 10740 | Adding a positive number to another number increases it. (Contributed by NM, 25-Aug-1999.) |
⊢ 𝐴 ∈ ℝ & ⊢ 𝐵 ∈ ℝ ⇒ ⊢ (0 < 𝐴 ↔ 𝐵 < (𝐵 + 𝐴)) | ||
Theorem | posdifi 10741 | Comparison of two numbers whose difference is positive. (Contributed by NM, 19-Aug-2001.) |
⊢ 𝐴 ∈ ℝ & ⊢ 𝐵 ∈ ℝ ⇒ ⊢ (𝐴 < 𝐵 ↔ 0 < (𝐵 − 𝐴)) | ||
Theorem | ltnegcon1i 10742 | Contraposition of negative in 'less than'. (Contributed by NM, 14-May-1999.) |
⊢ 𝐴 ∈ ℝ & ⊢ 𝐵 ∈ ℝ ⇒ ⊢ (-𝐴 < 𝐵 ↔ -𝐵 < 𝐴) | ||
Theorem | lenegcon1i 10743 | Contraposition of negative in 'less than or equal to'. (Contributed by NM, 6-Apr-2005.) |
⊢ 𝐴 ∈ ℝ & ⊢ 𝐵 ∈ ℝ ⇒ ⊢ (-𝐴 ≤ 𝐵 ↔ -𝐵 ≤ 𝐴) | ||
Theorem | subge0i 10744 | Nonnegative subtraction. (Contributed by NM, 13-Aug-2000.) |
⊢ 𝐴 ∈ ℝ & ⊢ 𝐵 ∈ ℝ ⇒ ⊢ (0 ≤ (𝐴 − 𝐵) ↔ 𝐵 ≤ 𝐴) | ||
Theorem | ltadd1i 10745 | Addition to both sides of 'less than'. Theorem I.18 of [Apostol] p. 20. (Contributed by NM, 21-Jan-1997.) |
⊢ 𝐴 ∈ ℝ & ⊢ 𝐵 ∈ ℝ & ⊢ 𝐶 ∈ ℝ ⇒ ⊢ (𝐴 < 𝐵 ↔ (𝐴 + 𝐶) < (𝐵 + 𝐶)) | ||
Theorem | leadd1i 10746 | Addition to both sides of 'less than or equal to'. (Contributed by NM, 11-Aug-1999.) |
⊢ 𝐴 ∈ ℝ & ⊢ 𝐵 ∈ ℝ & ⊢ 𝐶 ∈ ℝ ⇒ ⊢ (𝐴 ≤ 𝐵 ↔ (𝐴 + 𝐶) ≤ (𝐵 + 𝐶)) | ||
Theorem | leadd2i 10747 | Addition to both sides of 'less than or equal to'. (Contributed by NM, 11-Aug-1999.) |
⊢ 𝐴 ∈ ℝ & ⊢ 𝐵 ∈ ℝ & ⊢ 𝐶 ∈ ℝ ⇒ ⊢ (𝐴 ≤ 𝐵 ↔ (𝐶 + 𝐴) ≤ (𝐶 + 𝐵)) | ||
Theorem | ltsubaddi 10748 | 'Less than' relationship between subtraction and addition. (Contributed by NM, 21-Jan-1997.) (Proof shortened by Andrew Salmon, 19-Nov-2011.) |
⊢ 𝐴 ∈ ℝ & ⊢ 𝐵 ∈ ℝ & ⊢ 𝐶 ∈ ℝ ⇒ ⊢ ((𝐴 − 𝐵) < 𝐶 ↔ 𝐴 < (𝐶 + 𝐵)) | ||
Theorem | lesubaddi 10749 | 'Less than or equal to' relationship between subtraction and addition. (Contributed by NM, 30-Sep-1999.) (Proof shortened by Andrew Salmon, 19-Nov-2011.) |
⊢ 𝐴 ∈ ℝ & ⊢ 𝐵 ∈ ℝ & ⊢ 𝐶 ∈ ℝ ⇒ ⊢ ((𝐴 − 𝐵) ≤ 𝐶 ↔ 𝐴 ≤ (𝐶 + 𝐵)) | ||
Theorem | ltsubadd2i 10750 | 'Less than' relationship between subtraction and addition. (Contributed by NM, 21-Jan-1997.) |
⊢ 𝐴 ∈ ℝ & ⊢ 𝐵 ∈ ℝ & ⊢ 𝐶 ∈ ℝ ⇒ ⊢ ((𝐴 − 𝐵) < 𝐶 ↔ 𝐴 < (𝐵 + 𝐶)) | ||
Theorem | lesubadd2i 10751 | 'Less than or equal to' relationship between subtraction and addition. (Contributed by NM, 3-Aug-1999.) |
⊢ 𝐴 ∈ ℝ & ⊢ 𝐵 ∈ ℝ & ⊢ 𝐶 ∈ ℝ ⇒ ⊢ ((𝐴 − 𝐵) ≤ 𝐶 ↔ 𝐴 ≤ (𝐵 + 𝐶)) | ||
Theorem | ltaddsubi 10752 | 'Less than' relationship between subtraction and addition. (Contributed by NM, 14-May-1999.) |
⊢ 𝐴 ∈ ℝ & ⊢ 𝐵 ∈ ℝ & ⊢ 𝐶 ∈ ℝ ⇒ ⊢ ((𝐴 + 𝐵) < 𝐶 ↔ 𝐴 < (𝐶 − 𝐵)) | ||
Theorem | lt2addi 10753 | Adding both side of two inequalities. Theorem I.25 of [Apostol] p. 20. (Contributed by NM, 14-May-1999.) |
⊢ 𝐴 ∈ ℝ & ⊢ 𝐵 ∈ ℝ & ⊢ 𝐶 ∈ ℝ & ⊢ 𝐷 ∈ ℝ ⇒ ⊢ ((𝐴 < 𝐶 ∧ 𝐵 < 𝐷) → (𝐴 + 𝐵) < (𝐶 + 𝐷)) | ||
Theorem | le2addi 10754 | Adding both side of two inequalities. (Contributed by NM, 16-Sep-1999.) |
⊢ 𝐴 ∈ ℝ & ⊢ 𝐵 ∈ ℝ & ⊢ 𝐶 ∈ ℝ & ⊢ 𝐷 ∈ ℝ ⇒ ⊢ ((𝐴 ≤ 𝐶 ∧ 𝐵 ≤ 𝐷) → (𝐴 + 𝐵) ≤ (𝐶 + 𝐷)) | ||
Theorem | gt0ne0d 10755 | Positive implies nonzero. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 0 < 𝐴) ⇒ ⊢ (𝜑 → 𝐴 ≠ 0) | ||
Theorem | lt0ne0d 10756 | Something less than zero is not zero. Deduction form. (Contributed by David Moews, 28-Feb-2017.) |
⊢ (𝜑 → 𝐴 < 0) ⇒ ⊢ (𝜑 → 𝐴 ≠ 0) | ||
Theorem | leidd 10757 | 'Less than or equal to' is reflexive. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) ⇒ ⊢ (𝜑 → 𝐴 ≤ 𝐴) | ||
Theorem | msqgt0d 10758 | A nonzero square is positive. Theorem I.20 of [Apostol] p. 20. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐴 ≠ 0) ⇒ ⊢ (𝜑 → 0 < (𝐴 · 𝐴)) | ||
Theorem | msqge0d 10759 | A square is nonnegative. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) ⇒ ⊢ (𝜑 → 0 ≤ (𝐴 · 𝐴)) | ||
Theorem | lt0neg1d 10760 | Comparison of a number and its negative to zero. Theorem I.23 of [Apostol] p. 20. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) ⇒ ⊢ (𝜑 → (𝐴 < 0 ↔ 0 < -𝐴)) | ||
Theorem | lt0neg2d 10761 | Comparison of a number and its negative to zero. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) ⇒ ⊢ (𝜑 → (0 < 𝐴 ↔ -𝐴 < 0)) | ||
Theorem | le0neg1d 10762 | Comparison of a number and its negative to zero. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) ⇒ ⊢ (𝜑 → (𝐴 ≤ 0 ↔ 0 ≤ -𝐴)) | ||
Theorem | le0neg2d 10763 | Comparison of a number and its negative to zero. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) ⇒ ⊢ (𝜑 → (0 ≤ 𝐴 ↔ -𝐴 ≤ 0)) | ||
Theorem | addgegt0d 10764 | Addition of nonnegative and positive numbers is positive. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) & ⊢ (𝜑 → 0 ≤ 𝐴) & ⊢ (𝜑 → 0 < 𝐵) ⇒ ⊢ (𝜑 → 0 < (𝐴 + 𝐵)) | ||
Theorem | addgt0d 10765 | Addition of 2 positive numbers is positive. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) & ⊢ (𝜑 → 0 < 𝐴) & ⊢ (𝜑 → 0 < 𝐵) ⇒ ⊢ (𝜑 → 0 < (𝐴 + 𝐵)) | ||
Theorem | addge0d 10766 | Addition of 2 nonnegative numbers is nonnegative. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) & ⊢ (𝜑 → 0 ≤ 𝐴) & ⊢ (𝜑 → 0 ≤ 𝐵) ⇒ ⊢ (𝜑 → 0 ≤ (𝐴 + 𝐵)) | ||
Theorem | mulge0d 10767 | The product of two nonnegative numbers is nonnegative. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) & ⊢ (𝜑 → 0 ≤ 𝐴) & ⊢ (𝜑 → 0 ≤ 𝐵) ⇒ ⊢ (𝜑 → 0 ≤ (𝐴 · 𝐵)) | ||
Theorem | ltnegd 10768 | Negative of both sides of 'less than'. Theorem I.23 of [Apostol] p. 20. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) ⇒ ⊢ (𝜑 → (𝐴 < 𝐵 ↔ -𝐵 < -𝐴)) | ||
Theorem | lenegd 10769 | Negative of both sides of 'less than or equal to'. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) ⇒ ⊢ (𝜑 → (𝐴 ≤ 𝐵 ↔ -𝐵 ≤ -𝐴)) | ||
Theorem | ltnegcon1d 10770 | Contraposition of negative in 'less than'. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) & ⊢ (𝜑 → -𝐴 < 𝐵) ⇒ ⊢ (𝜑 → -𝐵 < 𝐴) | ||
Theorem | ltnegcon2d 10771 | Contraposition of negative in 'less than'. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) & ⊢ (𝜑 → 𝐴 < -𝐵) ⇒ ⊢ (𝜑 → 𝐵 < -𝐴) | ||
Theorem | lenegcon1d 10772 | Contraposition of negative in 'less than or equal to'. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) & ⊢ (𝜑 → -𝐴 ≤ 𝐵) ⇒ ⊢ (𝜑 → -𝐵 ≤ 𝐴) | ||
Theorem | lenegcon2d 10773 | Contraposition of negative in 'less than or equal to'. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) & ⊢ (𝜑 → 𝐴 ≤ -𝐵) ⇒ ⊢ (𝜑 → 𝐵 ≤ -𝐴) | ||
Theorem | ltaddposd 10774 | Adding a positive number to another number increases it. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) ⇒ ⊢ (𝜑 → (0 < 𝐴 ↔ 𝐵 < (𝐵 + 𝐴))) | ||
Theorem | ltaddpos2d 10775 | Adding a positive number to another number increases it. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) ⇒ ⊢ (𝜑 → (0 < 𝐴 ↔ 𝐵 < (𝐴 + 𝐵))) | ||
Theorem | ltsubposd 10776 | Subtracting a positive number from another number decreases it. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) ⇒ ⊢ (𝜑 → (0 < 𝐴 ↔ (𝐵 − 𝐴) < 𝐵)) | ||
Theorem | posdifd 10777 | Comparison of two numbers whose difference is positive. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) ⇒ ⊢ (𝜑 → (𝐴 < 𝐵 ↔ 0 < (𝐵 − 𝐴))) | ||
Theorem | addge01d 10778 | A number is less than or equal to itself plus a nonnegative number. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) ⇒ ⊢ (𝜑 → (0 ≤ 𝐵 ↔ 𝐴 ≤ (𝐴 + 𝐵))) | ||
Theorem | addge02d 10779 | A number is less than or equal to itself plus a nonnegative number. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) ⇒ ⊢ (𝜑 → (0 ≤ 𝐵 ↔ 𝐴 ≤ (𝐵 + 𝐴))) | ||
Theorem | subge0d 10780 | Nonnegative subtraction. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) ⇒ ⊢ (𝜑 → (0 ≤ (𝐴 − 𝐵) ↔ 𝐵 ≤ 𝐴)) | ||
Theorem | suble0d 10781 | Nonpositive subtraction. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) ⇒ ⊢ (𝜑 → ((𝐴 − 𝐵) ≤ 0 ↔ 𝐴 ≤ 𝐵)) | ||
Theorem | subge02d 10782 | Nonnegative subtraction. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) ⇒ ⊢ (𝜑 → (0 ≤ 𝐵 ↔ (𝐴 − 𝐵) ≤ 𝐴)) | ||
Theorem | ltadd1d 10783 | Addition to both sides of 'less than'. Theorem I.18 of [Apostol] p. 20. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) & ⊢ (𝜑 → 𝐶 ∈ ℝ) ⇒ ⊢ (𝜑 → (𝐴 < 𝐵 ↔ (𝐴 + 𝐶) < (𝐵 + 𝐶))) | ||
Theorem | leadd1d 10784 | Addition to both sides of 'less than or equal to'. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) & ⊢ (𝜑 → 𝐶 ∈ ℝ) ⇒ ⊢ (𝜑 → (𝐴 ≤ 𝐵 ↔ (𝐴 + 𝐶) ≤ (𝐵 + 𝐶))) | ||
Theorem | leadd2d 10785 | Addition to both sides of 'less than or equal to'. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) & ⊢ (𝜑 → 𝐶 ∈ ℝ) ⇒ ⊢ (𝜑 → (𝐴 ≤ 𝐵 ↔ (𝐶 + 𝐴) ≤ (𝐶 + 𝐵))) | ||
Theorem | ltsubaddd 10786 | 'Less than' relationship between subtraction and addition. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) & ⊢ (𝜑 → 𝐶 ∈ ℝ) ⇒ ⊢ (𝜑 → ((𝐴 − 𝐵) < 𝐶 ↔ 𝐴 < (𝐶 + 𝐵))) | ||
Theorem | lesubaddd 10787 | 'Less than or equal to' relationship between subtraction and addition. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) & ⊢ (𝜑 → 𝐶 ∈ ℝ) ⇒ ⊢ (𝜑 → ((𝐴 − 𝐵) ≤ 𝐶 ↔ 𝐴 ≤ (𝐶 + 𝐵))) | ||
Theorem | ltsubadd2d 10788 | 'Less than' relationship between subtraction and addition. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) & ⊢ (𝜑 → 𝐶 ∈ ℝ) ⇒ ⊢ (𝜑 → ((𝐴 − 𝐵) < 𝐶 ↔ 𝐴 < (𝐵 + 𝐶))) | ||
Theorem | lesubadd2d 10789 | 'Less than or equal to' relationship between subtraction and addition. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) & ⊢ (𝜑 → 𝐶 ∈ ℝ) ⇒ ⊢ (𝜑 → ((𝐴 − 𝐵) ≤ 𝐶 ↔ 𝐴 ≤ (𝐵 + 𝐶))) | ||
Theorem | ltaddsubd 10790 | 'Less than' relationship between subtraction and addition. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) & ⊢ (𝜑 → 𝐶 ∈ ℝ) ⇒ ⊢ (𝜑 → ((𝐴 + 𝐵) < 𝐶 ↔ 𝐴 < (𝐶 − 𝐵))) | ||
Theorem | ltaddsub2d 10791 | 'Less than' relationship between subtraction and addition. (Contributed by Mario Carneiro, 29-Dec-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) & ⊢ (𝜑 → 𝐶 ∈ ℝ) ⇒ ⊢ (𝜑 → ((𝐴 + 𝐵) < 𝐶 ↔ 𝐵 < (𝐶 − 𝐴))) | ||
Theorem | leaddsub2d 10792 | 'Less than or equal to' relationship between and addition and subtraction. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) & ⊢ (𝜑 → 𝐶 ∈ ℝ) ⇒ ⊢ (𝜑 → ((𝐴 + 𝐵) ≤ 𝐶 ↔ 𝐵 ≤ (𝐶 − 𝐴))) | ||
Theorem | subled 10793 | Swap subtrahends in an inequality. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) & ⊢ (𝜑 → 𝐶 ∈ ℝ) & ⊢ (𝜑 → (𝐴 − 𝐵) ≤ 𝐶) ⇒ ⊢ (𝜑 → (𝐴 − 𝐶) ≤ 𝐵) | ||
Theorem | lesubd 10794 | Swap subtrahends in an inequality. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) & ⊢ (𝜑 → 𝐶 ∈ ℝ) & ⊢ (𝜑 → 𝐴 ≤ (𝐵 − 𝐶)) ⇒ ⊢ (𝜑 → 𝐶 ≤ (𝐵 − 𝐴)) | ||
Theorem | ltsub23d 10795 | 'Less than' relationship between subtraction and addition. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) & ⊢ (𝜑 → 𝐶 ∈ ℝ) & ⊢ (𝜑 → (𝐴 − 𝐵) < 𝐶) ⇒ ⊢ (𝜑 → (𝐴 − 𝐶) < 𝐵) | ||
Theorem | ltsub13d 10796 | 'Less than' relationship between subtraction and addition. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) & ⊢ (𝜑 → 𝐶 ∈ ℝ) & ⊢ (𝜑 → 𝐴 < (𝐵 − 𝐶)) ⇒ ⊢ (𝜑 → 𝐶 < (𝐵 − 𝐴)) | ||
Theorem | lesub1d 10797 | Subtraction from both sides of 'less than or equal to'. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) & ⊢ (𝜑 → 𝐶 ∈ ℝ) ⇒ ⊢ (𝜑 → (𝐴 ≤ 𝐵 ↔ (𝐴 − 𝐶) ≤ (𝐵 − 𝐶))) | ||
Theorem | lesub2d 10798 | Subtraction of both sides of 'less than or equal to'. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) & ⊢ (𝜑 → 𝐶 ∈ ℝ) ⇒ ⊢ (𝜑 → (𝐴 ≤ 𝐵 ↔ (𝐶 − 𝐵) ≤ (𝐶 − 𝐴))) | ||
Theorem | ltsub1d 10799 | Subtraction from both sides of 'less than'. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) & ⊢ (𝜑 → 𝐶 ∈ ℝ) ⇒ ⊢ (𝜑 → (𝐴 < 𝐵 ↔ (𝐴 − 𝐶) < (𝐵 − 𝐶))) | ||
Theorem | ltsub2d 10800 | Subtraction of both sides of 'less than'. (Contributed by Mario Carneiro, 27-May-2016.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) & ⊢ (𝜑 → 𝐶 ∈ ℝ) ⇒ ⊢ (𝜑 → (𝐴 < 𝐵 ↔ (𝐶 − 𝐵) < (𝐶 − 𝐴))) |
< Previous Next > |
Copyright terms: Public domain | < Previous Next > |