Documentation

Mathlib.Algebra.CharP.ExpChar

Exponential characteristic #

This file defines the exponential characteristic, which is defined to be 1 for a ring with characteristic 0 and the same as the ordinary characteristic, if the ordinary characteristic is prime. This concept is useful to simplify some theorem statements. This file establishes a few basic results relating it to the (ordinary characteristic). The definition is stated for a semiring, but the actual results are for nontrivial rings (as far as exponential characteristic one is concerned), respectively a ring without zero-divisors (for prime characteristic).

Main results #

Tags #

exponential characteristic, characteristic

def LinearMap.frobenius (R : Type u) [CommSemiring R] (S : Type u_1) [CommSemiring S] (p : ) [ExpChar R p] [ExpChar S p] [Algebra R S] :

The frobenius map of an algebra as a frobenius-semilinear map.

Equations
Instances For
    def LinearMap.iterateFrobenius (R : Type u) [CommSemiring R] (S : Type u_1) [CommSemiring S] (p : ) (n : ) [ExpChar R p] [ExpChar S p] [Algebra R S] :

    The iterated frobenius map of an algebra as a iterated-frobenius-semilinear map.

    Equations
    Instances For
      theorem LinearMap.frobenius_def (R : Type u) [CommSemiring R] (S : Type u_1) [CommSemiring S] (p : ) [ExpChar R p] [ExpChar S p] [Algebra R S] (x : S) :
      (LinearMap.frobenius R S p) x = x ^ p
      theorem LinearMap.iterateFrobenius_def (R : Type u) [CommSemiring R] (S : Type u_1) [CommSemiring S] (p : ) [ExpChar R p] [ExpChar S p] [Algebra R S] (n : ) (x : S) :
      (LinearMap.iterateFrobenius R S p n) x = x ^ p ^ n
      theorem frobenius_zero (R : Type u) [CommSemiring R] (p : ) [ExpChar R p] :
      (frobenius R p) 0 = 0
      theorem frobenius_add (R : Type u) [CommSemiring R] (p : ) [ExpChar R p] (x : R) (y : R) :
      (frobenius R p) (x + y) = (frobenius R p) x + (frobenius R p) y
      theorem frobenius_natCast (R : Type u) [CommSemiring R] (p : ) [ExpChar R p] (n : ) :
      (frobenius R p) n = n
      @[deprecated frobenius_natCast]
      theorem frobenius_nat_cast (R : Type u) [CommSemiring R] (p : ) [ExpChar R p] (n : ) :
      (frobenius R p) n = n

      Alias of frobenius_natCast.