You signed in with another tab or window. Reload to refresh your session.You signed out in another tab or window. Reload to refresh your session.You switched accounts on another tab or window. Reload to refresh your session.Dismiss alert
refactor(NumberTheory/Ostrowski): use AbsoluteValue instead of MulRingNorm (#20362)
This PR
* replaces `MulRingNorm R` by `AbsoluteValue R ℝ` in the material developed in `Mathlib.NumberTheory.Ostrowski`
* does some cleanup (naming convention, remove redundant name parts etc.)
* and also some golfing...
In addition, it
* creates a new folder `Mathlib.Algebra.Order.AbsoluteValue`
* moves `Mathlib.Algebra.Order.AbsoluteValue` to `Mathlib.Algebra.Order.AbsoluteValue.Basic` and `Mathlib.Algebra.Order.EuclideanAbsoluteValue`to `Mathlib.Algebra.Order.AbsoluteValue.Euclidean`
* adds some API for `AbsoluteValue` to match `MulRingNorm` (in `Mathlib.Algebra.Order.AbsoluteValue.Basic`)
* adds a new file `Mathlib.Algebra.Order.AbsoluteValue.Equivalence` with material on equivalence of real-valued absolute values.
See the [discussion](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/MulRingNorm.20vs.2E.20AbsoluteValue/near/491324423) on Zulip.
Co-authored-by: Michael Stoll <99838730+MichaelStollBayreuth@users.noreply.github.com>
0 commit comments