Quadratic characters on ℤ/nℤ #
This file defines some quadratic characters on the rings ℤ/4ℤ and ℤ/8ℤ.
We set them up to be of type MulChar (ZMod n) ℤ
, where n
is 4
or 8
.
Tags #
quadratic character, zmod
Quadratic characters mod 4 and 8 #
We define the primitive quadratic characters χ₄
on ZMod 4
and χ₈
, χ₈'
on ZMod 8
.
@[simp]
@[simp]
theorem
ZMod.χ₈_apply
(a : ZMod 8)
:
ZMod.χ₈ a = match a with
| 0 => 0
| 2 => 0
| 4 => 0
| 6 => 0
| 1 => 1
| 7 => 1
| 3 => -1
| 5 => -1
@[simp]
theorem
ZMod.χ₈'_apply
(a : ZMod 8)
:
ZMod.χ₈' a = match a with
| 0 => 0
| 2 => 0
| 4 => 0
| 6 => 0
| 1 => 1
| 3 => 1
| 5 => -1
| 7 => -1