Equal and mixed characteristic #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In commutative algebra, some statments are simpler when working over a ℚ
-algebra R
, in which
case one also says that the ring has "equal characteristic zero". A ring that is not a
ℚ
-algebra has either positive characteristic or there exists a prime ideal I ⊂ R
such that
the quotient R ⧸ I
has positive characteristic p > 0
. In this case one speaks of
"mixed characteristic (0, p)
", where p
is only unique if R
is local.
Examples of mixed characteristic rings are ℤ
or the p
-adic integers/numbers.
This file provides the main theorem split_by_characteristic
that splits any proposition P
into
the following three cases:
- Positive characteristic:
char_p R p
(wherep ≠ 0
) - Equal characteristic zero:
algebra ℚ R
- Mixed characteristic:
mixed_char_zero R p
(wherep
is prime)
Main definitions #
mixed_char_zero
: A ring has mixed characteristic(0, p)
if it has characteristic zero and there exists an ideal such that the quotientR ⧸ I
has characteristicp
.
Main results #
split_equal_mixed_char
: Split a statement into equal/mixed characteristic zero.
This main theorem has the following three corollaries which include the positive characteristic case for convenience:
split_by_characteristic
: Generally consider positive charp ≠ 0
.split_by_characteristic_domain
: In a domain we can assume thatp
is prime.split_by_characteristic_local_ring
: In a local ring we can assume thatp
is a prime power.
TODO #
- Relate mixed characteristic in a local ring to p-adic numbers [number_theory.padics].
Mixed characteristic #
A ring of characteristic zero is of "mixed characteristic (0, p)
" if there exists an ideal
such that the quotient R ⧸ I
has caracteristic p
.
Remark: For p = 0
, mixed_char R 0
is a meaningless definition as R ⧸ ⊥ ≅ R
has by
definition always characteristic zero.
One could require (I ≠ ⊥)
in the definition, but then mixed_char R 0
would mean something
like ℤ
-algebra of extension degree ≥ 1
and would be completely independent from
whether something is a ℚ
-algebra or not (e.g. ℚ[X]
would satisfy it but ℚ
wouldn't).
Reduction to p
prime: When proving any statement P
about mixed characteristic rings we
can always assume that p
is prime.
Reduction to I
prime ideal: When proving statements about mixed characteristic rings,
after we reduced to p
prime, we can assume that the ideal I
in the definition is maximal.
Equal characteristic zero #
A commutative ring R
has "equal characteristic zero" if it satisfies one of the following
equivalent properties:
R
is aℚ
-algebra.- The quotient
R ⧸ I
has characteristic zero for any proper idealI ⊂ R
. R
has characteristic zero and does not have mixed characteristic for any primep
.
We show (1) ↔ (2) ↔ (3)
, and most of the following is concerned with constructing
an explicit algebra map ℚ →+* R
(given by x ↦ (x.num : R) /ₚ ↑x.pnat_denom
)
for the direction (1) ← (2)
.
Note: Property (2)
is denoted as equal_char_zero
in the statement names below.
Equal characteristic implies ℚ
-algebra.
Equations
- equal_char_zero_to_Q_algebra R h = {to_fun := λ (x : ℚ), ↑(x.num) /ₚ ↑(x.pnat_denom), map_one' := _, map_mul' := _, map_zero' := _, map_add' := _}.to_algebra
Splitting statements into different characteristic #
Statements to split a proof by characteristic. There are 3 theorems here that are very
similar. They only differ in the assumptions we can make on the positive characteristic
case:
Generally we need to consider all p ≠ 0
, but if R
is a local ring, we can assume
that p
is a prime power. And if R
is a domain, we can even assume that p
is prime.
Split any Prop
over R
into the three cases:
- positive characteristic.
- equal characteristic zero.
- mixed characteristic
(0, p)
.
In a is_domain R
, split any Prop
over R
into the three cases:
- prime characteristic.
- equal characteristic zero.
- mixed characteristic
(0, p)
.
In a local_ring R
, split any Prop
over R
into the three cases:
- prime power characteristic.
- equal characteristic zero.
- mixed characteristic
(0, p)
.