MPE Home Metamath Proof Explorer < Previous   Next >
Nearby theorems
Mirrors  >  Home  >  MPE Home  >  Th. List  >  addsqnreup Structured version   Visualization version   GIF version

Theorem addsqnreup 27406
Description: There is no unique decomposition of a complex number as a sum of a complex number and a square of a complex number.

Remark: This theorem, together with addsq2reu 27403, is a real life example (about a numerical property) showing that the pattern ∃!𝑎𝐴∃!𝑏𝐵𝜑 does not necessarily mean "There are unique sets 𝑎 and 𝑏 fulfilling 𝜑"). See also comments for df-eu 2568 and 2eu4 2654.

In the case of decompositions of complex numbers as a sum of a complex number and a square of a complex number, the only/unique complex number to which the square of a unique complex number is added yields in the given complex number is the given number itself, and the unique complex number to be squared is 0 (see comment for addsq2reu 27403). There are, however, complex numbers to which the square of more than one other complex numbers can be added to yield the given complex number (see addsqrexnreu 27405). For example, ⟨1, (√‘(𝐶 − 1))⟩ and ⟨1, -(√‘(𝐶 − 1))⟩ are two different decompositions of 𝐶 (if 𝐶 ≠ 1). Therefore, there is no unique decomposition of any complex number as a sum of a complex number and a square of a complex number, as generally proved by this theorem.

As a consequence, a theorem must claim the existence of a unique pair of sets to express "There are unique 𝑎 and 𝑏 so that .." (more formally ∃!𝑝 ∈ (𝐴 × 𝐵)𝜑 with 𝑝 = ⟨𝑎, 𝑏), or by showing (∃!𝑥𝐴𝑦𝐵𝜑 ∧ ∃!𝑦𝐵𝑥𝐴𝜑) (see 2reu4 4498 resp. 2eu4 2654). These two representations are equivalent (see opreu2reurex 6283). An analogon of this theorem using the latter variant is given in addsqn2reurex2 27408. In some cases, however, the variant with (ordered!) pairs may be possible only for ordered sets (like or ) and claiming that the first component is less than or equal to the second component (see, for example, 2sqreunnltb 27424 and 2sqreuopb 27431). Alternatively, (proper) unordered pairs can be used: ∃!𝑝𝑒𝒫 𝐴((♯‘𝑝) = 2 ∧ 𝜑), or, using the definition of proper pairs: ∃!𝑝 ∈ (Pairsproper𝐴)𝜑 (see, for example, inlinecirc02preu 48768). (Contributed by AV, 21-Jun-2023.)

Assertion
Ref Expression
addsqnreup (𝐶 ∈ ℂ → ¬ ∃!𝑝 ∈ (ℂ × ℂ)((1st𝑝) + ((2nd𝑝)↑2)) = 𝐶)
Distinct variable group:   𝐶,𝑝

Proof of Theorem addsqnreup
StepHypRef Expression
1 ax-1cn 11187 . . . . . . 7 1 ∈ ℂ
2 0cn 11227 . . . . . . 7 0 ∈ ℂ
3 opelxpi 5691 . . . . . . 7 ((1 ∈ ℂ ∧ 0 ∈ ℂ) → ⟨1, 0⟩ ∈ (ℂ × ℂ))
41, 2, 3mp2an 692 . . . . . 6 ⟨1, 0⟩ ∈ (ℂ × ℂ)
5 3cn 12321 . . . . . . . 8 3 ∈ ℂ
65negcli 11551 . . . . . . 7 -3 ∈ ℂ
7 2cn 12315 . . . . . . 7 2 ∈ ℂ
8 opelxpi 5691 . . . . . . 7 ((-3 ∈ ℂ ∧ 2 ∈ ℂ) → ⟨-3, 2⟩ ∈ (ℂ × ℂ))
96, 7, 8mp2an 692 . . . . . 6 ⟨-3, 2⟩ ∈ (ℂ × ℂ)
10 0ne2 12447 . . . . . . . 8 0 ≠ 2
1110olci 866 . . . . . . 7 (1 ≠ -3 ∨ 0 ≠ 2)
12 1ex 11231 . . . . . . . 8 1 ∈ V
13 c0ex 11229 . . . . . . . 8 0 ∈ V
1412, 13opthne 5457 . . . . . . 7 (⟨1, 0⟩ ≠ ⟨-3, 2⟩ ↔ (1 ≠ -3 ∨ 0 ≠ 2))
1511, 14mpbir 231 . . . . . 6 ⟨1, 0⟩ ≠ ⟨-3, 2⟩
164, 9, 153pm3.2i 1340 . . . . 5 (⟨1, 0⟩ ∈ (ℂ × ℂ) ∧ ⟨-3, 2⟩ ∈ (ℂ × ℂ) ∧ ⟨1, 0⟩ ≠ ⟨-3, 2⟩)
1712, 13op1st 7996 . . . . . . . 8 (1st ‘⟨1, 0⟩) = 1
1812, 13op2nd 7997 . . . . . . . . . 10 (2nd ‘⟨1, 0⟩) = 0
1918oveq1i 7415 . . . . . . . . 9 ((2nd ‘⟨1, 0⟩)↑2) = (0↑2)
20 sq0 14210 . . . . . . . . 9 (0↑2) = 0
2119, 20eqtri 2758 . . . . . . . 8 ((2nd ‘⟨1, 0⟩)↑2) = 0
2217, 21oveq12i 7417 . . . . . . 7 ((1st ‘⟨1, 0⟩) + ((2nd ‘⟨1, 0⟩)↑2)) = (1 + 0)
23 1p0e1 12364 . . . . . . 7 (1 + 0) = 1
2422, 23eqtri 2758 . . . . . 6 ((1st ‘⟨1, 0⟩) + ((2nd ‘⟨1, 0⟩)↑2)) = 1
25 negex 11480 . . . . . . . . 9 -3 ∈ V
26 2ex 12317 . . . . . . . . 9 2 ∈ V
2725, 26op1st 7996 . . . . . . . 8 (1st ‘⟨-3, 2⟩) = -3
2825, 26op2nd 7997 . . . . . . . . . 10 (2nd ‘⟨-3, 2⟩) = 2
2928oveq1i 7415 . . . . . . . . 9 ((2nd ‘⟨-3, 2⟩)↑2) = (2↑2)
30 sq2 14215 . . . . . . . . 9 (2↑2) = 4
3129, 30eqtri 2758 . . . . . . . 8 ((2nd ‘⟨-3, 2⟩)↑2) = 4
3227, 31oveq12i 7417 . . . . . . 7 ((1st ‘⟨-3, 2⟩) + ((2nd ‘⟨-3, 2⟩)↑2)) = (-3 + 4)
33 4cn 12325 . . . . . . . 8 4 ∈ ℂ
3433, 5negsubi 11561 . . . . . . . . 9 (4 + -3) = (4 − 3)
35 3p1e4 12385 . . . . . . . . . 10 (3 + 1) = 4
3633, 5, 1, 35subaddrii 11572 . . . . . . . . 9 (4 − 3) = 1
3734, 36eqtri 2758 . . . . . . . 8 (4 + -3) = 1
3833, 6, 37addcomli 11427 . . . . . . 7 (-3 + 4) = 1
3932, 38eqtri 2758 . . . . . 6 ((1st ‘⟨-3, 2⟩) + ((2nd ‘⟨-3, 2⟩)↑2)) = 1
4024, 39pm3.2i 470 . . . . 5 (((1st ‘⟨1, 0⟩) + ((2nd ‘⟨1, 0⟩)↑2)) = 1 ∧ ((1st ‘⟨-3, 2⟩) + ((2nd ‘⟨-3, 2⟩)↑2)) = 1)
41 fveq2 6876 . . . . . . . 8 (𝑝 = ⟨1, 0⟩ → (1st𝑝) = (1st ‘⟨1, 0⟩))
42 fveq2 6876 . . . . . . . . 9 (𝑝 = ⟨1, 0⟩ → (2nd𝑝) = (2nd ‘⟨1, 0⟩))
4342oveq1d 7420 . . . . . . . 8 (𝑝 = ⟨1, 0⟩ → ((2nd𝑝)↑2) = ((2nd ‘⟨1, 0⟩)↑2))
4441, 43oveq12d 7423 . . . . . . 7 (𝑝 = ⟨1, 0⟩ → ((1st𝑝) + ((2nd𝑝)↑2)) = ((1st ‘⟨1, 0⟩) + ((2nd ‘⟨1, 0⟩)↑2)))
4544eqeq1d 2737 . . . . . 6 (𝑝 = ⟨1, 0⟩ → (((1st𝑝) + ((2nd𝑝)↑2)) = 1 ↔ ((1st ‘⟨1, 0⟩) + ((2nd ‘⟨1, 0⟩)↑2)) = 1))
46 fveq2 6876 . . . . . . . 8 (𝑝 = ⟨-3, 2⟩ → (1st𝑝) = (1st ‘⟨-3, 2⟩))
47 fveq2 6876 . . . . . . . . 9 (𝑝 = ⟨-3, 2⟩ → (2nd𝑝) = (2nd ‘⟨-3, 2⟩))
4847oveq1d 7420 . . . . . . . 8 (𝑝 = ⟨-3, 2⟩ → ((2nd𝑝)↑2) = ((2nd ‘⟨-3, 2⟩)↑2))
4946, 48oveq12d 7423 . . . . . . 7 (𝑝 = ⟨-3, 2⟩ → ((1st𝑝) + ((2nd𝑝)↑2)) = ((1st ‘⟨-3, 2⟩) + ((2nd ‘⟨-3, 2⟩)↑2)))
5049eqeq1d 2737 . . . . . 6 (𝑝 = ⟨-3, 2⟩ → (((1st𝑝) + ((2nd𝑝)↑2)) = 1 ↔ ((1st ‘⟨-3, 2⟩) + ((2nd ‘⟨-3, 2⟩)↑2)) = 1))
5145, 502nreu 4419 . . . . 5 ((⟨1, 0⟩ ∈ (ℂ × ℂ) ∧ ⟨-3, 2⟩ ∈ (ℂ × ℂ) ∧ ⟨1, 0⟩ ≠ ⟨-3, 2⟩) → ((((1st ‘⟨1, 0⟩) + ((2nd ‘⟨1, 0⟩)↑2)) = 1 ∧ ((1st ‘⟨-3, 2⟩) + ((2nd ‘⟨-3, 2⟩)↑2)) = 1) → ¬ ∃!𝑝 ∈ (ℂ × ℂ)((1st𝑝) + ((2nd𝑝)↑2)) = 1))
5216, 40, 51mp2 9 . . . 4 ¬ ∃!𝑝 ∈ (ℂ × ℂ)((1st𝑝) + ((2nd𝑝)↑2)) = 1
53 eqeq2 2747 . . . . 5 (𝐶 = 1 → (((1st𝑝) + ((2nd𝑝)↑2)) = 𝐶 ↔ ((1st𝑝) + ((2nd𝑝)↑2)) = 1))
5453reubidv 3377 . . . 4 (𝐶 = 1 → (∃!𝑝 ∈ (ℂ × ℂ)((1st𝑝) + ((2nd𝑝)↑2)) = 𝐶 ↔ ∃!𝑝 ∈ (ℂ × ℂ)((1st𝑝) + ((2nd𝑝)↑2)) = 1))
5552, 54mtbiri 327 . . 3 (𝐶 = 1 → ¬ ∃!𝑝 ∈ (ℂ × ℂ)((1st𝑝) + ((2nd𝑝)↑2)) = 𝐶)
5655a1d 25 . 2 (𝐶 = 1 → (𝐶 ∈ ℂ → ¬ ∃!𝑝 ∈ (ℂ × ℂ)((1st𝑝) + ((2nd𝑝)↑2)) = 𝐶))
57 id 22 . . . . . . 7 (𝐶 ∈ ℂ → 𝐶 ∈ ℂ)
58 0cnd 11228 . . . . . . 7 (𝐶 ∈ ℂ → 0 ∈ ℂ)
5957, 58opelxpd 5693 . . . . . 6 (𝐶 ∈ ℂ → ⟨𝐶, 0⟩ ∈ (ℂ × ℂ))
6059adantr 480 . . . . 5 ((𝐶 ∈ ℂ ∧ 𝐶 ≠ 1) → ⟨𝐶, 0⟩ ∈ (ℂ × ℂ))
61 1cnd 11230 . . . . . . 7 (𝐶 ∈ ℂ → 1 ∈ ℂ)
62 peano2cnm 11549 . . . . . . . 8 (𝐶 ∈ ℂ → (𝐶 − 1) ∈ ℂ)
6362sqrtcld 15456 . . . . . . 7 (𝐶 ∈ ℂ → (√‘(𝐶 − 1)) ∈ ℂ)
6461, 63opelxpd 5693 . . . . . 6 (𝐶 ∈ ℂ → ⟨1, (√‘(𝐶 − 1))⟩ ∈ (ℂ × ℂ))
6564adantr 480 . . . . 5 ((𝐶 ∈ ℂ ∧ 𝐶 ≠ 1) → ⟨1, (√‘(𝐶 − 1))⟩ ∈ (ℂ × ℂ))
66 animorrl 982 . . . . . 6 ((𝐶 ∈ ℂ ∧ 𝐶 ≠ 1) → (𝐶 ≠ 1 ∨ 0 ≠ (√‘(𝐶 − 1))))
67 0cnd 11228 . . . . . . 7 (𝐶 ≠ 1 → 0 ∈ ℂ)
68 opthneg 5456 . . . . . . 7 ((𝐶 ∈ ℂ ∧ 0 ∈ ℂ) → (⟨𝐶, 0⟩ ≠ ⟨1, (√‘(𝐶 − 1))⟩ ↔ (𝐶 ≠ 1 ∨ 0 ≠ (√‘(𝐶 − 1)))))
6967, 68sylan2 593 . . . . . 6 ((𝐶 ∈ ℂ ∧ 𝐶 ≠ 1) → (⟨𝐶, 0⟩ ≠ ⟨1, (√‘(𝐶 − 1))⟩ ↔ (𝐶 ≠ 1 ∨ 0 ≠ (√‘(𝐶 − 1)))))
7066, 69mpbird 257 . . . . 5 ((𝐶 ∈ ℂ ∧ 𝐶 ≠ 1) → ⟨𝐶, 0⟩ ≠ ⟨1, (√‘(𝐶 − 1))⟩)
7160, 65, 703jca 1128 . . . 4 ((𝐶 ∈ ℂ ∧ 𝐶 ≠ 1) → (⟨𝐶, 0⟩ ∈ (ℂ × ℂ) ∧ ⟨1, (√‘(𝐶 − 1))⟩ ∈ (ℂ × ℂ) ∧ ⟨𝐶, 0⟩ ≠ ⟨1, (√‘(𝐶 − 1))⟩))
72 op1stg 8000 . . . . . . . . 9 ((𝐶 ∈ ℂ ∧ 0 ∈ ℂ) → (1st ‘⟨𝐶, 0⟩) = 𝐶)
7358, 72mpdan 687 . . . . . . . 8 (𝐶 ∈ ℂ → (1st ‘⟨𝐶, 0⟩) = 𝐶)
74 op2ndg 8001 . . . . . . . . . 10 ((𝐶 ∈ ℂ ∧ 0 ∈ ℂ) → (2nd ‘⟨𝐶, 0⟩) = 0)
7558, 74mpdan 687 . . . . . . . . 9 (𝐶 ∈ ℂ → (2nd ‘⟨𝐶, 0⟩) = 0)
7675sq0id 14212 . . . . . . . 8 (𝐶 ∈ ℂ → ((2nd ‘⟨𝐶, 0⟩)↑2) = 0)
7773, 76oveq12d 7423 . . . . . . 7 (𝐶 ∈ ℂ → ((1st ‘⟨𝐶, 0⟩) + ((2nd ‘⟨𝐶, 0⟩)↑2)) = (𝐶 + 0))
78 addrid 11415 . . . . . . 7 (𝐶 ∈ ℂ → (𝐶 + 0) = 𝐶)
7977, 78eqtrd 2770 . . . . . 6 (𝐶 ∈ ℂ → ((1st ‘⟨𝐶, 0⟩) + ((2nd ‘⟨𝐶, 0⟩)↑2)) = 𝐶)
80 op1stg 8000 . . . . . . . . 9 ((1 ∈ ℂ ∧ (√‘(𝐶 − 1)) ∈ ℂ) → (1st ‘⟨1, (√‘(𝐶 − 1))⟩) = 1)
8161, 63, 80syl2anc 584 . . . . . . . 8 (𝐶 ∈ ℂ → (1st ‘⟨1, (√‘(𝐶 − 1))⟩) = 1)
82 op2ndg 8001 . . . . . . . . . . 11 ((1 ∈ ℂ ∧ (√‘(𝐶 − 1)) ∈ ℂ) → (2nd ‘⟨1, (√‘(𝐶 − 1))⟩) = (√‘(𝐶 − 1)))
8361, 63, 82syl2anc 584 . . . . . . . . . 10 (𝐶 ∈ ℂ → (2nd ‘⟨1, (√‘(𝐶 − 1))⟩) = (√‘(𝐶 − 1)))
8483oveq1d 7420 . . . . . . . . 9 (𝐶 ∈ ℂ → ((2nd ‘⟨1, (√‘(𝐶 − 1))⟩)↑2) = ((√‘(𝐶 − 1))↑2))
8562sqsqrtd 15458 . . . . . . . . 9 (𝐶 ∈ ℂ → ((√‘(𝐶 − 1))↑2) = (𝐶 − 1))
8684, 85eqtrd 2770 . . . . . . . 8 (𝐶 ∈ ℂ → ((2nd ‘⟨1, (√‘(𝐶 − 1))⟩)↑2) = (𝐶 − 1))
8781, 86oveq12d 7423 . . . . . . 7 (𝐶 ∈ ℂ → ((1st ‘⟨1, (√‘(𝐶 − 1))⟩) + ((2nd ‘⟨1, (√‘(𝐶 − 1))⟩)↑2)) = (1 + (𝐶 − 1)))
8861, 57pncan3d 11597 . . . . . . 7 (𝐶 ∈ ℂ → (1 + (𝐶 − 1)) = 𝐶)
8987, 88eqtrd 2770 . . . . . 6 (𝐶 ∈ ℂ → ((1st ‘⟨1, (√‘(𝐶 − 1))⟩) + ((2nd ‘⟨1, (√‘(𝐶 − 1))⟩)↑2)) = 𝐶)
9079, 89jca 511 . . . . 5 (𝐶 ∈ ℂ → (((1st ‘⟨𝐶, 0⟩) + ((2nd ‘⟨𝐶, 0⟩)↑2)) = 𝐶 ∧ ((1st ‘⟨1, (√‘(𝐶 − 1))⟩) + ((2nd ‘⟨1, (√‘(𝐶 − 1))⟩)↑2)) = 𝐶))
9190adantr 480 . . . 4 ((𝐶 ∈ ℂ ∧ 𝐶 ≠ 1) → (((1st ‘⟨𝐶, 0⟩) + ((2nd ‘⟨𝐶, 0⟩)↑2)) = 𝐶 ∧ ((1st ‘⟨1, (√‘(𝐶 − 1))⟩) + ((2nd ‘⟨1, (√‘(𝐶 − 1))⟩)↑2)) = 𝐶))
92 fveq2 6876 . . . . . . 7 (𝑝 = ⟨𝐶, 0⟩ → (1st𝑝) = (1st ‘⟨𝐶, 0⟩))
93 fveq2 6876 . . . . . . . 8 (𝑝 = ⟨𝐶, 0⟩ → (2nd𝑝) = (2nd ‘⟨𝐶, 0⟩))
9493oveq1d 7420 . . . . . . 7 (𝑝 = ⟨𝐶, 0⟩ → ((2nd𝑝)↑2) = ((2nd ‘⟨𝐶, 0⟩)↑2))
9592, 94oveq12d 7423 . . . . . 6 (𝑝 = ⟨𝐶, 0⟩ → ((1st𝑝) + ((2nd𝑝)↑2)) = ((1st ‘⟨𝐶, 0⟩) + ((2nd ‘⟨𝐶, 0⟩)↑2)))
9695eqeq1d 2737 . . . . 5 (𝑝 = ⟨𝐶, 0⟩ → (((1st𝑝) + ((2nd𝑝)↑2)) = 𝐶 ↔ ((1st ‘⟨𝐶, 0⟩) + ((2nd ‘⟨𝐶, 0⟩)↑2)) = 𝐶))
97 fveq2 6876 . . . . . . 7 (𝑝 = ⟨1, (√‘(𝐶 − 1))⟩ → (1st𝑝) = (1st ‘⟨1, (√‘(𝐶 − 1))⟩))
98 fveq2 6876 . . . . . . . 8 (𝑝 = ⟨1, (√‘(𝐶 − 1))⟩ → (2nd𝑝) = (2nd ‘⟨1, (√‘(𝐶 − 1))⟩))
9998oveq1d 7420 . . . . . . 7 (𝑝 = ⟨1, (√‘(𝐶 − 1))⟩ → ((2nd𝑝)↑2) = ((2nd ‘⟨1, (√‘(𝐶 − 1))⟩)↑2))
10097, 99oveq12d 7423 . . . . . 6 (𝑝 = ⟨1, (√‘(𝐶 − 1))⟩ → ((1st𝑝) + ((2nd𝑝)↑2)) = ((1st ‘⟨1, (√‘(𝐶 − 1))⟩) + ((2nd ‘⟨1, (√‘(𝐶 − 1))⟩)↑2)))
101100eqeq1d 2737 . . . . 5 (𝑝 = ⟨1, (√‘(𝐶 − 1))⟩ → (((1st𝑝) + ((2nd𝑝)↑2)) = 𝐶 ↔ ((1st ‘⟨1, (√‘(𝐶 − 1))⟩) + ((2nd ‘⟨1, (√‘(𝐶 − 1))⟩)↑2)) = 𝐶))
10296, 1012nreu 4419 . . . 4 ((⟨𝐶, 0⟩ ∈ (ℂ × ℂ) ∧ ⟨1, (√‘(𝐶 − 1))⟩ ∈ (ℂ × ℂ) ∧ ⟨𝐶, 0⟩ ≠ ⟨1, (√‘(𝐶 − 1))⟩) → ((((1st ‘⟨𝐶, 0⟩) + ((2nd ‘⟨𝐶, 0⟩)↑2)) = 𝐶 ∧ ((1st ‘⟨1, (√‘(𝐶 − 1))⟩) + ((2nd ‘⟨1, (√‘(𝐶 − 1))⟩)↑2)) = 𝐶) → ¬ ∃!𝑝 ∈ (ℂ × ℂ)((1st𝑝) + ((2nd𝑝)↑2)) = 𝐶))
10371, 91, 102sylc 65 . . 3 ((𝐶 ∈ ℂ ∧ 𝐶 ≠ 1) → ¬ ∃!𝑝 ∈ (ℂ × ℂ)((1st𝑝) + ((2nd𝑝)↑2)) = 𝐶)
104103expcom 413 . 2 (𝐶 ≠ 1 → (𝐶 ∈ ℂ → ¬ ∃!𝑝 ∈ (ℂ × ℂ)((1st𝑝) + ((2nd𝑝)↑2)) = 𝐶))
10556, 104pm2.61ine 3015 1 (𝐶 ∈ ℂ → ¬ ∃!𝑝 ∈ (ℂ × ℂ)((1st𝑝) + ((2nd𝑝)↑2)) = 𝐶)
Colors of variables: wff setvar class
Syntax hints:  ¬ wn 3  wi 4  wb 206  wa 395  wo 847  w3a 1086   = wceq 1540  wcel 2108  wne 2932  ∃!wreu 3357  cop 4607   × cxp 5652  cfv 6531  (class class class)co 7405  1st c1st 7986  2nd c2nd 7987  cc 11127  0cc0 11129  1c1 11130   + caddc 11132  cmin 11466  -cneg 11467  2c2 12295  3c3 12296  4c4 12297  cexp 14079  csqrt 15252
This theorem was proved from axioms:  ax-mp 5  ax-1 6  ax-2 7  ax-3 8  ax-gen 1795  ax-4 1809  ax-5 1910  ax-6 1967  ax-7 2007  ax-8 2110  ax-9 2118  ax-10 2141  ax-11 2157  ax-12 2177  ax-ext 2707  ax-sep 5266  ax-nul 5276  ax-pow 5335  ax-pr 5402  ax-un 7729  ax-cnex 11185  ax-resscn 11186  ax-1cn 11187  ax-icn 11188  ax-addcl 11189  ax-addrcl 11190  ax-mulcl 11191  ax-mulrcl 11192  ax-mulcom 11193  ax-addass 11194  ax-mulass 11195  ax-distr 11196  ax-i2m1 11197  ax-1ne0 11198  ax-1rid 11199  ax-rnegex 11200  ax-rrecex 11201  ax-cnre 11202  ax-pre-lttri 11203  ax-pre-lttrn 11204  ax-pre-ltadd 11205  ax-pre-mulgt0 11206  ax-pre-sup 11207
This theorem depends on definitions:  df-bi 207  df-an 396  df-or 848  df-3or 1087  df-3an 1088  df-tru 1543  df-fal 1553  df-ex 1780  df-nf 1784  df-sb 2065  df-mo 2539  df-eu 2568  df-clab 2714  df-cleq 2727  df-clel 2809  df-nfc 2885  df-ne 2933  df-nel 3037  df-ral 3052  df-rex 3061  df-rmo 3359  df-reu 3360  df-rab 3416  df-v 3461  df-sbc 3766  df-csb 3875  df-dif 3929  df-un 3931  df-in 3933  df-ss 3943  df-pss 3946  df-nul 4309  df-if 4501  df-pw 4577  df-sn 4602  df-pr 4604  df-op 4608  df-uni 4884  df-iun 4969  df-br 5120  df-opab 5182  df-mpt 5202  df-tr 5230  df-id 5548  df-eprel 5553  df-po 5561  df-so 5562  df-fr 5606  df-we 5608  df-xp 5660  df-rel 5661  df-cnv 5662  df-co 5663  df-dm 5664  df-rn 5665  df-res 5666  df-ima 5667  df-pred 6290  df-ord 6355  df-on 6356  df-lim 6357  df-suc 6358  df-iota 6484  df-fun 6533  df-fn 6534  df-f 6535  df-f1 6536  df-fo 6537  df-f1o 6538  df-fv 6539  df-riota 7362  df-ov 7408  df-oprab 7409  df-mpo 7410  df-om 7862  df-1st 7988  df-2nd 7989  df-frecs 8280  df-wrecs 8311  df-recs 8385  df-rdg 8424  df-er 8719  df-en 8960  df-dom 8961  df-sdom 8962  df-sup 9454  df-pnf 11271  df-mnf 11272  df-xr 11273  df-ltxr 11274  df-le 11275  df-sub 11468  df-neg 11469  df-div 11895  df-nn 12241  df-2 12303  df-3 12304  df-4 12305  df-n0 12502  df-z 12589  df-uz 12853  df-rp 13009  df-seq 14020  df-exp 14080  df-cj 15118  df-re 15119  df-im 15120  df-sqrt 15254  df-abs 15255
This theorem is referenced by: (None)
  Copyright terms: Public domain W3C validator