Documentation
Mathlib
.
Algebra
.
Ring
.
Subring
.
Units
Search
return to top
source
Imports
Init
Mathlib.Algebra.Group.Subgroup.Defs
Mathlib.Algebra.Group.Submonoid.Operations
Mathlib.Algebra.Order.GroupWithZero.Submonoid
Mathlib.Algebra.Order.Ring.Defs
Imported by
Units
.
posSubgroup
Units
.
mem_posSubgroup
Unit subgroups of a ring
#
source
def
Units
.
posSubgroup
(R :
Type
u_1)
[
LinearOrderedSemiring
R
]
:
Subgroup
R
ˣ
The subgroup of positive units of a linear ordered semiring.
Equations
Units.posSubgroup
R
=
{
carrier
:=
{
x
:
R
ˣ
|
0
<
↑
x
}
,
mul_mem'
:=
⋯
,
one_mem'
:=
⋯
,
inv_mem'
:=
⋯
}
Instances For
source
@[simp]
theorem
Units
.
mem_posSubgroup
{R :
Type
u_1}
[
LinearOrderedSemiring
R
]
(u :
R
ˣ
)
:
u
∈
posSubgroup
R
↔
0
<
↑
u