Localizations away from an element #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
Main definitions #
is_localization.away (x : R) S
expresses thatS
is a localization away fromx
, as an abbreviation ofis_localization (submonoid.powers x) S
exists_reduced_fraction (hb : b ≠ 0)
produces a reduced fraction of the formb = a * x^n
for somen : ℤ
and somea : R
that is not divisible byx
.
Implementation notes #
See src/ring_theory/localization/basic.lean
for a design overview.
Tags #
localization, ring localization, commutative ring localization, characteristic predicate, commutative ring, field of fractions
Given x : R
, the typeclass is_localization.away x S
states that S
is
isomorphic to the localization of R
at the submonoid generated by x
.
Given x : R
and a localization map F : R →+* S
away from x
, inv_self
is (F x)⁻¹
.
Equations
- is_localization.away.inv_self x = is_localization.mk' S 1 ⟨x, _⟩
Given x : R
, a localization map F : R →+* S
away from x
, and a map of comm_semiring
s
g : R →+* P
such that g x
is invertible, the homomorphism induced from S
to P
sending
z : S
to g y * (g x)⁻ⁿ
, where y : R, n : ℕ
are such that z = F y * (F x)⁻ⁿ
.
Equations
Given x y : R
and localizations S
, P
away from x
and x * y
respectively, the homomorphism induced from S
to P
.
Equations
Given a map f : R →+* S
and an element r : R
, we may construct a map Rᵣ →+* Sᵣ
.
Equations
- is_localization.away.map S Q f r = is_localization.map Q f _
The localization at a module of units is isomorphic to the ring
Equations
- is_localization.at_units R M S H = alg_equiv.of_bijective (algebra.of_id R S) _
The localization away from a unit is isomorphic to the ring
Equations
- is_localization.at_unit R S x e = is_localization.at_units R (submonoid.powers x) S _
The localization at one is isomorphic to the ring.
Equations
- is_localization.at_one R S = is_localization.at_unit R S 1 _
Given a map f : R →+* S
and an element r : R
, such that f r
is invertible,
we may construct a map Rᵣ →+* S
.
Given a map f : R →+* S
and an element r : R
, we may construct a map Rᵣ →+* Sᵣ
.
self_zpow x (m : ℤ)
is x ^ m
as an element of the localization away from x
.
Equations
- self_zpow x B m = dite (0 ≤ m) (λ (hm : 0 ≤ m), ⇑(algebra_map R B) x ^ m.nat_abs) (λ (hm : ¬0 ≤ m), is_localization.mk' B 1 (submonoid.pow x m.nat_abs))