Zulip Chat Archive
Stream: Is there code for X?
Topic: clearing denominators
Jujian Zhang (Mar 12 2022 at 20:01):
Given a finset
of , do we have a lemma to clear their denominators, i.e.
Do we have the following:
import ring_theory.localization.basic
import ring_theory.graded_algebra.basic
section clear_denominator
variables (R : Type*) [comm_ring R] (f : R) [decidable_eq (localization.away f)]
lemma clear_denominator (s : finset (localization.away f)) :
∃ (n : ℕ), ∀ (x : localization.away f), x ∈ s →
x * localization.mk (f^n) 1 ∈
set.range (λ y, (localization.mk y 1 : localization.away f)) := sorry
end clear_denominator
If not, I will pr this and what should this lemma be called?
Johan Commelin (Mar 12 2022 at 20:08):
This generalises to arbitrary localisations, right?
Johan Commelin (Mar 12 2022 at 20:08):
Except that it will not be f^n
, but some random product of denominators.
Andrew Yang (Mar 12 2022 at 20:09):
Stuff related to these are in file#ring_theory/localization/integer. I think you could probably fiddle with them and get what you want.
Jujian Zhang (Mar 12 2022 at 20:13):
Thanks! there is docs#is_localization.common_denom
Last updated: Dec 20 2023 at 11:08 UTC