Documentation

Mathlib.Algebra.CharP.Reduced

Results about characteristic p reduced rings #

theorem iterateFrobenius_inj (R : Type u_1) [CommRing R] [IsReduced R] (p : ) (n : ) [ExpChar R p] :
theorem frobenius_inj (R : Type u_1) [CommRing R] [IsReduced R] (p : ) [ExpChar R p] :
theorem isSquare_of_charTwo' {R : Type u_1} [Finite R] [CommRing R] [IsReduced R] [CharP R 2] (a : R) :

If ringChar R = 2, where R is a finite reduced commutative ring, then every a : R is a square.

@[simp]
theorem ExpChar.pow_prime_pow_mul_eq_one_iff {R : Type u_1} [CommRing R] [IsReduced R] (p : ) (k : ) (m : ) [ExpChar R p] (x : R) :
x ^ (p ^ k * m) = 1 x ^ m = 1
@[deprecated ExpChar.pow_prime_pow_mul_eq_one_iff]
theorem CharP.pow_prime_pow_mul_eq_one_iff {R : Type u_1} [CommRing R] [IsReduced R] (p : ) (k : ) (m : ) [ExpChar R p] (x : R) :
x ^ (p ^ k * m) = 1 x ^ m = 1

Alias of ExpChar.pow_prime_pow_mul_eq_one_iff.