Documentation

Mathlib.Algebra.CharP.Subring

Characteristic of subrings #

instance CharP.subsemiring (R : Type u) [Semiring R] (p : ) [CharP R p] (S : Subsemiring R) :
CharP (S) p
Equations
  • =
instance CharP.subring (R : Type u) [Ring R] (p : ) [CharP R p] (S : Subring R) :
CharP (S) p
Equations
  • =
instance CharP.subring' (R : Type u) [CommRing R] (p : ) [CharP R p] (S : Subring R) :
CharP (S) p
Equations
  • =