Theorem List for Intuitionistic Logic Explorer - 13401-13500 *Has distinct variable
group(s)
Type | Label | Description |
Statement |
|
Theorem | sincos4thpi 13401 |
The sine and cosine of π / 4. (Contributed by Paul
Chapman,
25-Jan-2008.)
|
⊢ ((sin‘(π / 4)) = (1 /
(√‘2)) ∧ (cos‘(π / 4)) = (1 /
(√‘2))) |
|
Theorem | tan4thpi 13402 |
The tangent of π / 4. (Contributed by Mario
Carneiro,
5-Apr-2015.)
|
⊢ (tan‘(π / 4)) = 1 |
|
Theorem | sincos6thpi 13403 |
The sine and cosine of π / 6. (Contributed by Paul
Chapman,
25-Jan-2008.) (Revised by Wolf Lammen, 24-Sep-2020.)
|
⊢ ((sin‘(π / 6)) = (1 / 2) ∧
(cos‘(π / 6)) = ((√‘3) / 2)) |
|
Theorem | sincos3rdpi 13404 |
The sine and cosine of π / 3. (Contributed by Mario
Carneiro,
21-May-2016.)
|
⊢ ((sin‘(π / 3)) = ((√‘3)
/ 2) ∧ (cos‘(π / 3)) = (1 / 2)) |
|
Theorem | pigt3 13405 |
π is greater than 3. (Contributed by Brendan Leahy,
21-Aug-2020.)
|
⊢ 3 < π |
|
Theorem | pige3 13406 |
π is greater than or equal to 3. (Contributed by
Mario Carneiro,
21-May-2016.)
|
⊢ 3 ≤ π |
|
Theorem | abssinper 13407 |
The absolute value of sine has period π.
(Contributed by NM,
17-Aug-2008.)
|
⊢ ((𝐴 ∈ ℂ ∧ 𝐾 ∈ ℤ) →
(abs‘(sin‘(𝐴 +
(𝐾 · π)))) =
(abs‘(sin‘𝐴))) |
|
Theorem | sinkpi 13408 |
The sine of an integer multiple of π is 0.
(Contributed by NM,
11-Aug-2008.)
|
⊢ (𝐾 ∈ ℤ → (sin‘(𝐾 · π)) =
0) |
|
Theorem | coskpi 13409 |
The absolute value of the cosine of an integer multiple of π is 1.
(Contributed by NM, 19-Aug-2008.)
|
⊢ (𝐾 ∈ ℤ →
(abs‘(cos‘(𝐾
· π))) = 1) |
|
Theorem | cosordlem 13410 |
Cosine is decreasing over the closed interval from 0 to
π.
(Contributed by Mario Carneiro, 10-May-2014.)
|
⊢ (𝜑 → 𝐴 ∈ (0[,]π)) & ⊢ (𝜑 → 𝐵 ∈ (0[,]π)) & ⊢ (𝜑 → 𝐴 < 𝐵) ⇒ ⊢ (𝜑 → (cos‘𝐵) < (cos‘𝐴)) |
|
Theorem | cosq34lt1 13411 |
Cosine is less than one in the third and fourth quadrants. (Contributed
by Jim Kingdon, 19-Mar-2024.)
|
⊢ (𝐴 ∈ (π[,)(2 · π)) →
(cos‘𝐴) <
1) |
|
Theorem | cos02pilt1 13412 |
Cosine is less than one between zero and 2 ·
π. (Contributed by
Jim Kingdon, 19-Mar-2024.)
|
⊢ (𝐴 ∈ (0(,)(2 · π)) →
(cos‘𝐴) <
1) |
|
Theorem | cos0pilt1 13413 |
Cosine is between minus one and one on the open interval between zero and
π. (Contributed by Jim Kingdon, 7-May-2024.)
|
⊢ (𝐴 ∈ (0(,)π) → (cos‘𝐴) ∈
(-1(,)1)) |
|
Theorem | cos11 13414 |
Cosine is one-to-one over the closed interval from 0 to
π.
(Contributed by Paul Chapman, 16-Mar-2008.) (Revised by Jim Kingdon,
6-May-2024.)
|
⊢ ((𝐴 ∈ (0[,]π) ∧ 𝐵 ∈ (0[,]π)) → (𝐴 = 𝐵 ↔ (cos‘𝐴) = (cos‘𝐵))) |
|
Theorem | ioocosf1o 13415 |
The cosine function is a bijection when restricted to its principal
domain. (Contributed by Mario Carneiro, 12-May-2014.) (Revised by Jim
Kingdon, 7-May-2024.)
|
⊢ (cos ↾
(0(,)π)):(0(,)π)–1-1-onto→(-1(,)1) |
|
Theorem | negpitopissre 13416 |
The interval (-π(,]π) is a subset of the reals.
(Contributed by David Moews, 28-Feb-2017.)
|
⊢ (-π(,]π) ⊆
ℝ |
|
10.1.3 The natural logarithm on complex
numbers
|
|
Syntax | clog 13417 |
Extend class notation with the natural logarithm function on complex
numbers.
|
class log |
|
Syntax | ccxp 13418 |
Extend class notation with the complex power function.
|
class ↑𝑐 |
|
Definition | df-relog 13419 |
Define the natural logarithm function. Defining the logarithm on complex
numbers is similar to square root - there are ways to define it but they
tend to make use of excluded middle. Therefore, we merely define
logarithms on positive reals. See
http://en.wikipedia.org/wiki/Natural_logarithm
and
https://en.wikipedia.org/wiki/Complex_logarithm.
(Contributed by Jim
Kingdon, 14-May-2024.)
|
⊢ log = ◡(exp ↾ ℝ) |
|
Definition | df-rpcxp 13420* |
Define the power function on complex numbers. Because df-relog 13419 is
only defined on positive reals, this definition only allows for a base
which is a positive real. (Contributed by Jim Kingdon, 12-Jun-2024.)
|
⊢ ↑𝑐 = (𝑥 ∈ ℝ+,
𝑦 ∈ ℂ ↦
(exp‘(𝑦 ·
(log‘𝑥)))) |
|
Theorem | dfrelog 13421 |
The natural logarithm function on the positive reals in terms of the real
exponential function. (Contributed by Paul Chapman, 21-Apr-2008.)
|
⊢ (log ↾ ℝ+) = ◡(exp ↾ ℝ) |
|
Theorem | relogf1o 13422 |
The natural logarithm function maps the positive reals one-to-one onto the
real numbers. (Contributed by Paul Chapman, 21-Apr-2008.)
|
⊢ (log ↾
ℝ+):ℝ+–1-1-onto→ℝ |
|
Theorem | relogcl 13423 |
Closure of the natural logarithm function on positive reals. (Contributed
by Steve Rodriguez, 25-Nov-2007.)
|
⊢ (𝐴 ∈ ℝ+ →
(log‘𝐴) ∈
ℝ) |
|
Theorem | reeflog 13424 |
Relationship between the natural logarithm function and the exponential
function. (Contributed by Steve Rodriguez, 25-Nov-2007.)
|
⊢ (𝐴 ∈ ℝ+ →
(exp‘(log‘𝐴))
= 𝐴) |
|
Theorem | relogef 13425 |
Relationship between the natural logarithm function and the exponential
function. (Contributed by Steve Rodriguez, 25-Nov-2007.)
|
⊢ (𝐴 ∈ ℝ →
(log‘(exp‘𝐴))
= 𝐴) |
|
Theorem | relogeftb 13426 |
Relationship between the natural logarithm function and the exponential
function. (Contributed by Steve Rodriguez, 25-Nov-2007.)
|
⊢ ((𝐴 ∈ ℝ+ ∧ 𝐵 ∈ ℝ) →
((log‘𝐴) = 𝐵 ↔ (exp‘𝐵) = 𝐴)) |
|
Theorem | log1 13427 |
The natural logarithm of 1. One case of Property 1a of
[Cohen]
p. 301. (Contributed by Steve Rodriguez, 25-Nov-2007.)
|
⊢ (log‘1) = 0 |
|
Theorem | loge 13428 |
The natural logarithm of e. One case of Property 1b of
[Cohen]
p. 301. (Contributed by Steve Rodriguez, 25-Nov-2007.)
|
⊢ (log‘e) = 1 |
|
Theorem | relogoprlem 13429 |
Lemma for relogmul 13430 and relogdiv 13431. Remark of [Cohen] p. 301 ("The
proof of Property 3 is quite similar to the proof given for Property
2"). (Contributed by Steve Rodriguez, 25-Nov-2007.)
|
⊢ (((log‘𝐴) ∈ ℂ ∧ (log‘𝐵) ∈ ℂ) →
(exp‘((log‘𝐴)𝐹(log‘𝐵))) = ((exp‘(log‘𝐴))𝐺(exp‘(log‘𝐵)))) & ⊢
(((log‘𝐴)
∈ ℝ ∧ (log‘𝐵) ∈ ℝ) → ((log‘𝐴)𝐹(log‘𝐵)) ∈ ℝ)
⇒ ⊢ ((𝐴 ∈ ℝ+ ∧ 𝐵 ∈ ℝ+)
→ (log‘(𝐴𝐺𝐵)) = ((log‘𝐴)𝐹(log‘𝐵))) |
|
Theorem | relogmul 13430 |
The natural logarithm of the product of two positive real numbers is the
sum of natural logarithms. Property 2 of [Cohen] p. 301, restricted to
natural logarithms. (Contributed by Steve Rodriguez, 25-Nov-2007.)
|
⊢ ((𝐴 ∈ ℝ+ ∧ 𝐵 ∈ ℝ+)
→ (log‘(𝐴
· 𝐵)) =
((log‘𝐴) +
(log‘𝐵))) |
|
Theorem | relogdiv 13431 |
The natural logarithm of the quotient of two positive real numbers is the
difference of natural logarithms. Exercise 72(a) and Property 3 of
[Cohen] p. 301, restricted to natural
logarithms. (Contributed by Steve
Rodriguez, 25-Nov-2007.)
|
⊢ ((𝐴 ∈ ℝ+ ∧ 𝐵 ∈ ℝ+)
→ (log‘(𝐴 /
𝐵)) = ((log‘𝐴) − (log‘𝐵))) |
|
Theorem | reexplog 13432 |
Exponentiation of a positive real number to an integer power.
(Contributed by Steve Rodriguez, 25-Nov-2007.)
|
⊢ ((𝐴 ∈ ℝ+ ∧ 𝑁 ∈ ℤ) → (𝐴↑𝑁) = (exp‘(𝑁 · (log‘𝐴)))) |
|
Theorem | relogexp 13433 |
The natural logarithm of positive 𝐴 raised to an integer power.
Property 4 of [Cohen] p. 301-302, restricted
to natural logarithms and
integer powers 𝑁. (Contributed by Steve Rodriguez,
25-Nov-2007.)
|
⊢ ((𝐴 ∈ ℝ+ ∧ 𝑁 ∈ ℤ) →
(log‘(𝐴↑𝑁)) = (𝑁 · (log‘𝐴))) |
|
Theorem | relogiso 13434 |
The natural logarithm function on positive reals determines an isomorphism
from the positive reals onto the reals. (Contributed by Steve Rodriguez,
25-Nov-2007.)
|
⊢ (log ↾ ℝ+) Isom <
, < (ℝ+, ℝ) |
|
Theorem | logltb 13435 |
The natural logarithm function on positive reals is strictly monotonic.
(Contributed by Steve Rodriguez, 25-Nov-2007.)
|
⊢ ((𝐴 ∈ ℝ+ ∧ 𝐵 ∈ ℝ+)
→ (𝐴 < 𝐵 ↔ (log‘𝐴) < (log‘𝐵))) |
|
Theorem | logleb 13436 |
Natural logarithm preserves ≤. (Contributed by
Stefan O'Rear,
19-Sep-2014.)
|
⊢ ((𝐴 ∈ ℝ+ ∧ 𝐵 ∈ ℝ+)
→ (𝐴 ≤ 𝐵 ↔ (log‘𝐴) ≤ (log‘𝐵))) |
|
Theorem | logrpap0b 13437 |
The logarithm is apart from 0 if and only if its argument is apart from 1.
(Contributed by Jim Kingdon, 3-Jul-2024.)
|
⊢ (𝐴 ∈ ℝ+ → (𝐴 # 1 ↔ (log‘𝐴) # 0)) |
|
Theorem | logrpap0 13438 |
The logarithm is apart from 0 if its argument is apart from 1.
(Contributed by Jim Kingdon, 5-Jul-2024.)
|
⊢ ((𝐴 ∈ ℝ+ ∧ 𝐴 # 1) → (log‘𝐴) # 0) |
|
Theorem | logrpap0d 13439 |
Deduction form of logrpap0 13438. (Contributed by Jim Kingdon,
3-Jul-2024.)
|
⊢ (𝜑 → 𝐴 ∈ ℝ+) & ⊢ (𝜑 → 𝐴 # 1) ⇒ ⊢ (𝜑 → (log‘𝐴) # 0) |
|
Theorem | rplogcl 13440 |
Closure of the logarithm function in the positive reals. (Contributed by
Mario Carneiro, 21-Sep-2014.)
|
⊢ ((𝐴 ∈ ℝ ∧ 1 < 𝐴) → (log‘𝐴) ∈
ℝ+) |
|
Theorem | logge0 13441 |
The logarithm of a number greater than 1 is nonnegative. (Contributed by
Mario Carneiro, 29-May-2016.)
|
⊢ ((𝐴 ∈ ℝ ∧ 1 ≤ 𝐴) → 0 ≤
(log‘𝐴)) |
|
Theorem | logdivlti 13442 |
The log𝑥 /
𝑥 function is
strictly decreasing on the reals greater
than e. (Contributed by Mario Carneiro,
14-Mar-2014.)
|
⊢ (((𝐴 ∈ ℝ ∧ 𝐵 ∈ ℝ ∧ e ≤ 𝐴) ∧ 𝐴 < 𝐵) → ((log‘𝐵) / 𝐵) < ((log‘𝐴) / 𝐴)) |
|
Theorem | relogcld 13443 |
Closure of the natural logarithm function. (Contributed by Mario
Carneiro, 29-May-2016.)
|
⊢ (𝜑 → 𝐴 ∈
ℝ+) ⇒ ⊢ (𝜑 → (log‘𝐴) ∈ ℝ) |
|
Theorem | reeflogd 13444 |
Relationship between the natural logarithm function and the exponential
function. (Contributed by Mario Carneiro, 29-May-2016.)
|
⊢ (𝜑 → 𝐴 ∈
ℝ+) ⇒ ⊢ (𝜑 → (exp‘(log‘𝐴)) = 𝐴) |
|
Theorem | relogmuld 13445 |
The natural logarithm of the product of two positive real numbers is the
sum of natural logarithms. Property 2 of [Cohen] p. 301, restricted to
natural logarithms. (Contributed by Mario Carneiro, 29-May-2016.)
|
⊢ (𝜑 → 𝐴 ∈ ℝ+) & ⊢ (𝜑 → 𝐵 ∈
ℝ+) ⇒ ⊢ (𝜑 → (log‘(𝐴 · 𝐵)) = ((log‘𝐴) + (log‘𝐵))) |
|
Theorem | relogdivd 13446 |
The natural logarithm of the quotient of two positive real numbers is
the difference of natural logarithms. Exercise 72(a) and Property 3 of
[Cohen] p. 301, restricted to natural
logarithms. (Contributed by Mario
Carneiro, 29-May-2016.)
|
⊢ (𝜑 → 𝐴 ∈ ℝ+) & ⊢ (𝜑 → 𝐵 ∈
ℝ+) ⇒ ⊢ (𝜑 → (log‘(𝐴 / 𝐵)) = ((log‘𝐴) − (log‘𝐵))) |
|
Theorem | logled 13447 |
Natural logarithm preserves ≤. (Contributed by
Mario Carneiro,
29-May-2016.)
|
⊢ (𝜑 → 𝐴 ∈ ℝ+) & ⊢ (𝜑 → 𝐵 ∈
ℝ+) ⇒ ⊢ (𝜑 → (𝐴 ≤ 𝐵 ↔ (log‘𝐴) ≤ (log‘𝐵))) |
|
Theorem | relogefd 13448 |
Relationship between the natural logarithm function and the exponential
function. (Contributed by Mario Carneiro, 29-May-2016.)
|
⊢ (𝜑 → 𝐴 ∈ ℝ)
⇒ ⊢ (𝜑 → (log‘(exp‘𝐴)) = 𝐴) |
|
Theorem | rplogcld 13449 |
Closure of the logarithm function in the positive reals. (Contributed
by Mario Carneiro, 29-May-2016.)
|
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 1 < 𝐴) ⇒ ⊢ (𝜑 → (log‘𝐴) ∈
ℝ+) |
|
Theorem | logge0d 13450 |
The logarithm of a number greater than 1 is nonnegative. (Contributed
by Mario Carneiro, 29-May-2016.)
|
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 1 ≤ 𝐴) ⇒ ⊢ (𝜑 → 0 ≤ (log‘𝐴)) |
|
Theorem | logge0b 13451 |
The logarithm of a number is nonnegative iff the number is greater than or
equal to 1. (Contributed by AV, 30-May-2020.)
|
⊢ (𝐴 ∈ ℝ+ → (0 ≤
(log‘𝐴) ↔ 1
≤ 𝐴)) |
|
Theorem | loggt0b 13452 |
The logarithm of a number is positive iff the number is greater than 1.
(Contributed by AV, 30-May-2020.)
|
⊢ (𝐴 ∈ ℝ+ → (0 <
(log‘𝐴) ↔ 1
< 𝐴)) |
|
Theorem | logle1b 13453 |
The logarithm of a number is less than or equal to 1 iff the number is
less than or equal to Euler's constant. (Contributed by AV,
30-May-2020.)
|
⊢ (𝐴 ∈ ℝ+ →
((log‘𝐴) ≤ 1
↔ 𝐴 ≤
e)) |
|
Theorem | loglt1b 13454 |
The logarithm of a number is less than 1 iff the number is less than
Euler's constant. (Contributed by AV, 30-May-2020.)
|
⊢ (𝐴 ∈ ℝ+ →
((log‘𝐴) < 1
↔ 𝐴 <
e)) |
|
Theorem | rpcxpef 13455 |
Value of the complex power function. (Contributed by Mario Carneiro,
2-Aug-2014.) (Revised by Jim Kingdon, 12-Jun-2024.)
|
⊢ ((𝐴 ∈ ℝ+ ∧ 𝐵 ∈ ℂ) → (𝐴↑𝑐𝐵) = (exp‘(𝐵 · (log‘𝐴)))) |
|
Theorem | cxpexprp 13456 |
Relate the complex power function to the integer power function.
(Contributed by Mario Carneiro, 2-Aug-2014.) (Revised by Jim Kingdon,
12-Jun-2024.)
|
⊢ ((𝐴 ∈ ℝ+ ∧ 𝐵 ∈ ℤ) → (𝐴↑𝑐𝐵) = (𝐴↑𝐵)) |
|
Theorem | cxpexpnn 13457 |
Relate the complex power function to the integer power function.
(Contributed by Mario Carneiro, 2-Aug-2014.) (Revised by Jim Kingdon,
12-Jun-2024.)
|
⊢ ((𝐴 ∈ ℕ ∧ 𝐵 ∈ ℤ) → (𝐴↑𝑐𝐵) = (𝐴↑𝐵)) |
|
Theorem | logcxp 13458 |
Logarithm of a complex power. (Contributed by Mario Carneiro,
2-Aug-2014.)
|
⊢ ((𝐴 ∈ ℝ+ ∧ 𝐵 ∈ ℝ) →
(log‘(𝐴↑𝑐𝐵)) = (𝐵 · (log‘𝐴))) |
|
Theorem | rpcxp0 13459 |
Value of the complex power function when the second argument is zero.
(Contributed by Mario Carneiro, 2-Aug-2014.) (Revised by Jim Kingdon,
12-Jun-2024.)
|
⊢ (𝐴 ∈ ℝ+ → (𝐴↑𝑐0) =
1) |
|
Theorem | rpcxp1 13460 |
Value of the complex power function at one. (Contributed by Mario
Carneiro, 2-Aug-2014.)
|
⊢ (𝐴 ∈ ℝ+ → (𝐴↑𝑐1) =
𝐴) |
|
Theorem | 1cxp 13461 |
Value of the complex power function at one. (Contributed by Mario
Carneiro, 2-Aug-2014.)
|
⊢ (𝐴 ∈ ℂ →
(1↑𝑐𝐴) = 1) |
|
Theorem | ecxp 13462 |
Write the exponential function as an exponent to the power e.
(Contributed by Mario Carneiro, 2-Aug-2014.)
|
⊢ (𝐴 ∈ ℂ →
(e↑𝑐𝐴) = (exp‘𝐴)) |
|
Theorem | rpcncxpcl 13463 |
Closure of the complex power function. (Contributed by Jim Kingdon,
12-Jun-2024.)
|
⊢ ((𝐴 ∈ ℝ+ ∧ 𝐵 ∈ ℂ) → (𝐴↑𝑐𝐵) ∈
ℂ) |
|
Theorem | rpcxpcl 13464 |
Positive real closure of the complex power function. (Contributed by
Mario Carneiro, 2-Aug-2014.)
|
⊢ ((𝐴 ∈ ℝ+ ∧ 𝐵 ∈ ℝ) → (𝐴↑𝑐𝐵) ∈
ℝ+) |
|
Theorem | cxpap0 13465 |
Complex exponentiation is apart from zero. (Contributed by Mario
Carneiro, 2-Aug-2014.) (Revised by Jim Kingdon, 12-Jun-2024.)
|
⊢ ((𝐴 ∈ ℝ+ ∧ 𝐵 ∈ ℂ) → (𝐴↑𝑐𝐵) # 0) |
|
Theorem | rpcxpadd 13466 |
Sum of exponents law for complex exponentiation. (Contributed by Mario
Carneiro, 2-Aug-2014.) (Revised by Jim Kingdon, 13-Jun-2024.)
|
⊢ ((𝐴 ∈ ℝ+ ∧ 𝐵 ∈ ℂ ∧ 𝐶 ∈ ℂ) → (𝐴↑𝑐(𝐵 + 𝐶)) = ((𝐴↑𝑐𝐵) · (𝐴↑𝑐𝐶))) |
|
Theorem | rpcxpp1 13467 |
Value of a nonzero complex number raised to a complex power plus one.
(Contributed by Mario Carneiro, 2-Aug-2014.)
|
⊢ ((𝐴 ∈ ℝ+ ∧ 𝐵 ∈ ℂ) → (𝐴↑𝑐(𝐵 + 1)) = ((𝐴↑𝑐𝐵) · 𝐴)) |
|
Theorem | rpcxpneg 13468 |
Value of a complex number raised to a negative power. (Contributed by
Mario Carneiro, 2-Aug-2014.)
|
⊢ ((𝐴 ∈ ℝ+ ∧ 𝐵 ∈ ℂ) → (𝐴↑𝑐-𝐵) = (1 / (𝐴↑𝑐𝐵))) |
|
Theorem | rpcxpsub 13469 |
Exponent subtraction law for complex exponentiation. (Contributed by
Mario Carneiro, 22-Sep-2014.)
|
⊢ ((𝐴 ∈ ℝ+ ∧ 𝐵 ∈ ℂ ∧ 𝐶 ∈ ℂ) → (𝐴↑𝑐(𝐵 − 𝐶)) = ((𝐴↑𝑐𝐵) / (𝐴↑𝑐𝐶))) |
|
Theorem | rpmulcxp 13470 |
Complex exponentiation of a product. Proposition 10-4.2(c) of [Gleason]
p. 135. (Contributed by Mario Carneiro, 2-Aug-2014.)
|
⊢ ((𝐴 ∈ ℝ+ ∧ 𝐵 ∈ ℝ+
∧ 𝐶 ∈ ℂ)
→ ((𝐴 · 𝐵)↑𝑐𝐶) = ((𝐴↑𝑐𝐶) · (𝐵↑𝑐𝐶))) |
|
Theorem | cxprec 13471 |
Complex exponentiation of a reciprocal. (Contributed by Mario Carneiro,
2-Aug-2014.)
|
⊢ ((𝐴 ∈ ℝ+ ∧ 𝐵 ∈ ℂ) → ((1 /
𝐴)↑𝑐𝐵) = (1 / (𝐴↑𝑐𝐵))) |
|
Theorem | rpdivcxp 13472 |
Complex exponentiation of a quotient. (Contributed by Mario Carneiro,
8-Sep-2014.)
|
⊢ ((𝐴 ∈ ℝ+ ∧ 𝐵 ∈ ℝ+
∧ 𝐶 ∈ ℂ)
→ ((𝐴 / 𝐵)↑𝑐𝐶) = ((𝐴↑𝑐𝐶) / (𝐵↑𝑐𝐶))) |
|
Theorem | cxpmul 13473 |
Product of exponents law for complex exponentiation. Proposition
10-4.2(b) of [Gleason] p. 135.
(Contributed by Mario Carneiro,
2-Aug-2014.)
|
⊢ ((𝐴 ∈ ℝ+ ∧ 𝐵 ∈ ℝ ∧ 𝐶 ∈ ℂ) → (𝐴↑𝑐(𝐵 · 𝐶)) = ((𝐴↑𝑐𝐵)↑𝑐𝐶)) |
|
Theorem | rpcxproot 13474 |
The complex power function allows us to write n-th roots via the idiom
𝐴↑𝑐(1 / 𝑁). (Contributed by Mario
Carneiro, 6-May-2015.)
|
⊢ ((𝐴 ∈ ℝ+ ∧ 𝑁 ∈ ℕ) → ((𝐴↑𝑐(1 /
𝑁))↑𝑁) = 𝐴) |
|
Theorem | abscxp 13475 |
Absolute value of a power, when the base is real. (Contributed by Mario
Carneiro, 15-Sep-2014.)
|
⊢ ((𝐴 ∈ ℝ+ ∧ 𝐵 ∈ ℂ) →
(abs‘(𝐴↑𝑐𝐵)) = (𝐴↑𝑐(ℜ‘𝐵))) |
|
Theorem | cxplt 13476 |
Ordering property for complex exponentiation. (Contributed by Mario
Carneiro, 2-Aug-2014.)
|
⊢ (((𝐴 ∈ ℝ ∧ 1 < 𝐴) ∧ (𝐵 ∈ ℝ ∧ 𝐶 ∈ ℝ)) → (𝐵 < 𝐶 ↔ (𝐴↑𝑐𝐵) < (𝐴↑𝑐𝐶))) |
|
Theorem | cxple 13477 |
Ordering property for complex exponentiation. (Contributed by Mario
Carneiro, 2-Aug-2014.)
|
⊢ (((𝐴 ∈ ℝ ∧ 1 < 𝐴) ∧ (𝐵 ∈ ℝ ∧ 𝐶 ∈ ℝ)) → (𝐵 ≤ 𝐶 ↔ (𝐴↑𝑐𝐵) ≤ (𝐴↑𝑐𝐶))) |
|
Theorem | rpcxple2 13478 |
Ordering property for complex exponentiation. (Contributed by Mario
Carneiro, 8-Sep-2014.)
|
⊢ ((𝐴 ∈ ℝ+ ∧ 𝐵 ∈ ℝ+
∧ 𝐶 ∈
ℝ+) → (𝐴 ≤ 𝐵 ↔ (𝐴↑𝑐𝐶) ≤ (𝐵↑𝑐𝐶))) |
|
Theorem | rpcxplt2 13479 |
Ordering property for complex exponentiation. (Contributed by Mario
Carneiro, 15-Sep-2014.)
|
⊢ ((𝐴 ∈ ℝ+ ∧ 𝐵 ∈ ℝ+
∧ 𝐶 ∈
ℝ+) → (𝐴 < 𝐵 ↔ (𝐴↑𝑐𝐶) < (𝐵↑𝑐𝐶))) |
|
Theorem | cxplt3 13480 |
Ordering property for complex exponentiation. (Contributed by Mario
Carneiro, 2-May-2016.)
|
⊢ (((𝐴 ∈ ℝ+ ∧ 𝐴 < 1) ∧ (𝐵 ∈ ℝ ∧ 𝐶 ∈ ℝ)) → (𝐵 < 𝐶 ↔ (𝐴↑𝑐𝐶) < (𝐴↑𝑐𝐵))) |
|
Theorem | cxple3 13481 |
Ordering property for complex exponentiation. (Contributed by Mario
Carneiro, 2-May-2016.)
|
⊢ (((𝐴 ∈ ℝ+ ∧ 𝐴 < 1) ∧ (𝐵 ∈ ℝ ∧ 𝐶 ∈ ℝ)) → (𝐵 ≤ 𝐶 ↔ (𝐴↑𝑐𝐶) ≤ (𝐴↑𝑐𝐵))) |
|
Theorem | rpcxpsqrt 13482 |
The exponential function with exponent 1 / 2 exactly
matches the
square root function, and thus serves as a suitable generalization to
other 𝑛-th roots and irrational roots.
(Contributed by Mario
Carneiro, 2-Aug-2014.) (Revised by Jim Kingdon, 16-Jun-2024.)
|
⊢ (𝐴 ∈ ℝ+ → (𝐴↑𝑐(1 /
2)) = (√‘𝐴)) |
|
Theorem | logsqrt 13483 |
Logarithm of a square root. (Contributed by Mario Carneiro,
5-May-2016.)
|
⊢ (𝐴 ∈ ℝ+ →
(log‘(√‘𝐴)) = ((log‘𝐴) / 2)) |
|
Theorem | rpcxp0d 13484 |
Value of the complex power function when the second argument is zero.
(Contributed by Mario Carneiro, 30-May-2016.)
|
⊢ (𝜑 → 𝐴 ∈
ℝ+) ⇒ ⊢ (𝜑 → (𝐴↑𝑐0) =
1) |
|
Theorem | rpcxp1d 13485 |
Value of the complex power function at one. (Contributed by Mario
Carneiro, 30-May-2016.)
|
⊢ (𝜑 → 𝐴 ∈
ℝ+) ⇒ ⊢ (𝜑 → (𝐴↑𝑐1) = 𝐴) |
|
Theorem | 1cxpd 13486 |
Value of the complex power function at one. (Contributed by Mario
Carneiro, 30-May-2016.)
|
⊢ (𝜑 → 𝐴 ∈ ℂ)
⇒ ⊢ (𝜑 → (1↑𝑐𝐴) = 1) |
|
Theorem | rpcncxpcld 13487 |
Closure of the complex power function. (Contributed by Mario Carneiro,
30-May-2016.)
|
⊢ (𝜑 → 𝐴 ∈ ℝ+) & ⊢ (𝜑 → 𝐵 ∈ ℂ)
⇒ ⊢ (𝜑 → (𝐴↑𝑐𝐵) ∈ ℂ) |
|
Theorem | cxpltd 13488 |
Ordering property for complex exponentiation. (Contributed by Mario
Carneiro, 30-May-2016.)
|
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 1 < 𝐴)
& ⊢ (𝜑 → 𝐵 ∈ ℝ) & ⊢ (𝜑 → 𝐶 ∈ ℝ)
⇒ ⊢ (𝜑 → (𝐵 < 𝐶 ↔ (𝐴↑𝑐𝐵) < (𝐴↑𝑐𝐶))) |
|
Theorem | cxpled 13489 |
Ordering property for complex exponentiation. (Contributed by Mario
Carneiro, 30-May-2016.)
|
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 1 < 𝐴)
& ⊢ (𝜑 → 𝐵 ∈ ℝ) & ⊢ (𝜑 → 𝐶 ∈ ℝ)
⇒ ⊢ (𝜑 → (𝐵 ≤ 𝐶 ↔ (𝐴↑𝑐𝐵) ≤ (𝐴↑𝑐𝐶))) |
|
Theorem | rpcxpsqrtth 13490 |
Square root theorem over the complex numbers for the complex power
function. Compare with resqrtth 10973. (Contributed by AV, 23-Dec-2022.)
|
⊢ (𝐴 ∈ ℝ+ →
((√‘𝐴)↑𝑐2) = 𝐴) |
|
Theorem | cxprecd 13491 |
Complex exponentiation of a reciprocal. (Contributed by Mario
Carneiro, 30-May-2016.)
|
⊢ (𝜑 → 𝐴 ∈ ℝ+) & ⊢ (𝜑 → 𝐵 ∈ ℂ)
⇒ ⊢ (𝜑 → ((1 / 𝐴)↑𝑐𝐵) = (1 / (𝐴↑𝑐𝐵))) |
|
Theorem | rpcxpcld 13492 |
Positive real closure of the complex power function. (Contributed by
Mario Carneiro, 30-May-2016.)
|
⊢ (𝜑 → 𝐴 ∈ ℝ+) & ⊢ (𝜑 → 𝐵 ∈ ℝ)
⇒ ⊢ (𝜑 → (𝐴↑𝑐𝐵) ∈
ℝ+) |
|
Theorem | logcxpd 13493 |
Logarithm of a complex power. (Contributed by Mario Carneiro,
30-May-2016.)
|
⊢ (𝜑 → 𝐴 ∈ ℝ+) & ⊢ (𝜑 → 𝐵 ∈ ℝ)
⇒ ⊢ (𝜑 → (log‘(𝐴↑𝑐𝐵)) = (𝐵 · (log‘𝐴))) |
|
Theorem | cxplt3d 13494 |
Ordering property for complex exponentiation. (Contributed by Mario
Carneiro, 30-May-2016.)
|
⊢ (𝜑 → 𝐴 ∈ ℝ+) & ⊢ (𝜑 → 𝐵 ∈ ℝ) & ⊢ (𝜑 → 𝐴 < 1) & ⊢ (𝜑 → 𝐶 ∈ ℝ)
⇒ ⊢ (𝜑 → (𝐵 < 𝐶 ↔ (𝐴↑𝑐𝐶) < (𝐴↑𝑐𝐵))) |
|
Theorem | cxple3d 13495 |
Ordering property for complex exponentiation. (Contributed by Mario
Carneiro, 30-May-2016.)
|
⊢ (𝜑 → 𝐴 ∈ ℝ+) & ⊢ (𝜑 → 𝐵 ∈ ℝ) & ⊢ (𝜑 → 𝐴 < 1) & ⊢ (𝜑 → 𝐶 ∈ ℝ)
⇒ ⊢ (𝜑 → (𝐵 ≤ 𝐶 ↔ (𝐴↑𝑐𝐶) ≤ (𝐴↑𝑐𝐵))) |
|
Theorem | cxpmuld 13496 |
Product of exponents law for complex exponentiation. Proposition
10-4.2(b) of [Gleason] p. 135.
(Contributed by Mario Carneiro,
30-May-2016.)
|
⊢ (𝜑 → 𝐴 ∈ ℝ+) & ⊢ (𝜑 → 𝐵 ∈ ℝ) & ⊢ (𝜑 → 𝐶 ∈ ℂ)
⇒ ⊢ (𝜑 → (𝐴↑𝑐(𝐵 · 𝐶)) = ((𝐴↑𝑐𝐵)↑𝑐𝐶)) |
|
Theorem | cxpcom 13497 |
Commutative law for real exponentiation. (Contributed by AV,
29-Dec-2022.)
|
⊢ ((𝐴 ∈ ℝ+ ∧ 𝐵 ∈ ℝ ∧ 𝐶 ∈ ℝ) → ((𝐴↑𝑐𝐵)↑𝑐𝐶) = ((𝐴↑𝑐𝐶)↑𝑐𝐵)) |
|
Theorem | apcxp2 13498 |
Apartness and real exponentiation. (Contributed by Jim Kingdon,
10-Jul-2024.)
|
⊢ (((𝐴 ∈ ℝ+ ∧ 𝐴 # 1) ∧ (𝐵 ∈ ℝ ∧ 𝐶 ∈ ℝ)) → (𝐵 # 𝐶 ↔ (𝐴↑𝑐𝐵) # (𝐴↑𝑐𝐶))) |
|
Theorem | rpabscxpbnd 13499 |
Bound on the absolute value of a complex power. (Contributed by Mario
Carneiro, 15-Sep-2014.) (Revised by Jim Kingdon, 19-Jun-2024.)
|
⊢ (𝜑 → 𝐴 ∈ ℝ+) & ⊢ (𝜑 → 𝐵 ∈ ℂ) & ⊢ (𝜑 → 0 <
(ℜ‘𝐵)) & ⊢ (𝜑 → 𝑀 ∈ ℝ) & ⊢ (𝜑 → (abs‘𝐴) ≤ 𝑀) ⇒ ⊢ (𝜑 → (abs‘(𝐴↑𝑐𝐵)) ≤ ((𝑀↑𝑐(ℜ‘𝐵)) ·
(exp‘((abs‘𝐵)
· π)))) |
|
Theorem | ltexp2 13500 |
Ordering law for exponentiation. (Contributed by NM, 2-Aug-2006.)
(Revised by Mario Carneiro, 5-Jun-2014.)
|
⊢ (((𝐴 ∈ ℝ ∧ 𝑀 ∈ ℤ ∧ 𝑁 ∈ ℤ) ∧ 1 < 𝐴) → (𝑀 < 𝑁 ↔ (𝐴↑𝑀) < (𝐴↑𝑁))) |