mathlib documentation

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 : } (h : a b) :
x ^ 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 : } (h : min a b c) :
x ^ -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 : } (hz : z 0) :
p ^ z 1

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

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

theorem one_lt_fpow {K : Type u_1} [discrete_linear_ordered_field K] {p : K} (hp : 1 < p) (z : ) (a : 0 < z) :
1 < 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} (hx : 1 < x) :
strict_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} (h₀ : 0 < x) (h₁ : x 1) :

@[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