mathlib documentation

ring_theory.​principal_ideal_domain

ring_theory.​principal_ideal_domain

Principal ideal rings and principal ideal domains

A principal ideal ring (PIR) is a commutative ring in which all ideals are principal. A principal ideal domain (PID) is an integral domain which is a principal ideal ring.

Main definitions

Note that for principal ideal domains, one should use [integral domain R] [is_principal_ideal_ring R]. There is no explicit definition of a PID. Theorems about PID's are in the principal_ideal_ring namespace.

Main results

@[class]
structure submodule.​is_principal {R : Type u} {M : Type v} [ring R] [add_comm_group M] [module R M] :
submodule R M → Prop

An R-submodule of M is principal if it is generated by one element.

Instances
@[class]
structure is_principal_ideal_ring (R : Type u) [comm_ring R] :
Prop

A commutative ring is a principal ideal ring if all ideals are principal.

Instances
def submodule.​is_principal.​generator {R : Type u} {M : Type v} [comm_ring R] [add_comm_group M] [module R M] (S : submodule R M) [S.is_principal] :
M

generator I, if I is a principal submodule, is the x ∈ M such that span R {x} = I

Equations
theorem submodule.​is_principal.​mem_iff_eq_smul_generator {R : Type u} {M : Type v} [comm_ring R] [add_comm_group M] [module R M] (S : submodule R M) [S.is_principal] {x : M} :

theorem is_prime.​to_maximal_ideal {R : Type u} [integral_domain R] [is_principal_ideal_ring R] {S : ideal R} [hpi : S.is_prime] :

theorem mod_mem_iff {R : Type u} [euclidean_domain R] {S : ideal R} {x y : R} :
y S(x % y S x S)

factors a is a multiset of irreducible elements whose product is a, up to units

Equations

The unique factorization domain structure given by the principal ideal domain.

This is not added as type class instance, since the factors might be computed in a different way. E.g. factors could return normalized values.

Equations