Documentation

Mathlib.Algebra.CharP.IntermediateField

Characteristic of intermediate fields #

This file contains some convenient instances for determining the characteristic of intermediate fields. Some char zero instances are not provided, since they are already covered by SubsemiringClass.instCharZero.

instance Subfield.charP {F : Type u_1} [Field F] (L : Subfield F) (p : ) [CharP F p] :
CharP (L) p
Equations
  • =
instance Subfield.expChar {F : Type u_1} [Field F] (L : Subfield F) (p : ) [ExpChar F p] :
ExpChar (L) p
Equations
  • =
instance IntermediateField.charZero {F : Type u_1} {E : Type u_2} [Field F] [Field E] [Algebra F E] (L : IntermediateField F E) [CharZero F] :
Equations
  • =
instance IntermediateField.charP {F : Type u_1} {E : Type u_2} [Field F] [Field E] [Algebra F E] (L : IntermediateField F E) (p : ) [CharP F p] :
CharP (L) p
Equations
  • =
instance IntermediateField.expChar {F : Type u_1} {E : Type u_2} [Field F] [Field E] [Algebra F E] (L : IntermediateField F E) (p : ) [ExpChar F p] :
ExpChar (L) p
Equations
  • =
instance IntermediateField.charP' {F : Type u_1} {E : Type u_2} [Field F] [Field E] [Algebra F E] (L : IntermediateField F E) (p : ) [CharP E p] :
CharP (L) p
Equations
  • =
instance IntermediateField.expChar' {F : Type u_1} {E : Type u_2} [Field F] [Field E] [Algebra F E] (L : IntermediateField F E) (p : ) [ExpChar E p] :
ExpChar (L) p
Equations
  • =