| Metamath
Proof Explorer Theorem List (p. 120 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 | reccl 11901 | Closure law for reciprocal. (Contributed by NM, 30-Apr-2005.) |
| ⊢ ((𝐴 ∈ ℂ ∧ 𝐴 ≠ 0) → (1 / 𝐴) ∈ ℂ) | ||
| Theorem | divcan2 11902 | A cancellation law for division. (Contributed by NM, 3-Feb-2004.) (Revised by Mario Carneiro, 27-May-2016.) |
| ⊢ ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ ∧ 𝐵 ≠ 0) → (𝐵 · (𝐴 / 𝐵)) = 𝐴) | ||
| Theorem | divcan1 11903 | A cancellation law for division. (Contributed by NM, 5-Jun-2004.) (Revised by Mario Carneiro, 27-May-2016.) |
| ⊢ ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ ∧ 𝐵 ≠ 0) → ((𝐴 / 𝐵) · 𝐵) = 𝐴) | ||
| Theorem | diveq0 11904 | A ratio is zero iff the numerator is zero. (Contributed by NM, 20-Apr-2006.) (Revised by Mario Carneiro, 27-May-2016.) |
| ⊢ ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ ∧ 𝐵 ≠ 0) → ((𝐴 / 𝐵) = 0 ↔ 𝐴 = 0)) | ||
| Theorem | divne0b 11905 | The ratio of nonzero numbers is nonzero. (Contributed by NM, 2-Aug-2004.) (Proof shortened by Mario Carneiro, 27-May-2016.) |
| ⊢ ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ ∧ 𝐵 ≠ 0) → (𝐴 ≠ 0 ↔ (𝐴 / 𝐵) ≠ 0)) | ||
| Theorem | divne0 11906 | The ratio of nonzero numbers is nonzero. (Contributed by NM, 28-Dec-2007.) |
| ⊢ (((𝐴 ∈ ℂ ∧ 𝐴 ≠ 0) ∧ (𝐵 ∈ ℂ ∧ 𝐵 ≠ 0)) → (𝐴 / 𝐵) ≠ 0) | ||
| Theorem | recne0 11907 | The reciprocal of a nonzero number is nonzero. (Contributed by NM, 9-Feb-2006.) (Proof shortened by Mario Carneiro, 27-May-2016.) |
| ⊢ ((𝐴 ∈ ℂ ∧ 𝐴 ≠ 0) → (1 / 𝐴) ≠ 0) | ||
| Theorem | recid 11908 | Multiplication of a number and its reciprocal. (Contributed by NM, 25-Oct-1999.) (Proof shortened by Mario Carneiro, 27-May-2016.) |
| ⊢ ((𝐴 ∈ ℂ ∧ 𝐴 ≠ 0) → (𝐴 · (1 / 𝐴)) = 1) | ||
| Theorem | recid2 11909 | Multiplication of a number and its reciprocal. (Contributed by NM, 22-Jun-2006.) (Proof shortened by Mario Carneiro, 27-May-2016.) |
| ⊢ ((𝐴 ∈ ℂ ∧ 𝐴 ≠ 0) → ((1 / 𝐴) · 𝐴) = 1) | ||
| Theorem | divrec 11910 | Relationship between division and reciprocal. Theorem I.9 of [Apostol] p. 18. (Contributed by NM, 2-Aug-2004.) (Revised by Mario Carneiro, 27-May-2016.) |
| ⊢ ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ ∧ 𝐵 ≠ 0) → (𝐴 / 𝐵) = (𝐴 · (1 / 𝐵))) | ||
| Theorem | divrec2 11911 | Relationship between division and reciprocal. (Contributed by NM, 7-Feb-2006.) |
| ⊢ ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ ∧ 𝐵 ≠ 0) → (𝐴 / 𝐵) = ((1 / 𝐵) · 𝐴)) | ||
| Theorem | divass 11912 | An associative law for division. (Contributed by NM, 2-Aug-2004.) |
| ⊢ ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ ∧ (𝐶 ∈ ℂ ∧ 𝐶 ≠ 0)) → ((𝐴 · 𝐵) / 𝐶) = (𝐴 · (𝐵 / 𝐶))) | ||
| Theorem | div23 11913 | A commutative/associative law for division. (Contributed by NM, 2-Aug-2004.) |
| ⊢ ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ ∧ (𝐶 ∈ ℂ ∧ 𝐶 ≠ 0)) → ((𝐴 · 𝐵) / 𝐶) = ((𝐴 / 𝐶) · 𝐵)) | ||
| Theorem | div32 11914 | A commutative/associative law for division. (Contributed by Mario Carneiro, 27-May-2016.) |
| ⊢ ((𝐴 ∈ ℂ ∧ (𝐵 ∈ ℂ ∧ 𝐵 ≠ 0) ∧ 𝐶 ∈ ℂ) → ((𝐴 / 𝐵) · 𝐶) = (𝐴 · (𝐶 / 𝐵))) | ||
| Theorem | div13 11915 | A commutative/associative law for division. (Contributed by NM, 22-Apr-2005.) |
| ⊢ ((𝐴 ∈ ℂ ∧ (𝐵 ∈ ℂ ∧ 𝐵 ≠ 0) ∧ 𝐶 ∈ ℂ) → ((𝐴 / 𝐵) · 𝐶) = ((𝐶 / 𝐵) · 𝐴)) | ||
| Theorem | div12 11916 | A commutative/associative law for division. (Contributed by NM, 30-Apr-2005.) |
| ⊢ ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ ∧ (𝐶 ∈ ℂ ∧ 𝐶 ≠ 0)) → (𝐴 · (𝐵 / 𝐶)) = (𝐵 · (𝐴 / 𝐶))) | ||
| Theorem | divmulass 11917 | An associative law for division and multiplication. (Contributed by AV, 10-Jul-2021.) |
| ⊢ (((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ ∧ 𝐶 ∈ ℂ) ∧ (𝐷 ∈ ℂ ∧ 𝐷 ≠ 0)) → ((𝐴 · (𝐵 / 𝐷)) · 𝐶) = ((𝐴 · 𝐵) · (𝐶 / 𝐷))) | ||
| Theorem | divmulasscom 11918 | An associative/commutative law for division and multiplication. (Contributed by AV, 10-Jul-2021.) |
| ⊢ (((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ ∧ 𝐶 ∈ ℂ) ∧ (𝐷 ∈ ℂ ∧ 𝐷 ≠ 0)) → ((𝐴 · (𝐵 / 𝐷)) · 𝐶) = (𝐵 · ((𝐴 · 𝐶) / 𝐷))) | ||
| Theorem | divdir 11919 | Distribution of division over addition. (Contributed by NM, 31-Jul-2004.) (Proof shortened by Mario Carneiro, 27-May-2016.) |
| ⊢ ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ ∧ (𝐶 ∈ ℂ ∧ 𝐶 ≠ 0)) → ((𝐴 + 𝐵) / 𝐶) = ((𝐴 / 𝐶) + (𝐵 / 𝐶))) | ||
| Theorem | divcan3 11920 | A cancellation law for division. (Contributed by NM, 3-Feb-2004.) (Proof shortened by Mario Carneiro, 27-May-2016.) |
| ⊢ ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ ∧ 𝐵 ≠ 0) → ((𝐵 · 𝐴) / 𝐵) = 𝐴) | ||
| Theorem | divcan4 11921 | A cancellation law for division. (Contributed by NM, 8-Feb-2005.) |
| ⊢ ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ ∧ 𝐵 ≠ 0) → ((𝐴 · 𝐵) / 𝐵) = 𝐴) | ||
| Theorem | div11 11922 | One-to-one relationship for division. (Contributed by NM, 20-Apr-2006.) (Proof shortened by Mario Carneiro, 27-May-2016.) (Proof shortened by SN, 9-Jul-2025.) |
| ⊢ ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ ∧ (𝐶 ∈ ℂ ∧ 𝐶 ≠ 0)) → ((𝐴 / 𝐶) = (𝐵 / 𝐶) ↔ 𝐴 = 𝐵)) | ||
| Theorem | div11OLD 11923 | Obsolete version of div11 11922 as of 9-Jul-2025. (Contributed by NM, 20-Apr-2006.) (Proof shortened by Mario Carneiro, 27-May-2016.) (Proof modification is discouraged.) (New usage is discouraged.) |
| ⊢ ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ ∧ (𝐶 ∈ ℂ ∧ 𝐶 ≠ 0)) → ((𝐴 / 𝐶) = (𝐵 / 𝐶) ↔ 𝐴 = 𝐵)) | ||
| Theorem | diveq1 11924 | Equality in terms of unit ratio. (Contributed by Stefan O'Rear, 27-Aug-2015.) |
| ⊢ ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ ∧ 𝐵 ≠ 0) → ((𝐴 / 𝐵) = 1 ↔ 𝐴 = 𝐵)) | ||
| Theorem | divid 11925 | A number divided by itself is one. (Contributed by NM, 1-Aug-2004.) (Proof shortened by SN, 9-Jul-2025.) |
| ⊢ ((𝐴 ∈ ℂ ∧ 𝐴 ≠ 0) → (𝐴 / 𝐴) = 1) | ||
| Theorem | dividOLD 11926 | Obsolete version of divid 11925 as of 9-Jul-2025. (Contributed by NM, 1-Aug-2004.) (Proof modification is discouraged.) (New usage is discouraged.) |
| ⊢ ((𝐴 ∈ ℂ ∧ 𝐴 ≠ 0) → (𝐴 / 𝐴) = 1) | ||
| Theorem | div0 11927 | Division into zero is zero. (Contributed by NM, 14-Mar-2005.) (Proof shortened by SN, 9-Jul-2025.) |
| ⊢ ((𝐴 ∈ ℂ ∧ 𝐴 ≠ 0) → (0 / 𝐴) = 0) | ||
| Theorem | div0OLD 11928 | Obsolete version of div0 11927 as of 9-Jul-2025. (Contributed by NM, 14-Mar-2005.) (Proof modification is discouraged.) (New usage is discouraged.) |
| ⊢ ((𝐴 ∈ ℂ ∧ 𝐴 ≠ 0) → (0 / 𝐴) = 0) | ||
| Theorem | div1 11929 | A number divided by 1 is itself. (Contributed by NM, 9-Jan-2002.) (Proof shortened by Mario Carneiro, 27-May-2016.) |
| ⊢ (𝐴 ∈ ℂ → (𝐴 / 1) = 𝐴) | ||
| Theorem | 1div1e1 11930 | 1 divided by 1 is 1. (Contributed by David A. Wheeler, 7-Dec-2018.) |
| ⊢ (1 / 1) = 1 | ||
| Theorem | divneg 11931 | Move negative sign inside of a division. (Contributed by NM, 17-Sep-2004.) |
| ⊢ ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ ∧ 𝐵 ≠ 0) → -(𝐴 / 𝐵) = (-𝐴 / 𝐵)) | ||
| Theorem | muldivdir 11932 | Distribution of division over addition with a multiplication. (Contributed by AV, 1-Jul-2021.) |
| ⊢ ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ ∧ (𝐶 ∈ ℂ ∧ 𝐶 ≠ 0)) → (((𝐶 · 𝐴) + 𝐵) / 𝐶) = (𝐴 + (𝐵 / 𝐶))) | ||
| Theorem | divsubdir 11933 | Distribution of division over subtraction. (Contributed by NM, 4-Mar-2005.) |
| ⊢ ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ ∧ (𝐶 ∈ ℂ ∧ 𝐶 ≠ 0)) → ((𝐴 − 𝐵) / 𝐶) = ((𝐴 / 𝐶) − (𝐵 / 𝐶))) | ||
| Theorem | subdivcomb1 11934 | Bring a term in a subtraction into the numerator. (Contributed by Scott Fenton, 3-Jul-2013.) |
| ⊢ ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ ∧ (𝐶 ∈ ℂ ∧ 𝐶 ≠ 0)) → (((𝐶 · 𝐴) − 𝐵) / 𝐶) = (𝐴 − (𝐵 / 𝐶))) | ||
| Theorem | subdivcomb2 11935 | Bring a term in a subtraction into the numerator. (Contributed by Scott Fenton, 3-Jul-2013.) |
| ⊢ ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ ∧ (𝐶 ∈ ℂ ∧ 𝐶 ≠ 0)) → ((𝐴 − (𝐶 · 𝐵)) / 𝐶) = ((𝐴 / 𝐶) − 𝐵)) | ||
| Theorem | recrec 11936 | A number is equal to the reciprocal of its reciprocal. Theorem I.10 of [Apostol] p. 18. (Contributed by NM, 26-Sep-1999.) (Proof shortened by Mario Carneiro, 27-May-2016.) |
| ⊢ ((𝐴 ∈ ℂ ∧ 𝐴 ≠ 0) → (1 / (1 / 𝐴)) = 𝐴) | ||
| Theorem | rec11 11937 | Reciprocal is one-to-one. (Contributed by NM, 16-Sep-1999.) (Revised by Mario Carneiro, 27-May-2016.) |
| ⊢ (((𝐴 ∈ ℂ ∧ 𝐴 ≠ 0) ∧ (𝐵 ∈ ℂ ∧ 𝐵 ≠ 0)) → ((1 / 𝐴) = (1 / 𝐵) ↔ 𝐴 = 𝐵)) | ||
| Theorem | rec11r 11938 | Mutual reciprocals. (Contributed by Paul Chapman, 18-Oct-2007.) |
| ⊢ (((𝐴 ∈ ℂ ∧ 𝐴 ≠ 0) ∧ (𝐵 ∈ ℂ ∧ 𝐵 ≠ 0)) → ((1 / 𝐴) = 𝐵 ↔ (1 / 𝐵) = 𝐴)) | ||
| Theorem | divmuldiv 11939 | Multiplication of two ratios. Theorem I.14 of [Apostol] p. 18. (Contributed by NM, 1-Aug-2004.) |
| ⊢ (((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ) ∧ ((𝐶 ∈ ℂ ∧ 𝐶 ≠ 0) ∧ (𝐷 ∈ ℂ ∧ 𝐷 ≠ 0))) → ((𝐴 / 𝐶) · (𝐵 / 𝐷)) = ((𝐴 · 𝐵) / (𝐶 · 𝐷))) | ||
| Theorem | divdivdiv 11940 | Division of two ratios. Theorem I.15 of [Apostol] p. 18. (Contributed by NM, 2-Aug-2004.) |
| ⊢ (((𝐴 ∈ ℂ ∧ (𝐵 ∈ ℂ ∧ 𝐵 ≠ 0)) ∧ ((𝐶 ∈ ℂ ∧ 𝐶 ≠ 0) ∧ (𝐷 ∈ ℂ ∧ 𝐷 ≠ 0))) → ((𝐴 / 𝐵) / (𝐶 / 𝐷)) = ((𝐴 · 𝐷) / (𝐵 · 𝐶))) | ||
| Theorem | divcan5 11941 | Cancellation of common factor in a ratio. (Contributed by NM, 9-Jan-2006.) |
| ⊢ ((𝐴 ∈ ℂ ∧ (𝐵 ∈ ℂ ∧ 𝐵 ≠ 0) ∧ (𝐶 ∈ ℂ ∧ 𝐶 ≠ 0)) → ((𝐶 · 𝐴) / (𝐶 · 𝐵)) = (𝐴 / 𝐵)) | ||
| Theorem | divmul13 11942 | Swap the denominators in the product of two ratios. (Contributed by NM, 3-May-2005.) |
| ⊢ (((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ) ∧ ((𝐶 ∈ ℂ ∧ 𝐶 ≠ 0) ∧ (𝐷 ∈ ℂ ∧ 𝐷 ≠ 0))) → ((𝐴 / 𝐶) · (𝐵 / 𝐷)) = ((𝐵 / 𝐶) · (𝐴 / 𝐷))) | ||
| Theorem | divmul24 11943 | Swap the numerators in the product of two ratios. (Contributed by NM, 3-May-2005.) |
| ⊢ (((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ) ∧ ((𝐶 ∈ ℂ ∧ 𝐶 ≠ 0) ∧ (𝐷 ∈ ℂ ∧ 𝐷 ≠ 0))) → ((𝐴 / 𝐶) · (𝐵 / 𝐷)) = ((𝐴 / 𝐷) · (𝐵 / 𝐶))) | ||
| Theorem | divmuleq 11944 | Cross-multiply in an equality of ratios. (Contributed by Mario Carneiro, 23-Feb-2014.) |
| ⊢ (((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ) ∧ ((𝐶 ∈ ℂ ∧ 𝐶 ≠ 0) ∧ (𝐷 ∈ ℂ ∧ 𝐷 ≠ 0))) → ((𝐴 / 𝐶) = (𝐵 / 𝐷) ↔ (𝐴 · 𝐷) = (𝐵 · 𝐶))) | ||
| Theorem | recdiv 11945 | The reciprocal of a ratio. (Contributed by NM, 3-Aug-2004.) |
| ⊢ (((𝐴 ∈ ℂ ∧ 𝐴 ≠ 0) ∧ (𝐵 ∈ ℂ ∧ 𝐵 ≠ 0)) → (1 / (𝐴 / 𝐵)) = (𝐵 / 𝐴)) | ||
| Theorem | divcan6 11946 | Cancellation of inverted fractions. (Contributed by NM, 28-Dec-2007.) |
| ⊢ (((𝐴 ∈ ℂ ∧ 𝐴 ≠ 0) ∧ (𝐵 ∈ ℂ ∧ 𝐵 ≠ 0)) → ((𝐴 / 𝐵) · (𝐵 / 𝐴)) = 1) | ||
| Theorem | divdiv32 11947 | Swap denominators in a division. (Contributed by NM, 2-Aug-2004.) |
| ⊢ ((𝐴 ∈ ℂ ∧ (𝐵 ∈ ℂ ∧ 𝐵 ≠ 0) ∧ (𝐶 ∈ ℂ ∧ 𝐶 ≠ 0)) → ((𝐴 / 𝐵) / 𝐶) = ((𝐴 / 𝐶) / 𝐵)) | ||
| Theorem | divcan7 11948 | Cancel equal divisors in a division. (Contributed by Jeff Hankins, 29-Sep-2013.) |
| ⊢ ((𝐴 ∈ ℂ ∧ (𝐵 ∈ ℂ ∧ 𝐵 ≠ 0) ∧ (𝐶 ∈ ℂ ∧ 𝐶 ≠ 0)) → ((𝐴 / 𝐶) / (𝐵 / 𝐶)) = (𝐴 / 𝐵)) | ||
| Theorem | dmdcan 11949 | Cancellation law for division and multiplication. (Contributed by Scott Fenton, 7-Jun-2013.) (Proof shortened by Fan Zheng, 3-Jul-2016.) |
| ⊢ (((𝐴 ∈ ℂ ∧ 𝐴 ≠ 0) ∧ (𝐵 ∈ ℂ ∧ 𝐵 ≠ 0) ∧ 𝐶 ∈ ℂ) → ((𝐴 / 𝐵) · (𝐶 / 𝐴)) = (𝐶 / 𝐵)) | ||
| Theorem | divdiv1 11950 | Division into a fraction. (Contributed by NM, 31-Dec-2007.) |
| ⊢ ((𝐴 ∈ ℂ ∧ (𝐵 ∈ ℂ ∧ 𝐵 ≠ 0) ∧ (𝐶 ∈ ℂ ∧ 𝐶 ≠ 0)) → ((𝐴 / 𝐵) / 𝐶) = (𝐴 / (𝐵 · 𝐶))) | ||
| Theorem | divdiv2 11951 | Division by a fraction. (Contributed by NM, 27-Dec-2008.) |
| ⊢ ((𝐴 ∈ ℂ ∧ (𝐵 ∈ ℂ ∧ 𝐵 ≠ 0) ∧ (𝐶 ∈ ℂ ∧ 𝐶 ≠ 0)) → (𝐴 / (𝐵 / 𝐶)) = ((𝐴 · 𝐶) / 𝐵)) | ||
| Theorem | recdiv2 11952 | Division into a reciprocal. (Contributed by NM, 19-Oct-2007.) |
| ⊢ (((𝐴 ∈ ℂ ∧ 𝐴 ≠ 0) ∧ (𝐵 ∈ ℂ ∧ 𝐵 ≠ 0)) → ((1 / 𝐴) / 𝐵) = (1 / (𝐴 · 𝐵))) | ||
| Theorem | ddcan 11953 | Cancellation in a double division. (Contributed by Mario Carneiro, 26-Apr-2015.) |
| ⊢ (((𝐴 ∈ ℂ ∧ 𝐴 ≠ 0) ∧ (𝐵 ∈ ℂ ∧ 𝐵 ≠ 0)) → (𝐴 / (𝐴 / 𝐵)) = 𝐵) | ||
| Theorem | divadddiv 11954 | Addition of two ratios. Theorem I.13 of [Apostol] p. 18. (Contributed by NM, 1-Aug-2004.) (Revised by Mario Carneiro, 2-May-2016.) |
| ⊢ (((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ) ∧ ((𝐶 ∈ ℂ ∧ 𝐶 ≠ 0) ∧ (𝐷 ∈ ℂ ∧ 𝐷 ≠ 0))) → ((𝐴 / 𝐶) + (𝐵 / 𝐷)) = (((𝐴 · 𝐷) + (𝐵 · 𝐶)) / (𝐶 · 𝐷))) | ||
| Theorem | divsubdiv 11955 | Subtraction of two ratios. (Contributed by Scott Fenton, 22-Apr-2014.) (Revised by Mario Carneiro, 2-May-2016.) |
| ⊢ (((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ) ∧ ((𝐶 ∈ ℂ ∧ 𝐶 ≠ 0) ∧ (𝐷 ∈ ℂ ∧ 𝐷 ≠ 0))) → ((𝐴 / 𝐶) − (𝐵 / 𝐷)) = (((𝐴 · 𝐷) − (𝐵 · 𝐶)) / (𝐶 · 𝐷))) | ||
| Theorem | conjmul 11956 | Two numbers whose reciprocals sum to 1 are called "conjugates" and satisfy this relationship. Equation 5 of [Kreyszig] p. 12. (Contributed by NM, 12-Nov-2006.) |
| ⊢ (((𝑃 ∈ ℂ ∧ 𝑃 ≠ 0) ∧ (𝑄 ∈ ℂ ∧ 𝑄 ≠ 0)) → (((1 / 𝑃) + (1 / 𝑄)) = 1 ↔ ((𝑃 − 1) · (𝑄 − 1)) = 1)) | ||
| Theorem | rereccl 11957 | Closure law for reciprocal. (Contributed by NM, 30-Apr-2005.) (Revised by Mario Carneiro, 27-May-2016.) |
| ⊢ ((𝐴 ∈ ℝ ∧ 𝐴 ≠ 0) → (1 / 𝐴) ∈ ℝ) | ||
| Theorem | redivcl 11958 | Closure law for division of reals. (Contributed by NM, 27-Sep-1999.) (Revised by Mario Carneiro, 27-May-2016.) |
| ⊢ ((𝐴 ∈ ℝ ∧ 𝐵 ∈ ℝ ∧ 𝐵 ≠ 0) → (𝐴 / 𝐵) ∈ ℝ) | ||
| Theorem | eqneg 11959 | A number equal to its negative is zero. (Contributed by NM, 12-Jul-2005.) (Revised by Mario Carneiro, 27-May-2016.) |
| ⊢ (𝐴 ∈ ℂ → (𝐴 = -𝐴 ↔ 𝐴 = 0)) | ||
| Theorem | eqnegd 11960 | A complex number equals its negative iff it is zero. Deduction form of eqneg 11959. (Contributed by David Moews, 28-Feb-2017.) |
| ⊢ (𝜑 → 𝐴 ∈ ℂ) ⇒ ⊢ (𝜑 → (𝐴 = -𝐴 ↔ 𝐴 = 0)) | ||
| Theorem | eqnegad 11961 | If a complex number equals its own negative, it is zero. One-way deduction form of eqneg 11959. (Contributed by David Moews, 28-Feb-2017.) |
| ⊢ (𝜑 → 𝐴 ∈ ℂ) & ⊢ (𝜑 → 𝐴 = -𝐴) ⇒ ⊢ (𝜑 → 𝐴 = 0) | ||
| Theorem | div2neg 11962 | Quotient of two negatives. (Contributed by Paul Chapman, 10-Nov-2012.) |
| ⊢ ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ ∧ 𝐵 ≠ 0) → (-𝐴 / -𝐵) = (𝐴 / 𝐵)) | ||
| Theorem | divneg2 11963 | Move negative sign inside of a division. (Contributed by Mario Carneiro, 15-Sep-2014.) |
| ⊢ ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ ∧ 𝐵 ≠ 0) → -(𝐴 / 𝐵) = (𝐴 / -𝐵)) | ||
| Theorem | recclzi 11964 | Closure law for reciprocal. (Contributed by NM, 30-Apr-2005.) |
| ⊢ 𝐴 ∈ ℂ ⇒ ⊢ (𝐴 ≠ 0 → (1 / 𝐴) ∈ ℂ) | ||
| Theorem | recne0zi 11965 | The reciprocal of a nonzero number is nonzero. (Contributed by NM, 14-May-1999.) |
| ⊢ 𝐴 ∈ ℂ ⇒ ⊢ (𝐴 ≠ 0 → (1 / 𝐴) ≠ 0) | ||
| Theorem | recidzi 11966 | Multiplication of a number and its reciprocal. (Contributed by NM, 14-May-1999.) |
| ⊢ 𝐴 ∈ ℂ ⇒ ⊢ (𝐴 ≠ 0 → (𝐴 · (1 / 𝐴)) = 1) | ||
| Theorem | div1i 11967 | A number divided by 1 is itself. (Contributed by NM, 9-Jan-2002.) |
| ⊢ 𝐴 ∈ ℂ ⇒ ⊢ (𝐴 / 1) = 𝐴 | ||
| Theorem | eqnegi 11968 | A number equal to its negative is zero. (Contributed by NM, 29-May-1999.) |
| ⊢ 𝐴 ∈ ℂ ⇒ ⊢ (𝐴 = -𝐴 ↔ 𝐴 = 0) | ||
| Theorem | reccli 11969 | Closure law for reciprocal. (Contributed by NM, 30-Apr-2005.) |
| ⊢ 𝐴 ∈ ℂ & ⊢ 𝐴 ≠ 0 ⇒ ⊢ (1 / 𝐴) ∈ ℂ | ||
| Theorem | recidi 11970 | Multiplication of a number and its reciprocal. (Contributed by NM, 9-Feb-1995.) |
| ⊢ 𝐴 ∈ ℂ & ⊢ 𝐴 ≠ 0 ⇒ ⊢ (𝐴 · (1 / 𝐴)) = 1 | ||
| Theorem | recreci 11971 | A number is equal to the reciprocal of its reciprocal. Theorem I.10 of [Apostol] p. 18. (Contributed by NM, 9-Feb-1995.) |
| ⊢ 𝐴 ∈ ℂ & ⊢ 𝐴 ≠ 0 ⇒ ⊢ (1 / (1 / 𝐴)) = 𝐴 | ||
| Theorem | dividi 11972 | A number divided by itself is one. (Contributed by NM, 9-Feb-1995.) |
| ⊢ 𝐴 ∈ ℂ & ⊢ 𝐴 ≠ 0 ⇒ ⊢ (𝐴 / 𝐴) = 1 | ||
| Theorem | div0i 11973 | Division into zero is zero. (Contributed by NM, 12-Aug-1999.) |
| ⊢ 𝐴 ∈ ℂ & ⊢ 𝐴 ≠ 0 ⇒ ⊢ (0 / 𝐴) = 0 | ||
| Theorem | divclzi 11974 | Closure law for division. (Contributed by NM, 7-May-1999.) (Revised by Mario Carneiro, 17-Feb-2014.) |
| ⊢ 𝐴 ∈ ℂ & ⊢ 𝐵 ∈ ℂ ⇒ ⊢ (𝐵 ≠ 0 → (𝐴 / 𝐵) ∈ ℂ) | ||
| Theorem | divcan1zi 11975 | A cancellation law for division. (Contributed by NM, 2-Oct-1999.) |
| ⊢ 𝐴 ∈ ℂ & ⊢ 𝐵 ∈ ℂ ⇒ ⊢ (𝐵 ≠ 0 → ((𝐴 / 𝐵) · 𝐵) = 𝐴) | ||
| Theorem | divcan2zi 11976 | A cancellation law for division. (Contributed by NM, 10-Aug-1999.) |
| ⊢ 𝐴 ∈ ℂ & ⊢ 𝐵 ∈ ℂ ⇒ ⊢ (𝐵 ≠ 0 → (𝐵 · (𝐴 / 𝐵)) = 𝐴) | ||
| Theorem | divreczi 11977 | Relationship between division and reciprocal. Theorem I.9 of [Apostol] p. 18. (Contributed by NM, 11-Oct-1999.) |
| ⊢ 𝐴 ∈ ℂ & ⊢ 𝐵 ∈ ℂ ⇒ ⊢ (𝐵 ≠ 0 → (𝐴 / 𝐵) = (𝐴 · (1 / 𝐵))) | ||
| Theorem | divcan3zi 11978 | A cancellation law for division. (Eliminates a hypothesis of divcan3i 11985 with the weak deduction theorem.) (Contributed by NM, 3-Feb-2004.) |
| ⊢ 𝐴 ∈ ℂ & ⊢ 𝐵 ∈ ℂ ⇒ ⊢ (𝐵 ≠ 0 → ((𝐵 · 𝐴) / 𝐵) = 𝐴) | ||
| Theorem | divcan4zi 11979 | A cancellation law for division. (Contributed by NM, 12-Oct-1999.) |
| ⊢ 𝐴 ∈ ℂ & ⊢ 𝐵 ∈ ℂ ⇒ ⊢ (𝐵 ≠ 0 → ((𝐴 · 𝐵) / 𝐵) = 𝐴) | ||
| Theorem | rec11i 11980 | Reciprocal is one-to-one. (Contributed by NM, 16-Sep-1999.) |
| ⊢ 𝐴 ∈ ℂ & ⊢ 𝐵 ∈ ℂ ⇒ ⊢ ((𝐴 ≠ 0 ∧ 𝐵 ≠ 0) → ((1 / 𝐴) = (1 / 𝐵) ↔ 𝐴 = 𝐵)) | ||
| Theorem | divcli 11981 | Closure law for division. (Contributed by NM, 2-Feb-1995.) (Revised by Mario Carneiro, 17-Feb-2014.) |
| ⊢ 𝐴 ∈ ℂ & ⊢ 𝐵 ∈ ℂ & ⊢ 𝐵 ≠ 0 ⇒ ⊢ (𝐴 / 𝐵) ∈ ℂ | ||
| Theorem | divcan2i 11982 | A cancellation law for division. (Contributed by NM, 9-Feb-1995.) |
| ⊢ 𝐴 ∈ ℂ & ⊢ 𝐵 ∈ ℂ & ⊢ 𝐵 ≠ 0 ⇒ ⊢ (𝐵 · (𝐴 / 𝐵)) = 𝐴 | ||
| Theorem | divcan1i 11983 | A cancellation law for division. (Contributed by NM, 18-May-1999.) |
| ⊢ 𝐴 ∈ ℂ & ⊢ 𝐵 ∈ ℂ & ⊢ 𝐵 ≠ 0 ⇒ ⊢ ((𝐴 / 𝐵) · 𝐵) = 𝐴 | ||
| Theorem | divreci 11984 | Relationship between division and reciprocal. Theorem I.9 of [Apostol] p. 18. (Contributed by NM, 9-Feb-1995.) |
| ⊢ 𝐴 ∈ ℂ & ⊢ 𝐵 ∈ ℂ & ⊢ 𝐵 ≠ 0 ⇒ ⊢ (𝐴 / 𝐵) = (𝐴 · (1 / 𝐵)) | ||
| Theorem | divcan3i 11985 | A cancellation law for division. (Contributed by NM, 16-Feb-1995.) |
| ⊢ 𝐴 ∈ ℂ & ⊢ 𝐵 ∈ ℂ & ⊢ 𝐵 ≠ 0 ⇒ ⊢ ((𝐵 · 𝐴) / 𝐵) = 𝐴 | ||
| Theorem | divcan4i 11986 | A cancellation law for division. (Contributed by NM, 18-May-1999.) |
| ⊢ 𝐴 ∈ ℂ & ⊢ 𝐵 ∈ ℂ & ⊢ 𝐵 ≠ 0 ⇒ ⊢ ((𝐴 · 𝐵) / 𝐵) = 𝐴 | ||
| Theorem | divne0i 11987 | The ratio of nonzero numbers is nonzero. (Contributed by NM, 9-Feb-1995.) |
| ⊢ 𝐴 ∈ ℂ & ⊢ 𝐵 ∈ ℂ & ⊢ 𝐴 ≠ 0 & ⊢ 𝐵 ≠ 0 ⇒ ⊢ (𝐴 / 𝐵) ≠ 0 | ||
| Theorem | rec11ii 11988 | Reciprocal is one-to-one. (Contributed by NM, 16-Sep-1999.) |
| ⊢ 𝐴 ∈ ℂ & ⊢ 𝐵 ∈ ℂ & ⊢ 𝐴 ≠ 0 & ⊢ 𝐵 ≠ 0 ⇒ ⊢ ((1 / 𝐴) = (1 / 𝐵) ↔ 𝐴 = 𝐵) | ||
| Theorem | divasszi 11989 | An associative law for division. (Contributed by NM, 12-Aug-1999.) |
| ⊢ 𝐴 ∈ ℂ & ⊢ 𝐵 ∈ ℂ & ⊢ 𝐶 ∈ ℂ ⇒ ⊢ (𝐶 ≠ 0 → ((𝐴 · 𝐵) / 𝐶) = (𝐴 · (𝐵 / 𝐶))) | ||
| Theorem | divmulzi 11990 | Relationship between division and multiplication. (Contributed by NM, 8-May-1999.) (Revised by Mario Carneiro, 17-Feb-2014.) |
| ⊢ 𝐴 ∈ ℂ & ⊢ 𝐵 ∈ ℂ & ⊢ 𝐶 ∈ ℂ ⇒ ⊢ (𝐵 ≠ 0 → ((𝐴 / 𝐵) = 𝐶 ↔ (𝐵 · 𝐶) = 𝐴)) | ||
| Theorem | divdirzi 11991 | Distribution of division over addition. (Contributed by NM, 31-Jul-2004.) |
| ⊢ 𝐴 ∈ ℂ & ⊢ 𝐵 ∈ ℂ & ⊢ 𝐶 ∈ ℂ ⇒ ⊢ (𝐶 ≠ 0 → ((𝐴 + 𝐵) / 𝐶) = ((𝐴 / 𝐶) + (𝐵 / 𝐶))) | ||
| Theorem | divdiv23zi 11992 | Swap denominators in a division. (Contributed by NM, 15-Sep-1999.) |
| ⊢ 𝐴 ∈ ℂ & ⊢ 𝐵 ∈ ℂ & ⊢ 𝐶 ∈ ℂ ⇒ ⊢ ((𝐵 ≠ 0 ∧ 𝐶 ≠ 0) → ((𝐴 / 𝐵) / 𝐶) = ((𝐴 / 𝐶) / 𝐵)) | ||
| Theorem | divmuli 11993 | Relationship between division and multiplication. (Contributed by NM, 2-Feb-1995.) (Revised by Mario Carneiro, 17-Feb-2014.) |
| ⊢ 𝐴 ∈ ℂ & ⊢ 𝐵 ∈ ℂ & ⊢ 𝐶 ∈ ℂ & ⊢ 𝐵 ≠ 0 ⇒ ⊢ ((𝐴 / 𝐵) = 𝐶 ↔ (𝐵 · 𝐶) = 𝐴) | ||
| Theorem | divdiv32i 11994 | Swap denominators in a division. (Contributed by NM, 15-Sep-1999.) |
| ⊢ 𝐴 ∈ ℂ & ⊢ 𝐵 ∈ ℂ & ⊢ 𝐶 ∈ ℂ & ⊢ 𝐵 ≠ 0 & ⊢ 𝐶 ≠ 0 ⇒ ⊢ ((𝐴 / 𝐵) / 𝐶) = ((𝐴 / 𝐶) / 𝐵) | ||
| Theorem | divassi 11995 | An associative law for division. (Contributed by NM, 15-Feb-1995.) |
| ⊢ 𝐴 ∈ ℂ & ⊢ 𝐵 ∈ ℂ & ⊢ 𝐶 ∈ ℂ & ⊢ 𝐶 ≠ 0 ⇒ ⊢ ((𝐴 · 𝐵) / 𝐶) = (𝐴 · (𝐵 / 𝐶)) | ||
| Theorem | divdiri 11996 | Distribution of division over addition. (Contributed by NM, 16-Feb-1995.) |
| ⊢ 𝐴 ∈ ℂ & ⊢ 𝐵 ∈ ℂ & ⊢ 𝐶 ∈ ℂ & ⊢ 𝐶 ≠ 0 ⇒ ⊢ ((𝐴 + 𝐵) / 𝐶) = ((𝐴 / 𝐶) + (𝐵 / 𝐶)) | ||
| Theorem | div23i 11997 | A commutative/associative law for division. (Contributed by NM, 3-Sep-1999.) |
| ⊢ 𝐴 ∈ ℂ & ⊢ 𝐵 ∈ ℂ & ⊢ 𝐶 ∈ ℂ & ⊢ 𝐶 ≠ 0 ⇒ ⊢ ((𝐴 · 𝐵) / 𝐶) = ((𝐴 / 𝐶) · 𝐵) | ||
| Theorem | div11i 11998 | One-to-one relationship for division. (Contributed by NM, 20-Aug-2001.) |
| ⊢ 𝐴 ∈ ℂ & ⊢ 𝐵 ∈ ℂ & ⊢ 𝐶 ∈ ℂ & ⊢ 𝐶 ≠ 0 ⇒ ⊢ ((𝐴 / 𝐶) = (𝐵 / 𝐶) ↔ 𝐴 = 𝐵) | ||
| Theorem | divmuldivi 11999 | Multiplication of two ratios. Theorem I.14 of [Apostol] p. 18. (Contributed by NM, 16-Feb-1995.) |
| ⊢ 𝐴 ∈ ℂ & ⊢ 𝐵 ∈ ℂ & ⊢ 𝐶 ∈ ℂ & ⊢ 𝐷 ∈ ℂ & ⊢ 𝐵 ≠ 0 & ⊢ 𝐷 ≠ 0 ⇒ ⊢ ((𝐴 / 𝐵) · (𝐶 / 𝐷)) = ((𝐴 · 𝐶) / (𝐵 · 𝐷)) | ||
| Theorem | divmul13i 12000 | Swap denominators of two ratios. (Contributed by NM, 6-Aug-1999.) |
| ⊢ 𝐴 ∈ ℂ & ⊢ 𝐵 ∈ ℂ & ⊢ 𝐶 ∈ ℂ & ⊢ 𝐷 ∈ ℂ & ⊢ 𝐵 ≠ 0 & ⊢ 𝐷 ≠ 0 ⇒ ⊢ ((𝐴 / 𝐵) · (𝐶 / 𝐷)) = ((𝐶 / 𝐵) · (𝐴 / 𝐷)) | ||
| < Previous Next > |
| Copyright terms: Public domain | < Previous Next > |