| Metamath
Proof Explorer Theorem List (p. 112 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-30904) |
(30905-32427) |
(32428-49649) |
| Type | Label | Description |
|---|---|---|
| Statement | ||
| Theorem | m1r 11101 | The constant -1R is a signed real. (Contributed by NM, 9-Aug-1995.) (New usage is discouraged.) |
| ⊢ -1R ∈ R | ||
| Theorem | addclsr 11102 | Closure of addition on signed reals. (Contributed by NM, 25-Jul-1995.) (New usage is discouraged.) |
| ⊢ ((𝐴 ∈ R ∧ 𝐵 ∈ R) → (𝐴 +R 𝐵) ∈ R) | ||
| Theorem | mulclsr 11103 | Closure of multiplication on signed reals. (Contributed by NM, 10-Aug-1995.) (New usage is discouraged.) |
| ⊢ ((𝐴 ∈ R ∧ 𝐵 ∈ R) → (𝐴 ·R 𝐵) ∈ R) | ||
| Theorem | dmaddsr 11104 | Domain of addition on signed reals. (Contributed by NM, 25-Aug-1995.) (New usage is discouraged.) |
| ⊢ dom +R = (R × R) | ||
| Theorem | dmmulsr 11105 | Domain of multiplication on signed reals. (Contributed by NM, 25-Aug-1995.) (New usage is discouraged.) |
| ⊢ dom ·R = (R × R) | ||
| Theorem | addcomsr 11106 | Addition of signed reals is commutative. (Contributed by NM, 31-Aug-1995.) (Revised by Mario Carneiro, 28-Apr-2015.) (New usage is discouraged.) |
| ⊢ (𝐴 +R 𝐵) = (𝐵 +R 𝐴) | ||
| Theorem | addasssr 11107 | Addition of signed reals is associative. (Contributed by NM, 2-Sep-1995.) (Revised by Mario Carneiro, 28-Apr-2015.) (New usage is discouraged.) |
| ⊢ ((𝐴 +R 𝐵) +R 𝐶) = (𝐴 +R (𝐵 +R 𝐶)) | ||
| Theorem | mulcomsr 11108 | Multiplication of signed reals is commutative. (Contributed by NM, 31-Aug-1995.) (Revised by Mario Carneiro, 28-Apr-2015.) (New usage is discouraged.) |
| ⊢ (𝐴 ·R 𝐵) = (𝐵 ·R 𝐴) | ||
| Theorem | mulasssr 11109 | Multiplication of signed reals is associative. (Contributed by NM, 2-Sep-1995.) (Revised by Mario Carneiro, 28-Apr-2015.) (New usage is discouraged.) |
| ⊢ ((𝐴 ·R 𝐵) ·R 𝐶) = (𝐴 ·R (𝐵 ·R 𝐶)) | ||
| Theorem | distrsr 11110 | Multiplication of signed reals is distributive. (Contributed by NM, 2-Sep-1995.) (Revised by Mario Carneiro, 28-Apr-2015.) (New usage is discouraged.) |
| ⊢ (𝐴 ·R (𝐵 +R 𝐶)) = ((𝐴 ·R 𝐵) +R (𝐴 ·R 𝐶)) | ||
| Theorem | m1p1sr 11111 | Minus one plus one is zero for signed reals. (Contributed by NM, 5-May-1996.) (New usage is discouraged.) |
| ⊢ (-1R +R 1R) = 0R | ||
| Theorem | m1m1sr 11112 | Minus one times minus one is plus one for signed reals. (Contributed by NM, 14-May-1996.) (New usage is discouraged.) |
| ⊢ (-1R ·R -1R) = 1R | ||
| Theorem | ltsosr 11113 | Signed real 'less than' is a strict ordering. (Contributed by NM, 19-Feb-1996.) (New usage is discouraged.) |
| ⊢ <R Or R | ||
| Theorem | 0lt1sr 11114 | 0 is less than 1 for signed reals. (Contributed by NM, 26-Mar-1996.) (New usage is discouraged.) |
| ⊢ 0R <R 1R | ||
| Theorem | 1ne0sr 11115 | 1 and 0 are distinct for signed reals. (Contributed by NM, 26-Mar-1996.) (New usage is discouraged.) |
| ⊢ ¬ 1R = 0R | ||
| Theorem | 0idsr 11116 | The signed real number 0 is an identity element for addition of signed reals. (Contributed by NM, 10-Apr-1996.) (New usage is discouraged.) |
| ⊢ (𝐴 ∈ R → (𝐴 +R 0R) = 𝐴) | ||
| Theorem | 1idsr 11117 | 1 is an identity element for multiplication. (Contributed by NM, 2-May-1996.) (New usage is discouraged.) |
| ⊢ (𝐴 ∈ R → (𝐴 ·R 1R) = 𝐴) | ||
| Theorem | 00sr 11118 | A signed real times 0 is 0. (Contributed by NM, 10-Apr-1996.) (New usage is discouraged.) |
| ⊢ (𝐴 ∈ R → (𝐴 ·R 0R) = 0R) | ||
| Theorem | ltasr 11119 | Ordering property of addition. (Contributed by NM, 10-May-1996.) (New usage is discouraged.) |
| ⊢ (𝐶 ∈ R → (𝐴 <R 𝐵 ↔ (𝐶 +R 𝐴) <R (𝐶 +R 𝐵))) | ||
| Theorem | pn0sr 11120 | A signed real plus its negative is zero. (Contributed by NM, 14-May-1996.) (New usage is discouraged.) |
| ⊢ (𝐴 ∈ R → (𝐴 +R (𝐴 ·R -1R)) = 0R) | ||
| Theorem | negexsr 11121* | Existence of negative signed real. Part of Proposition 9-4.3 of [Gleason] p. 126. (Contributed by NM, 2-May-1996.) (New usage is discouraged.) |
| ⊢ (𝐴 ∈ R → ∃𝑥 ∈ R (𝐴 +R 𝑥) = 0R) | ||
| Theorem | recexsrlem 11122* | The reciprocal of a positive signed real exists. Part of Proposition 9-4.3 of [Gleason] p. 126. (Contributed by NM, 15-May-1996.) (New usage is discouraged.) |
| ⊢ (0R <R 𝐴 → ∃𝑥 ∈ R (𝐴 ·R 𝑥) = 1R) | ||
| Theorem | addgt0sr 11123 | The sum of two positive signed reals is positive. (Contributed by NM, 14-May-1996.) (New usage is discouraged.) |
| ⊢ ((0R <R 𝐴 ∧ 0R <R 𝐵) → 0R <R (𝐴 +R 𝐵)) | ||
| Theorem | mulgt0sr 11124 | The product of two positive signed reals is positive. (Contributed by NM, 13-May-1996.) (New usage is discouraged.) |
| ⊢ ((0R <R 𝐴 ∧ 0R <R 𝐵) → 0R <R (𝐴 ·R 𝐵)) | ||
| Theorem | sqgt0sr 11125 | The square of a nonzero signed real is positive. (Contributed by NM, 14-May-1996.) (New usage is discouraged.) |
| ⊢ ((𝐴 ∈ R ∧ 𝐴 ≠ 0R) → 0R <R (𝐴 ·R 𝐴)) | ||
| Theorem | recexsr 11126* | The reciprocal of a nonzero signed real exists. Part of Proposition 9-4.3 of [Gleason] p. 126. (Contributed by NM, 15-May-1996.) (New usage is discouraged.) |
| ⊢ ((𝐴 ∈ R ∧ 𝐴 ≠ 0R) → ∃𝑥 ∈ R (𝐴 ·R 𝑥) = 1R) | ||
| Theorem | mappsrpr 11127 | Mapping from positive signed reals to positive reals. (Contributed by NM, 17-May-1996.) (Revised by Mario Carneiro, 15-Jun-2013.) (New usage is discouraged.) |
| ⊢ 𝐶 ∈ R ⇒ ⊢ ((𝐶 +R -1R) <R (𝐶 +R [〈𝐴, 1P〉] ~R ) ↔ 𝐴 ∈ P) | ||
| Theorem | ltpsrpr 11128 | Mapping of order from positive signed reals to positive reals. (Contributed by NM, 17-May-1996.) (Revised by Mario Carneiro, 15-Jun-2013.) (New usage is discouraged.) |
| ⊢ 𝐶 ∈ R ⇒ ⊢ ((𝐶 +R [〈𝐴, 1P〉] ~R ) <R (𝐶 +R [〈𝐵, 1P〉] ~R ) ↔ 𝐴<P 𝐵) | ||
| Theorem | map2psrpr 11129* | Equivalence for positive signed real. (Contributed by NM, 17-May-1996.) (Revised by Mario Carneiro, 15-Jun-2013.) (New usage is discouraged.) |
| ⊢ 𝐶 ∈ R ⇒ ⊢ ((𝐶 +R -1R) <R 𝐴 ↔ ∃𝑥 ∈ P (𝐶 +R [〈𝑥, 1P〉] ~R ) = 𝐴) | ||
| Theorem | supsrlem 11130* | Lemma for supremum theorem. (Contributed by NM, 21-May-1996.) (Revised by Mario Carneiro, 15-Jun-2013.) (New usage is discouraged.) |
| ⊢ 𝐵 = {𝑤 ∣ (𝐶 +R [〈𝑤, 1P〉] ~R ) ∈ 𝐴} & ⊢ 𝐶 ∈ R ⇒ ⊢ ((𝐶 ∈ 𝐴 ∧ ∃𝑥 ∈ R ∀𝑦 ∈ 𝐴 𝑦 <R 𝑥) → ∃𝑥 ∈ R (∀𝑦 ∈ 𝐴 ¬ 𝑥 <R 𝑦 ∧ ∀𝑦 ∈ R (𝑦 <R 𝑥 → ∃𝑧 ∈ 𝐴 𝑦 <R 𝑧))) | ||
| Theorem | supsr 11131* | A nonempty, bounded set of signed reals has a supremum. (Contributed by NM, 21-May-1996.) (Revised by Mario Carneiro, 15-Jun-2013.) (New usage is discouraged.) |
| ⊢ ((𝐴 ≠ ∅ ∧ ∃𝑥 ∈ R ∀𝑦 ∈ 𝐴 𝑦 <R 𝑥) → ∃𝑥 ∈ R (∀𝑦 ∈ 𝐴 ¬ 𝑥 <R 𝑦 ∧ ∀𝑦 ∈ R (𝑦 <R 𝑥 → ∃𝑧 ∈ 𝐴 𝑦 <R 𝑧))) | ||
| Syntax | cc 11132 | Class of complex numbers. |
| class ℂ | ||
| Syntax | cr 11133 | Class of real numbers. |
| class ℝ | ||
| Syntax | cc0 11134 | Extend class notation to include the complex number 0. |
| class 0 | ||
| Syntax | c1 11135 | Extend class notation to include the complex number 1. |
| class 1 | ||
| Syntax | ci 11136 | Extend class notation to include the complex number i. |
| class i | ||
| Syntax | caddc 11137 | Addition on complex numbers. |
| class + | ||
| Syntax | cltrr 11138 | 'Less than' predicate (defined over real subset of complex numbers). |
| class <ℝ | ||
| Syntax | cmul 11139 | Multiplication on complex numbers. The token · is a center dot. |
| class · | ||
| Definition | df-c 11140 | Define the set of complex numbers. The 23 axioms for complex numbers start at axresscn 11167. (Contributed by NM, 22-Feb-1996.) (New usage is discouraged.) |
| ⊢ ℂ = (R × R) | ||
| Definition | df-0 11141 | Define the complex number 0. (Contributed by NM, 22-Feb-1996.) (New usage is discouraged.) |
| ⊢ 0 = 〈0R, 0R〉 | ||
| Definition | df-1 11142 | Define the complex number 1. (Contributed by NM, 22-Feb-1996.) (New usage is discouraged.) |
| ⊢ 1 = 〈1R, 0R〉 | ||
| Definition | df-i 11143 | Define the complex number i (the imaginary unit). (Contributed by NM, 22-Feb-1996.) (New usage is discouraged.) |
| ⊢ i = 〈0R, 1R〉 | ||
| Definition | df-r 11144 | Define the set of real numbers. (Contributed by NM, 22-Feb-1996.) (New usage is discouraged.) |
| ⊢ ℝ = (R × {0R}) | ||
| Definition | df-add 11145* | Define addition over complex numbers. (Contributed by NM, 28-May-1995.) (New usage is discouraged.) |
| ⊢ + = {〈〈𝑥, 𝑦〉, 𝑧〉 ∣ ((𝑥 ∈ ℂ ∧ 𝑦 ∈ ℂ) ∧ ∃𝑤∃𝑣∃𝑢∃𝑓((𝑥 = 〈𝑤, 𝑣〉 ∧ 𝑦 = 〈𝑢, 𝑓〉) ∧ 𝑧 = 〈(𝑤 +R 𝑢), (𝑣 +R 𝑓)〉))} | ||
| Definition | df-mul 11146* | Define multiplication over complex numbers. (Contributed by NM, 9-Aug-1995.) (New usage is discouraged.) |
| ⊢ · = {〈〈𝑥, 𝑦〉, 𝑧〉 ∣ ((𝑥 ∈ ℂ ∧ 𝑦 ∈ ℂ) ∧ ∃𝑤∃𝑣∃𝑢∃𝑓((𝑥 = 〈𝑤, 𝑣〉 ∧ 𝑦 = 〈𝑢, 𝑓〉) ∧ 𝑧 = 〈((𝑤 ·R 𝑢) +R (-1R ·R (𝑣 ·R 𝑓))), ((𝑣 ·R 𝑢) +R (𝑤 ·R 𝑓))〉))} | ||
| Definition | df-lt 11147* | Define 'less than' on the real subset of complex numbers. Proofs should typically use < instead; see df-ltxr 11279. (Contributed by NM, 22-Feb-1996.) (New usage is discouraged.) |
| ⊢ <ℝ = {〈𝑥, 𝑦〉 ∣ ((𝑥 ∈ ℝ ∧ 𝑦 ∈ ℝ) ∧ ∃𝑧∃𝑤((𝑥 = 〈𝑧, 0R〉 ∧ 𝑦 = 〈𝑤, 0R〉) ∧ 𝑧 <R 𝑤))} | ||
| Theorem | opelcn 11148 | Ordered pair membership in the class of complex numbers. (Contributed by NM, 14-May-1996.) (New usage is discouraged.) |
| ⊢ (〈𝐴, 𝐵〉 ∈ ℂ ↔ (𝐴 ∈ R ∧ 𝐵 ∈ R)) | ||
| Theorem | opelreal 11149 | Ordered pair membership in class of real subset of complex numbers. (Contributed by NM, 22-Feb-1996.) (New usage is discouraged.) |
| ⊢ (〈𝐴, 0R〉 ∈ ℝ ↔ 𝐴 ∈ R) | ||
| Theorem | elreal 11150* | Membership in class of real numbers. (Contributed by NM, 31-Mar-1996.) (New usage is discouraged.) |
| ⊢ (𝐴 ∈ ℝ ↔ ∃𝑥 ∈ R 〈𝑥, 0R〉 = 𝐴) | ||
| Theorem | elreal2 11151 | Ordered pair membership in the class of complex numbers. (Contributed by Mario Carneiro, 15-Jun-2013.) (New usage is discouraged.) |
| ⊢ (𝐴 ∈ ℝ ↔ ((1st ‘𝐴) ∈ R ∧ 𝐴 = 〈(1st ‘𝐴), 0R〉)) | ||
| Theorem | 0ncn 11152 | The empty set is not a complex number. Note: do not use this after the real number axioms are developed, since it is a construction-dependent property. (Contributed by NM, 2-May-1996.) (New usage is discouraged.) |
| ⊢ ¬ ∅ ∈ ℂ | ||
| Theorem | ltrelre 11153 | 'Less than' is a relation on real numbers. (Contributed by NM, 22-Feb-1996.) (New usage is discouraged.) |
| ⊢ <ℝ ⊆ (ℝ × ℝ) | ||
| Theorem | addcnsr 11154 | Addition of complex numbers in terms of signed reals. (Contributed by NM, 28-May-1995.) (New usage is discouraged.) |
| ⊢ (((𝐴 ∈ R ∧ 𝐵 ∈ R) ∧ (𝐶 ∈ R ∧ 𝐷 ∈ R)) → (〈𝐴, 𝐵〉 + 〈𝐶, 𝐷〉) = 〈(𝐴 +R 𝐶), (𝐵 +R 𝐷)〉) | ||
| Theorem | mulcnsr 11155 | Multiplication of complex numbers in terms of signed reals. (Contributed by NM, 9-Aug-1995.) (New usage is discouraged.) |
| ⊢ (((𝐴 ∈ R ∧ 𝐵 ∈ R) ∧ (𝐶 ∈ R ∧ 𝐷 ∈ R)) → (〈𝐴, 𝐵〉 · 〈𝐶, 𝐷〉) = 〈((𝐴 ·R 𝐶) +R (-1R ·R (𝐵 ·R 𝐷))), ((𝐵 ·R 𝐶) +R (𝐴 ·R 𝐷))〉) | ||
| Theorem | eqresr 11156 | Equality of real numbers in terms of intermediate signed reals. (Contributed by NM, 10-May-1996.) (New usage is discouraged.) |
| ⊢ 𝐴 ∈ V ⇒ ⊢ (〈𝐴, 0R〉 = 〈𝐵, 0R〉 ↔ 𝐴 = 𝐵) | ||
| Theorem | addresr 11157 | Addition of real numbers in terms of intermediate signed reals. (Contributed by NM, 10-May-1996.) (New usage is discouraged.) |
| ⊢ ((𝐴 ∈ R ∧ 𝐵 ∈ R) → (〈𝐴, 0R〉 + 〈𝐵, 0R〉) = 〈(𝐴 +R 𝐵), 0R〉) | ||
| Theorem | mulresr 11158 | Multiplication of real numbers in terms of intermediate signed reals. (Contributed by NM, 10-May-1996.) (New usage is discouraged.) |
| ⊢ ((𝐴 ∈ R ∧ 𝐵 ∈ R) → (〈𝐴, 0R〉 · 〈𝐵, 0R〉) = 〈(𝐴 ·R 𝐵), 0R〉) | ||
| Theorem | ltresr 11159 | Ordering of real subset of complex numbers in terms of signed reals. (Contributed by NM, 22-Feb-1996.) (New usage is discouraged.) |
| ⊢ (〈𝐴, 0R〉 <ℝ 〈𝐵, 0R〉 ↔ 𝐴 <R 𝐵) | ||
| Theorem | ltresr2 11160 | Ordering of real subset of complex numbers in terms of signed reals. (Contributed by NM, 22-Feb-1996.) (New usage is discouraged.) |
| ⊢ ((𝐴 ∈ ℝ ∧ 𝐵 ∈ ℝ) → (𝐴 <ℝ 𝐵 ↔ (1st ‘𝐴) <R (1st ‘𝐵))) | ||
| Theorem | dfcnqs 11161 | Technical trick to permit reuse of previous lemmas to prove arithmetic operation laws in ℂ from those in R. The trick involves qsid 8802, which shows that the coset of the converse membership relation (which is not an equivalence relation) acts as an identity divisor for the quotient set operation. This lets us "pretend" that ℂ is a quotient set, even though it is not (compare df-c 11140), and allows to reuse some of the equivalence class lemmas we developed for the transition from positive reals to signed reals, etc. (Contributed by NM, 13-Aug-1995.) (New usage is discouraged.) |
| ⊢ ℂ = ((R × R) / ◡ E ) | ||
| Theorem | addcnsrec 11162 | Technical trick to permit re-use of some equivalence class lemmas for operation laws. See dfcnqs 11161 and mulcnsrec 11163. (Contributed by NM, 13-Aug-1995.) (New usage is discouraged.) |
| ⊢ (((𝐴 ∈ R ∧ 𝐵 ∈ R) ∧ (𝐶 ∈ R ∧ 𝐷 ∈ R)) → ([〈𝐴, 𝐵〉]◡ E + [〈𝐶, 𝐷〉]◡ E ) = [〈(𝐴 +R 𝐶), (𝐵 +R 𝐷)〉]◡ E ) | ||
| Theorem | mulcnsrec 11163 |
Technical trick to permit re-use of some equivalence class lemmas for
operation laws. The trick involves ecid 8801,
which shows that the coset of
the converse membership relation (which is not an equivalence relation)
leaves a set unchanged. See also dfcnqs 11161.
Note: This is the last lemma (from which the axioms will be derived) in the construction of real and complex numbers. The construction starts at cnpi 10863. (Contributed by NM, 13-Aug-1995.) (New usage is discouraged.) |
| ⊢ (((𝐴 ∈ R ∧ 𝐵 ∈ R) ∧ (𝐶 ∈ R ∧ 𝐷 ∈ R)) → ([〈𝐴, 𝐵〉]◡ E · [〈𝐶, 𝐷〉]◡ E ) = [〈((𝐴 ·R 𝐶) +R (-1R ·R (𝐵 ·R 𝐷))), ((𝐵 ·R 𝐶) +R (𝐴 ·R 𝐷))〉]◡ E ) | ||
| Theorem | axaddf 11164 | Addition is an operation on the complex numbers. This theorem can be used as an alternate axiom for complex numbers in place of the less specific axaddcl 11170. This construction-dependent theorem should not be referenced directly; instead, use ax-addf 11213. (Contributed by NM, 8-Feb-2005.) (New usage is discouraged.) |
| ⊢ + :(ℂ × ℂ)⟶ℂ | ||
| Theorem | axmulf 11165 | Multiplication is an operation on the complex numbers. This is the construction-dependent version of ax-mulf 11214 and it should not be referenced outside the construction. We generally prefer to develop our theory using the less specific mulcl 11218. (Contributed by NM, 8-Feb-2005.) (New usage is discouraged.) |
| ⊢ · :(ℂ × ℂ)⟶ℂ | ||
| Theorem | axcnex 11166 | The complex numbers form a set. This axiom is redundant in the presence of the other axioms (see cnexALT 13007), but the proof requires the axiom of replacement, while the derivation from the construction here does not. Thus, we can avoid ax-rep 5254 in later theorems by invoking Axiom ax-cnex 11190 instead of cnexALT 13007. Use cnex 11215 instead. (Contributed by Mario Carneiro, 17-Nov-2014.) (New usage is discouraged.) |
| ⊢ ℂ ∈ V | ||
| Theorem | axresscn 11167 | The real numbers are a subset of the complex numbers. Axiom 1 of 22 for real and complex numbers, derived from ZF set theory. This construction-dependent theorem should not be referenced directly; instead, use ax-resscn 11191. (Contributed by NM, 1-Mar-1995.) (Proof shortened by Andrew Salmon, 12-Aug-2011.) (New usage is discouraged.) |
| ⊢ ℝ ⊆ ℂ | ||
| Theorem | ax1cn 11168 | 1 is a complex number. Axiom 2 of 22 for real and complex numbers, derived from ZF set theory. This construction-dependent theorem should not be referenced directly; instead, use ax-1cn 11192. (Contributed by NM, 12-Apr-2007.) (New usage is discouraged.) |
| ⊢ 1 ∈ ℂ | ||
| Theorem | axicn 11169 | i is a complex number. Axiom 3 of 22 for real and complex numbers, derived from ZF set theory. This construction-dependent theorem should not be referenced directly; instead, use ax-icn 11193. (Contributed by NM, 23-Feb-1996.) (New usage is discouraged.) |
| ⊢ i ∈ ℂ | ||
| Theorem | axaddcl 11170 | Closure law for addition of complex numbers. Axiom 4 of 22 for real and complex numbers, derived from ZF set theory. This construction-dependent theorem should not be referenced directly, nor should the proven axiom ax-addcl 11194 be used later. Instead, in most cases use addcl 11216. (Contributed by NM, 14-Jun-1995.) (New usage is discouraged.) |
| ⊢ ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ) → (𝐴 + 𝐵) ∈ ℂ) | ||
| Theorem | axaddrcl 11171 | Closure law for addition in the real subfield of complex numbers. Axiom 5 of 22 for real and complex numbers, derived from ZF set theory. This construction-dependent theorem should not be referenced directly, nor should the proven axiom ax-addrcl 11195 be used later. Instead, in most cases use readdcl 11217. (Contributed by NM, 31-Mar-1996.) (New usage is discouraged.) |
| ⊢ ((𝐴 ∈ ℝ ∧ 𝐵 ∈ ℝ) → (𝐴 + 𝐵) ∈ ℝ) | ||
| Theorem | axmulcl 11172 | Closure law for multiplication of complex numbers. Axiom 6 of 22 for real and complex numbers, derived from ZF set theory. This construction-dependent theorem should not be referenced directly, nor should the proven axiom ax-mulcl 11196 be used later. Instead, in most cases use mulcl 11218. (Contributed by NM, 10-Aug-1995.) (New usage is discouraged.) |
| ⊢ ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ) → (𝐴 · 𝐵) ∈ ℂ) | ||
| Theorem | axmulrcl 11173 | Closure law for multiplication in the real subfield of complex numbers. Axiom 7 of 22 for real and complex numbers, derived from ZF set theory. This construction-dependent theorem should not be referenced directly, nor should the proven axiom ax-mulrcl 11197 be used later. Instead, in most cases use remulcl 11219. (New usage is discouraged.) (Contributed by NM, 31-Mar-1996.) |
| ⊢ ((𝐴 ∈ ℝ ∧ 𝐵 ∈ ℝ) → (𝐴 · 𝐵) ∈ ℝ) | ||
| Theorem | axmulcom 11174 | Multiplication of complex numbers is commutative. Axiom 8 of 22 for real and complex numbers, derived from ZF set theory. This construction-dependent theorem should not be referenced directly, nor should the proven axiom ax-mulcom 11198 be used later. Instead, use mulcom 11220. (Contributed by NM, 31-Aug-1995.) (New usage is discouraged.) |
| ⊢ ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ) → (𝐴 · 𝐵) = (𝐵 · 𝐴)) | ||
| Theorem | axaddass 11175 | Addition of complex numbers is associative. This theorem transfers the associative laws for the real and imaginary signed real components of complex number pairs, to complex number addition itself. Axiom 9 of 22 for real and complex numbers, derived from ZF set theory. This construction-dependent theorem should not be referenced directly, nor should the proven axiom ax-addass 11199 be used later. Instead, use addass 11221. (Contributed by NM, 2-Sep-1995.) (New usage is discouraged.) |
| ⊢ ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ ∧ 𝐶 ∈ ℂ) → ((𝐴 + 𝐵) + 𝐶) = (𝐴 + (𝐵 + 𝐶))) | ||
| Theorem | axmulass 11176 | Multiplication of complex numbers is associative. Axiom 10 of 22 for real and complex numbers, derived from ZF set theory. This construction-dependent theorem should not be referenced directly; instead, use ax-mulass 11200. (Contributed by NM, 3-Sep-1995.) (New usage is discouraged.) |
| ⊢ ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ ∧ 𝐶 ∈ ℂ) → ((𝐴 · 𝐵) · 𝐶) = (𝐴 · (𝐵 · 𝐶))) | ||
| Theorem | axdistr 11177 | Distributive law for complex numbers (left-distributivity). Axiom 11 of 22 for real and complex numbers, derived from ZF set theory. This construction-dependent theorem should not be referenced directly, nor should the proven axiom ax-distr 11201 be used later. Instead, use adddi 11223. (Contributed by NM, 2-Sep-1995.) (New usage is discouraged.) |
| ⊢ ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ ∧ 𝐶 ∈ ℂ) → (𝐴 · (𝐵 + 𝐶)) = ((𝐴 · 𝐵) + (𝐴 · 𝐶))) | ||
| Theorem | axi2m1 11178 | i-squared equals -1 (expressed as i-squared plus 1 is 0). Axiom 12 of 22 for real and complex numbers, derived from ZF set theory. This construction-dependent theorem should not be referenced directly; instead, use ax-i2m1 11202. (Contributed by NM, 5-May-1996.) (New usage is discouraged.) |
| ⊢ ((i · i) + 1) = 0 | ||
| Theorem | ax1ne0 11179 | 1 and 0 are distinct. Axiom 13 of 22 for real and complex numbers, derived from ZF set theory. This construction-dependent theorem should not be referenced directly; instead, use ax-1ne0 11203. (Contributed by NM, 19-Mar-1996.) (New usage is discouraged.) |
| ⊢ 1 ≠ 0 | ||
| Theorem | ax1rid 11180 | 1 is an identity element for real multiplication. Axiom 14 of 22 for real and complex numbers, derived from ZF set theory. Weakened from the original axiom in the form of statement in mulrid 11238, based on ideas by Eric Schmidt. This construction-dependent theorem should not be referenced directly; instead, use ax-1rid 11204. (Contributed by Scott Fenton, 3-Jan-2013.) (New usage is discouraged.) |
| ⊢ (𝐴 ∈ ℝ → (𝐴 · 1) = 𝐴) | ||
| Theorem | axrnegex 11181* | Existence of negative of real number. Axiom 15 of 22 for real and complex numbers, derived from ZF set theory. This construction-dependent theorem should not be referenced directly; instead, use ax-rnegex 11205. (Contributed by NM, 15-May-1996.) (New usage is discouraged.) |
| ⊢ (𝐴 ∈ ℝ → ∃𝑥 ∈ ℝ (𝐴 + 𝑥) = 0) | ||
| Theorem | axrrecex 11182* | Existence of reciprocal of nonzero real number. Axiom 16 of 22 for real and complex numbers, derived from ZF set theory. This construction-dependent theorem should not be referenced directly; instead, use ax-rrecex 11206. (Contributed by NM, 15-May-1996.) (New usage is discouraged.) |
| ⊢ ((𝐴 ∈ ℝ ∧ 𝐴 ≠ 0) → ∃𝑥 ∈ ℝ (𝐴 · 𝑥) = 1) | ||
| Theorem | axcnre 11183* | A complex number can be expressed in terms of two reals. Definition 10-1.1(v) of [Gleason] p. 130. Axiom 17 of 22 for real and complex numbers, derived from ZF set theory. This construction-dependent theorem should not be referenced directly; instead, use ax-cnre 11207. (Contributed by NM, 13-May-1996.) (New usage is discouraged.) |
| ⊢ (𝐴 ∈ ℂ → ∃𝑥 ∈ ℝ ∃𝑦 ∈ ℝ 𝐴 = (𝑥 + (i · 𝑦))) | ||
| Theorem | axpre-lttri 11184 | Ordering on reals satisfies strict trichotomy. Axiom 18 of 22 for real and complex numbers, derived from ZF set theory. Note: The more general version for extended reals is axlttri 11311. This construction-dependent theorem should not be referenced directly; instead, use ax-pre-lttri 11208. (Contributed by NM, 19-May-1996.) (Revised by Mario Carneiro, 16-Jun-2013.) (New usage is discouraged.) |
| ⊢ ((𝐴 ∈ ℝ ∧ 𝐵 ∈ ℝ) → (𝐴 <ℝ 𝐵 ↔ ¬ (𝐴 = 𝐵 ∨ 𝐵 <ℝ 𝐴))) | ||
| Theorem | axpre-lttrn 11185 | Ordering on reals is transitive. Axiom 19 of 22 for real and complex numbers, derived from ZF set theory. Note: The more general version for extended reals is axlttrn 11312. This construction-dependent theorem should not be referenced directly; instead, use ax-pre-lttrn 11209. (Contributed by NM, 19-May-1996.) (Revised by Mario Carneiro, 16-Jun-2013.) (New usage is discouraged.) |
| ⊢ ((𝐴 ∈ ℝ ∧ 𝐵 ∈ ℝ ∧ 𝐶 ∈ ℝ) → ((𝐴 <ℝ 𝐵 ∧ 𝐵 <ℝ 𝐶) → 𝐴 <ℝ 𝐶)) | ||
| Theorem | axpre-ltadd 11186 | Ordering property of addition on reals. Axiom 20 of 22 for real and complex numbers, derived from ZF set theory. Note: The more general version for extended reals is axltadd 11313. This construction-dependent theorem should not be referenced directly; instead, use ax-pre-ltadd 11210. (Contributed by NM, 11-May-1996.) (New usage is discouraged.) |
| ⊢ ((𝐴 ∈ ℝ ∧ 𝐵 ∈ ℝ ∧ 𝐶 ∈ ℝ) → (𝐴 <ℝ 𝐵 → (𝐶 + 𝐴) <ℝ (𝐶 + 𝐵))) | ||
| Theorem | axpre-mulgt0 11187 | The product of two positive reals is positive. Axiom 21 of 22 for real and complex numbers, derived from ZF set theory. Note: The more general version for extended reals is axmulgt0 11314. This construction-dependent theorem should not be referenced directly; instead, use ax-pre-mulgt0 11211. (Contributed by NM, 13-May-1996.) (New usage is discouraged.) |
| ⊢ ((𝐴 ∈ ℝ ∧ 𝐵 ∈ ℝ) → ((0 <ℝ 𝐴 ∧ 0 <ℝ 𝐵) → 0 <ℝ (𝐴 · 𝐵))) | ||
| Theorem | axpre-sup 11188* | A nonempty, bounded-above set of reals has a supremum. Axiom 22 of 22 for real and complex numbers, derived from ZF set theory. Note: The more general version with ordering on extended reals is axsup 11315. This construction-dependent theorem should not be referenced directly; instead, use ax-pre-sup 11212. (Contributed by NM, 19-May-1996.) (Revised by Mario Carneiro, 16-Jun-2013.) (New usage is discouraged.) |
| ⊢ ((𝐴 ⊆ ℝ ∧ 𝐴 ≠ ∅ ∧ ∃𝑥 ∈ ℝ ∀𝑦 ∈ 𝐴 𝑦 <ℝ 𝑥) → ∃𝑥 ∈ ℝ (∀𝑦 ∈ 𝐴 ¬ 𝑥 <ℝ 𝑦 ∧ ∀𝑦 ∈ ℝ (𝑦 <ℝ 𝑥 → ∃𝑧 ∈ 𝐴 𝑦 <ℝ 𝑧))) | ||
| Theorem | wuncn 11189 | A weak universe containing ω contains the complex number construction. This theorem is construction-dependent in the literal sense, but will also be satisfied by any other reasonable implementation of the complex numbers. (Contributed by Mario Carneiro, 2-Jan-2017.) |
| ⊢ (𝜑 → 𝑈 ∈ WUni) & ⊢ (𝜑 → ω ∈ 𝑈) ⇒ ⊢ (𝜑 → ℂ ∈ 𝑈) | ||
| Axiom | ax-cnex 11190 | The complex numbers form a set. This axiom is redundant - see cnexALT 13007- but we provide this axiom because the justification theorem axcnex 11166 does not use ax-rep 5254 even though the redundancy proof does. Proofs should normally use cnex 11215 instead. (New usage is discouraged.) (Contributed by NM, 1-Mar-1995.) |
| ⊢ ℂ ∈ V | ||
| Axiom | ax-resscn 11191 | The real numbers are a subset of the complex numbers. Axiom 1 of 22 for real and complex numbers, justified by Theorem axresscn 11167. (Contributed by NM, 1-Mar-1995.) |
| ⊢ ℝ ⊆ ℂ | ||
| Axiom | ax-1cn 11192 | 1 is a complex number. Axiom 2 of 22 for real and complex numbers, justified by Theorem ax1cn 11168. (Contributed by NM, 1-Mar-1995.) |
| ⊢ 1 ∈ ℂ | ||
| Axiom | ax-icn 11193 | i is a complex number. Axiom 3 of 22 for real and complex numbers, justified by Theorem axicn 11169. (Contributed by NM, 1-Mar-1995.) |
| ⊢ i ∈ ℂ | ||
| Axiom | ax-addcl 11194 | Closure law for addition of complex numbers. Axiom 4 of 22 for real and complex numbers, justified by Theorem axaddcl 11170. Proofs should normally use addcl 11216 instead, which asserts the same thing but follows our naming conventions for closures. (New usage is discouraged.) (Contributed by NM, 22-Nov-1994.) |
| ⊢ ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ) → (𝐴 + 𝐵) ∈ ℂ) | ||
| Axiom | ax-addrcl 11195 | Closure law for addition in the real subfield of complex numbers. Axiom 6 of 23 for real and complex numbers, justified by Theorem axaddrcl 11171. Proofs should normally use readdcl 11217 instead. (New usage is discouraged.) (Contributed by NM, 22-Nov-1994.) |
| ⊢ ((𝐴 ∈ ℝ ∧ 𝐵 ∈ ℝ) → (𝐴 + 𝐵) ∈ ℝ) | ||
| Axiom | ax-mulcl 11196 | Closure law for multiplication of complex numbers. Axiom 6 of 22 for real and complex numbers, justified by Theorem axmulcl 11172. Proofs should normally use mulcl 11218 instead. (New usage is discouraged.) (Contributed by NM, 22-Nov-1994.) |
| ⊢ ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ) → (𝐴 · 𝐵) ∈ ℂ) | ||
| Axiom | ax-mulrcl 11197 | Closure law for multiplication in the real subfield of complex numbers. Axiom 7 of 22 for real and complex numbers, justified by Theorem axmulrcl 11173. Proofs should normally use remulcl 11219 instead. (New usage is discouraged.) (Contributed by NM, 22-Nov-1994.) |
| ⊢ ((𝐴 ∈ ℝ ∧ 𝐵 ∈ ℝ) → (𝐴 · 𝐵) ∈ ℝ) | ||
| Axiom | ax-mulcom 11198 | Multiplication of complex numbers is commutative. Axiom 8 of 22 for real and complex numbers, justified by Theorem axmulcom 11174. Proofs should normally use mulcom 11220 instead. (New usage is discouraged.) (Contributed by NM, 22-Nov-1994.) |
| ⊢ ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ) → (𝐴 · 𝐵) = (𝐵 · 𝐴)) | ||
| Axiom | ax-addass 11199 | Addition of complex numbers is associative. Axiom 9 of 22 for real and complex numbers, justified by Theorem axaddass 11175. Proofs should normally use addass 11221 instead. (New usage is discouraged.) (Contributed by NM, 22-Nov-1994.) |
| ⊢ ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ ∧ 𝐶 ∈ ℂ) → ((𝐴 + 𝐵) + 𝐶) = (𝐴 + (𝐵 + 𝐶))) | ||
| Axiom | ax-mulass 11200 | Multiplication of complex numbers is associative. Axiom 10 of 22 for real and complex numbers, justified by Theorem axmulass 11176. Proofs should normally use mulass 11222 instead. (New usage is discouraged.) (Contributed by NM, 22-Nov-1994.) |
| ⊢ ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ ∧ 𝐶 ∈ ℂ) → ((𝐴 · 𝐵) · 𝐶) = (𝐴 · (𝐵 · 𝐶))) | ||
| < Previous Next > |
| Copyright terms: Public domain | < Previous Next > |