Documentation

Mathlib.Algebra.Order.Field.Canonical

Canonically ordered semifields #

@[reducible, inline]

Construct a LinearOrderedCommGroupWithZero from a canonically linear ordered semifield.

Equations
  • One or more equations did not get rendered due to their size.
Instances For
    theorem tsub_div {α : Type u_1} [Semifield α] [LinearOrder α] [CanonicallyOrderedAdd α] [IsStrictOrderedRing α] [Sub α] [OrderedSub α] (a b c : α) :
    (a - b) / c = a / c - b / c