Mathlib v3 is deprecated. Go to Mathlib v4

Commit 2020-09-25 00:12 f9a667d3

View on Github →

refactor(algebra/group_power, data/nat/basic): remove redundant lemmas (#4243) This removes lemmas about pow on nat which are redundant with more general versions in the root namespace. One notable removal is nat.pow_succ; use pow_succ' instead. In order that the general versions are available already in data.nat.basic, many lemmas from algebra.group_power.lemmas have been moved to algebra.group_power.basic (basically as many as possible without adding imports).

Estimated changes

added theorem abs_neg_one_pow
added theorem bit0_nsmul
added theorem bit1_nsmul
added theorem commute.gpow_gpow
added theorem commute.gpow_gpow_self
added theorem commute.gpow_left
added theorem commute.gpow_right
added theorem commute.gpow_self
added theorem commute.mul_gpow
added theorem commute.mul_pow
added theorem commute.self_gpow
added theorem dvd_pow
added theorem gpow_coe_nat
added theorem gpow_neg
added theorem gpow_neg_one
added theorem gpow_neg_succ_of_nat
added theorem gpow_of_nat
added theorem gpow_one
added theorem gpow_zero
added theorem gsmul_add
added theorem gsmul_coe_nat
added theorem gsmul_neg
added theorem gsmul_neg_succ_of_nat
added theorem gsmul_of_nat
added theorem gsmul_sub
added theorem gsmul_zero
added theorem inv_gpow
added theorem inv_pow
added theorem is_monoid_hom.map_pow
added theorem ite_pow
added theorem lt_of_pow_lt_pow
added theorem monoid_hom.map_pow
added theorem mul_gpow
added theorem mul_gpow_neg_one
added theorem mul_nsmul'
added theorem mul_nsmul
added theorem mul_pow
added theorem neg_gsmul
added theorem neg_nsmul
added theorem neg_one_gsmul
added theorem neg_one_pow_eq_or
added theorem neg_pow
added theorem neg_square
added theorem nsmul_add
added theorem nsmul_add_comm
added theorem nsmul_add_sub_nsmul
added theorem nsmul_le_nsmul
added theorem nsmul_neg_comm
added theorem nsmul_nonneg
added theorem nsmul_sub
added theorem nsmul_zero
added theorem of_add_gsmul
added theorem of_add_nsmul
added theorem one_gpow
added theorem one_gsmul
added theorem one_le_pow_of_one_le
added theorem one_nsmul
added theorem one_pow
added theorem pow_abs
added theorem pow_bit0
added theorem pow_bit1
added theorem pow_boole
added theorem pow_dvd_pow
added theorem pow_dvd_pow_of_dvd
added theorem pow_eq_zero
added theorem pow_inv_comm
added theorem pow_ite
added theorem pow_le_pow
added theorem pow_le_pow_of_le_left
added theorem pow_left_inj
added theorem pow_lt_pow
added theorem pow_lt_pow_of_lt_left
added theorem pow_mul'
added theorem pow_mul
added theorem pow_mul_comm
added theorem pow_mul_pow_sub
added theorem pow_ne_zero
added theorem pow_nonneg
added theorem pow_one
added theorem pow_pos
added theorem pow_sub
added theorem pow_sub_mul_pow
added theorem pow_two_nonneg
added theorem pow_two_pos_of_ne_zero
added theorem pow_two_sub_pow_two
added theorem ring_hom.map_pow
added theorem semiconj_by.gpow_right
added theorem sq_sub_sq
added theorem sub_nsmul_nsmul_add
added theorem zero_gsmul
added theorem zero_pow
deleted theorem abs_neg_one_pow
deleted theorem add_monoid_hom.map_nsmul
deleted theorem bit0_nsmul
deleted theorem bit1_nsmul
deleted theorem commute.gpow_gpow
deleted theorem commute.gpow_gpow_self
deleted theorem commute.gpow_left
deleted theorem commute.gpow_right
deleted theorem commute.gpow_self
deleted theorem commute.mul_gpow
deleted theorem commute.mul_pow
deleted theorem commute.self_gpow
deleted theorem dvd_pow
deleted theorem gpow_coe_nat
deleted theorem gpow_neg
deleted theorem gpow_neg_one
deleted theorem gpow_neg_succ_of_nat
deleted theorem gpow_of_nat
deleted theorem gpow_one
deleted theorem gpow_zero
deleted theorem gsmul_add
deleted theorem gsmul_coe_nat
deleted theorem gsmul_neg
deleted theorem gsmul_neg_succ_of_nat
deleted theorem gsmul_of_nat
deleted theorem gsmul_sub
deleted theorem gsmul_zero
deleted theorem inv_gpow
deleted theorem inv_pow
deleted theorem is_monoid_hom.map_pow
deleted theorem ite_pow
deleted theorem lt_of_pow_lt_pow
deleted theorem monoid_hom.map_pow
deleted theorem mul_gpow
deleted theorem mul_gpow_neg_one
deleted theorem mul_nsmul'
deleted theorem mul_nsmul
deleted theorem mul_pow
deleted theorem neg_gsmul
deleted theorem neg_nsmul
deleted theorem neg_one_gsmul
deleted theorem neg_one_pow_eq_or
deleted theorem neg_pow
deleted theorem neg_square
deleted theorem nsmul_add
deleted theorem nsmul_add_comm
deleted theorem nsmul_add_sub_nsmul
deleted theorem nsmul_le_nsmul
deleted theorem nsmul_neg_comm
deleted theorem nsmul_nonneg
deleted theorem nsmul_sub
deleted theorem nsmul_zero
deleted theorem of_add_gsmul
deleted theorem of_add_nsmul
deleted theorem one_gpow
deleted theorem one_gsmul
deleted theorem one_le_pow_of_one_le
deleted theorem one_nsmul
deleted theorem one_pow
deleted theorem pow_abs
deleted theorem pow_bit0
deleted theorem pow_bit1
deleted theorem pow_boole
deleted theorem pow_dvd_pow
deleted theorem pow_dvd_pow_of_dvd
deleted theorem pow_eq_zero
deleted theorem pow_inv_comm
deleted theorem pow_ite
deleted theorem pow_le_pow
deleted theorem pow_le_pow_of_le_left
deleted theorem pow_left_inj
deleted theorem pow_lt_pow
deleted theorem pow_lt_pow_of_lt_left
deleted theorem pow_mul'
deleted theorem pow_mul
deleted theorem pow_mul_comm
deleted theorem pow_mul_pow_sub
deleted theorem pow_ne_zero
deleted theorem pow_nonneg
deleted theorem pow_one
deleted theorem pow_pos
deleted theorem pow_sub
deleted theorem pow_sub_mul_pow
deleted theorem pow_two_nonneg
deleted theorem pow_two_pos_of_ne_zero
deleted theorem pow_two_sub_pow_two
deleted theorem ring_hom.map_pow
deleted theorem semiconj_by.gpow_right
deleted theorem sq_sub_sq
deleted theorem sub_nsmul_nsmul_add
deleted theorem zero_gsmul
deleted theorem zero_pow
deleted theorem nat.mul_pow
deleted theorem nat.one_pow
deleted theorem nat.pos_pow_of_pos
deleted theorem nat.pow_add
deleted theorem nat.pow_dvd_pow
deleted theorem nat.pow_dvd_pow_of_dvd
deleted theorem nat.pow_eq_mul_pow_sub
deleted theorem nat.pow_le_pow_of_le_left
deleted theorem nat.pow_one
deleted theorem nat.pow_pos
deleted theorem nat.pow_succ
deleted theorem nat.pow_two
deleted theorem nat.pow_zero
deleted theorem nat.zero_pow