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

Definition df-sqrt 14594
Description: Define a function whose value is the square root of a complex number. For example, (√‘25) = 5 (ex-sqrt 28233).

Since (𝑦↑2) = 𝑥 iff (-𝑦↑2) = 𝑥, we ensure uniqueness by restricting the range to numbers with positive real part, or numbers with 0 real part and nonnegative imaginary part. A description can be found under "Principal square root of a complex number" at http://en.wikipedia.org/wiki/Square_root 28233. The square root symbol was introduced in 1525 by Christoff Rudolff.

See sqrtcl 14721 for its closure, sqrtval 14596 for its value, sqrtth 14724 and sqsqrti 14735 for its relationship to squares, and sqrt11i 14744 for uniqueness. (Contributed by NM, 27-Jul-1999.) (Revised by Mario Carneiro, 8-Jul-2013.)

Assertion
Ref Expression
df-sqrt √ = (𝑥 ∈ ℂ ↦ (𝑦 ∈ ℂ ((𝑦↑2) = 𝑥 ∧ 0 ≤ (ℜ‘𝑦) ∧ (i · 𝑦) ∉ ℝ+)))
Distinct variable group:   𝑥,𝑦

Detailed syntax breakdown of Definition df-sqrt
StepHypRef Expression
1 csqrt 14592 . 2 class
2 vx . . 3 setvar 𝑥
3 cc 10535 . . 3 class
4 vy . . . . . . . 8 setvar 𝑦
54cv 1536 . . . . . . 7 class 𝑦
6 c2 11693 . . . . . . 7 class 2
7 cexp 13430 . . . . . . 7 class
85, 6, 7co 7156 . . . . . 6 class (𝑦↑2)
92cv 1536 . . . . . 6 class 𝑥
108, 9wceq 1537 . . . . 5 wff (𝑦↑2) = 𝑥
11 cc0 10537 . . . . . 6 class 0
12 cre 14456 . . . . . . 7 class
135, 12cfv 6355 . . . . . 6 class (ℜ‘𝑦)
14 cle 10676 . . . . . 6 class
1511, 13, 14wbr 5066 . . . . 5 wff 0 ≤ (ℜ‘𝑦)
16 ci 10539 . . . . . . 7 class i
17 cmul 10542 . . . . . . 7 class ·
1816, 5, 17co 7156 . . . . . 6 class (i · 𝑦)
19 crp 12390 . . . . . 6 class +
2018, 19wnel 3123 . . . . 5 wff (i · 𝑦) ∉ ℝ+
2110, 15, 20w3a 1083 . . . 4 wff ((𝑦↑2) = 𝑥 ∧ 0 ≤ (ℜ‘𝑦) ∧ (i · 𝑦) ∉ ℝ+)
2221, 4, 3crio 7113 . . 3 class (𝑦 ∈ ℂ ((𝑦↑2) = 𝑥 ∧ 0 ≤ (ℜ‘𝑦) ∧ (i · 𝑦) ∉ ℝ+))
232, 3, 22cmpt 5146 . 2 class (𝑥 ∈ ℂ ↦ (𝑦 ∈ ℂ ((𝑦↑2) = 𝑥 ∧ 0 ≤ (ℜ‘𝑦) ∧ (i · 𝑦) ∉ ℝ+)))
241, 23wceq 1537 1 wff √ = (𝑥 ∈ ℂ ↦ (𝑦 ∈ ℂ ((𝑦↑2) = 𝑥 ∧ 0 ≤ (ℜ‘𝑦) ∧ (i · 𝑦) ∉ ℝ+)))
Colors of variables: wff setvar class
This definition is referenced by:  sqrtval  14596  sqrtf  14723  cphsscph  23854
  Copyright terms: Public domain W3C validator