Documentation

Mathlib.Algebra.Ring.Semireal.Defs

Semireal rings #

A semireal ring is a commutative ring (with unit) in which -1 is not a sum of squares.

For instance, linearly ordered rings are semireal, because sums of squares are positive and -1 is not.

Main declaration #

References #

class IsSemireal (R : Type u_1) [Add R] [Mul R] [One R] [Zero R] :

A semireal ring is a commutative ring (with unit) in which -1 is not a sum of squares. We define the predicate IsSemireal R for structures R equipped with a multiplication, an addition, a multiplicative unit and an additive unit.

Instances
    theorem isSemireal_iff (R : Type u_1) [Add R] [Mul R] [One R] [Zero R] :
    IsSemireal R ∀ {s : R}, IsSumSq s1 + s 0
    @[deprecated IsSemireal (since := "2024-08-09")]
    def isSemireal (R : Type u_1) [Add R] [Mul R] [One R] [Zero R] :

    Alias of IsSemireal.


    A semireal ring is a commutative ring (with unit) in which -1 is not a sum of squares. We define the predicate IsSemireal R for structures R equipped with a multiplication, an addition, a multiplicative unit and an additive unit.

    Equations
    Instances For
      theorem IsSemireal.not_isSumSq_neg_one {R : Type u_1} [AddGroup R] [One R] [Mul R] [IsSemireal R] :

      In a semireal ring, -1 is not a sum of squares.

      @[deprecated IsSemireal.not_isSumSq_neg_one (since := "2024-08-09")]
      theorem isSemireal.neg_one_not_SumSq {R : Type u_1} [AddGroup R] [One R] [Mul R] [IsSemireal R] :

      Alias of IsSemireal.not_isSumSq_neg_one.


      In a semireal ring, -1 is not a sum of squares.

      Linearly ordered semirings with the property a ≤ b → ∃ c, a + c = b (e.g. ) are semireal.