Documentation

Mathlib.RingTheory.Subring.Order

Subrings of ordered rings #

We study subrings of ordered rings and prove their basic properties.

Main definitions and results #

instance SubringClass.toOrderedRing {R : Type u_1} {S : Type u_2} [SetLike S R] (s : S) [OrderedRing R] [SubringClass S R] :

A subring of an OrderedRing is an OrderedRing.

Equations
instance SubringClass.toOrderedCommRing {R : Type u_1} {S : Type u_2} [SetLike S R] (s : S) [OrderedCommRing R] [SubringClass S R] :

A subring of an OrderedCommRing is an OrderedCommRing.

Equations
instance SubringClass.toLinearOrderedRing {R : Type u_1} {S : Type u_2} [SetLike S R] (s : S) [LinearOrderedRing R] [SubringClass S R] :

A subring of a LinearOrderedRing is a LinearOrderedRing.

Equations

A subring of a LinearOrderedCommRing is a LinearOrderedCommRing.

Equations
def Subring.orderedSubtype {R : Type u_2} [OrderedRing R] (s : Subring R) :
s →+*o R

The inclusion S → R of a subring, as an ordered ring homomorphism.

Equations
Instances For