| Intuitionistic Logic Explorer |
< Previous
Next >
Nearby theorems |
||
| Mirrors > Home > ILE Home > Th. List > df-rsqrt | GIF version | ||
| Description: Define a function whose
value is the square root of a nonnegative real
number.
Defining the square root for complex numbers has one difficult part: choosing between the two roots. The usual way to define a principal square root for all complex numbers relies on excluded middle or something similar. But in the case of a nonnegative real number, we don't have the complications presented for general complex numbers, and we can choose the nonnegative root. (Contributed by Jim Kingdon, 23-Aug-2020.) |
| Ref | Expression |
|---|---|
| df-rsqrt | ⊢ √ = (𝑥 ∈ ℝ ↦ (℩𝑦 ∈ ℝ ((𝑦↑2) = 𝑥 ∧ 0 ≤ 𝑦))) |
| Step | Hyp | Ref | Expression |
|---|---|---|---|
| 1 | csqrt 11178 | . 2 class √ | |
| 2 | vx | . . 3 setvar 𝑥 | |
| 3 | cr 7895 | . . 3 class ℝ | |
| 4 | vy | . . . . . . . 8 setvar 𝑦 | |
| 5 | 4 | cv 1363 | . . . . . . 7 class 𝑦 |
| 6 | c2 9058 | . . . . . . 7 class 2 | |
| 7 | cexp 10647 | . . . . . . 7 class ↑ | |
| 8 | 5, 6, 7 | co 5925 | . . . . . 6 class (𝑦↑2) |
| 9 | 2 | cv 1363 | . . . . . 6 class 𝑥 |
| 10 | 8, 9 | wceq 1364 | . . . . 5 wff (𝑦↑2) = 𝑥 |
| 11 | cc0 7896 | . . . . . 6 class 0 | |
| 12 | cle 8079 | . . . . . 6 class ≤ | |
| 13 | 11, 5, 12 | wbr 4034 | . . . . 5 wff 0 ≤ 𝑦 |
| 14 | 10, 13 | wa 104 | . . . 4 wff ((𝑦↑2) = 𝑥 ∧ 0 ≤ 𝑦) |
| 15 | 14, 4, 3 | crio 5879 | . . 3 class (℩𝑦 ∈ ℝ ((𝑦↑2) = 𝑥 ∧ 0 ≤ 𝑦)) |
| 16 | 2, 3, 15 | cmpt 4095 | . 2 class (𝑥 ∈ ℝ ↦ (℩𝑦 ∈ ℝ ((𝑦↑2) = 𝑥 ∧ 0 ≤ 𝑦))) |
| 17 | 1, 16 | wceq 1364 | 1 wff √ = (𝑥 ∈ ℝ ↦ (℩𝑦 ∈ ℝ ((𝑦↑2) = 𝑥 ∧ 0 ≤ 𝑦))) |
| Colors of variables: wff set class |
| This definition is referenced by: sqrtrval 11182 absval 11183 |
| Copyright terms: Public domain | W3C validator |