Documentation

Mathlib.Data.ZMod.Defs

Definition of ZMod n + basic results. #

This file provides the basic details of ZMod n, including its commutative ring structure.

Implementation details #

This used to be inlined into Data.ZMod.Basic. This file imports CharP.Lemmas, which is an issue; all CharP instances create an Algebra (ZMod p) R instance; however, this instance may not be definitionally equal to other Algebra instances (for example, GaloisField also has an Algebra instance as it is defined as a SplittingField). The way to fix this is to use the forgetful inheritance pattern, and make CharP carry the data of what the smul should be (so for example, the smul on the GaloisField CharP instance should be equal to the smul from its SplittingField structure); there is only one possible ZMod p algebra for any p, so this is not an issue mathematically. For this to be possible, however, we need CharP.Lemmas to be able to import some part of ZMod.

Ring structure on Fin n #

We define a commutative ring structure on Fin n. Afterwards, when we define ZMod n in terms of Fin n, we use these definitions to register the ring structure on ZMod n as type class instance.

Multiplicative commutative semigroup structure on Fin n.

Equations
instance Fin.instDistrib (n : ) :

Distributive structure on Fin n.

Equations
Equations
  • One or more equations did not get rendered due to their size.
instance Fin.instCommMonoid (n : ) [NeZero n] :
Equations
  • One or more equations did not get rendered due to their size.

Note this is more general than Fin.instCommRing as it applies (vacuously) to Fin 0 too.

Equations

Commutative ring structure on Fin n.

This is not a global instance, but can introduced locally using open Fin.CommRing in ....

This is not an instance because the binop% elaborator assumes that htere are no non-trivial coercion loops, but this instance would introduce a coercion from Nat to Fin n and back. Non-trivial loops lead to undesirable and counterintuitive elaboration behavior.

For example, for x : Fin k and n : Nat, it causes x < n to be elaborated as x < ↑n rather than ↑x < n, silently introducing wraparound arithmetic.

Equations
  • One or more equations did not get rendered due to their size.
Instances For
    def ZMod :
    Type

    The integers modulo n : ℕ.

    Equations
    Instances For
      instance ZMod.fintype (n : ) [NeZero n] :
      Equations
      @[simp]
      theorem ZMod.card (n : ) [Fintype (ZMod n)] :
      instance ZMod.commRing (n : ) :
      Equations
      • One or more equations did not get rendered due to their size.
      instance ZMod.inhabited (n : ) :
      Equations