mathlib documentation

algebra.​field_power

algebra.​field_power

@[simp]
theorem ring_hom.​map_fpow {K : Type u_1} {L : Type u_2} [division_ring K] [division_ring L] (f : K →+* L) (a : K) (n : ) :
f (a ^ n) = f a ^ n

theorem fpow_nonneg_of_nonneg {K : Type u} [discrete_linear_ordered_field K] {a : K} (ha : 0 a) (z : ) :
0 a ^ z

theorem fpow_pos_of_pos {K : Type u} [discrete_linear_ordered_field K] {a : K} (ha : 0 < a) (z : ) :
0 < a ^ z

theorem fpow_le_of_le {K : Type u} [discrete_linear_ordered_field K] {x : K} (hx : 1 x) {a b : } :
a bx ^ a x ^ b

theorem pow_le_max_of_min_le {K : Type u} [discrete_linear_ordered_field K] {x : K} (hx : 1 x) {a b c : } :
min a b cx ^ -c max (x ^ -a) (x ^ -b)

theorem fpow_le_one_of_nonpos {K : Type u} [discrete_linear_ordered_field K] {p : K} (hp : 1 p) {z : } :
z 0p ^ z 1

theorem one_le_fpow_of_nonneg {K : Type u} [discrete_linear_ordered_field K] {p : K} (hp : 1 p) {z : } :
0 z1 p ^ z

theorem one_lt_pow {K : Type u_1} [linear_ordered_semiring K] {p : K} (hp : 1 < p) {n : } :
1 n1 < p ^ n

theorem one_lt_fpow {K : Type u_1} [discrete_linear_ordered_field K] {p : K} (hp : 1 < p) (z : ) :
0 < z1 < p ^ z

theorem nat.​fpow_pos_of_pos {K : Type u_1} [discrete_linear_ordered_field K] {p : } (h : 0 < p) (n : ) :
0 < p ^ n

theorem nat.​fpow_ne_zero_of_pos {K : Type u_1} [discrete_linear_ordered_field K] {p : } (h : 0 < p) (n : ) :
p ^ n 0

theorem fpow_strict_mono {K : Type u_1} [discrete_linear_ordered_field K] {x : K} :
1 < xstrict_mono (λ (n : ), x ^ n)

@[simp]
theorem fpow_lt_iff_lt {K : Type u_1} [discrete_linear_ordered_field K] {x : K} (hx : 1 < x) {m n : } :
x ^ m < x ^ n m < n

@[simp]
theorem fpow_le_iff_le {K : Type u_1} [discrete_linear_ordered_field K] {x : K} (hx : 1 < x) {m n : } :
x ^ m x ^ n m n

@[simp]
theorem pos_div_pow_pos {K : Type u_1} [discrete_linear_ordered_field K] {a b : K} (ha : 0 < a) (hb : 0 < b) (k : ) :
0 < a / b ^ k

@[simp]
theorem div_pow_le {K : Type u_1} [discrete_linear_ordered_field K] {a b : K} (ha : 0 < a) (hb : 1 b) (k : ) :
a / b ^ k a

theorem fpow_injective {K : Type u_1} [discrete_linear_ordered_field K] {x : K} :
0 < xx 1function.injective (has_pow.pow x)

@[simp]
theorem fpow_inj {K : Type u_1} [discrete_linear_ordered_field K] {x : K} (h₀ : 0 < x) (h₁ : x 1) {m n : } :
x ^ m = x ^ n m = n

@[simp]
theorem rat.​cast_fpow {K : Type u_1} [field K] [char_zero K] (q : ) (n : ) :
(q ^ n) = q ^ n