Pull back ordered groups along injective maps. #
@[reducible]
def
Function.Injective.orderedAddCommGroup
{α : Type u_1}
[OrderedAddCommGroup α]
{β : Type u_3}
[Zero β]
[Add β]
[Neg β]
[Sub β]
[SMul ℕ β]
[SMul ℤ β]
(f : β → α)
(hf : Function.Injective f)
(one : f 0 = 0)
(mul : ∀ (x y : β), f (x + y) = f x + f y)
(inv : ∀ (x : β), f (-x) = -f x)
(div : ∀ (x y : β), f (x - y) = f x - f y)
(npow : ∀ (x : β) (n : ℕ), f (n • x) = n • f x)
(zpow : ∀ (x : β) (n : ℤ), f (n • x) = n • f x)
 :
Pullback an OrderedAddCommGroup under an injective map.
Equations
- Function.Injective.orderedAddCommGroup f hf one mul inv div npow zpow = let __spread.0 := Function.Injective.orderedAddCommMonoid f hf one mul npow; OrderedAddCommGroup.mk ⋯
Instances For
@[reducible]
def
Function.Injective.orderedCommGroup
{α : Type u_1}
[OrderedCommGroup α]
{β : Type u_3}
[One β]
[Mul β]
[Inv β]
[Div β]
[Pow β ℕ]
[Pow β ℤ]
(f : β → α)
(hf : Function.Injective f)
(one : f 1 = 1)
(mul : ∀ (x y : β), f (x * y) = f x * f y)
(inv : ∀ (x : β), f x⁻¹ = (f x)⁻¹)
(div : ∀ (x y : β), f (x / y) = f x / f y)
(npow : ∀ (x : β) (n : ℕ), f (x ^ n) = f x ^ n)
(zpow : ∀ (x : β) (n : ℤ), f (x ^ n) = f x ^ n)
 :
Pullback an OrderedCommGroup under an injective map.
See note [reducible non-instances].
Equations
- Function.Injective.orderedCommGroup f hf one mul inv div npow zpow = let __spread.0 := Function.Injective.orderedCommMonoid f hf one mul npow; OrderedCommGroup.mk ⋯
Instances For
@[reducible]
def
Function.Injective.linearOrderedAddCommGroup
{α : Type u_1}
[LinearOrderedAddCommGroup α]
{β : Type u_3}
[Zero β]
[Add β]
[Neg β]
[Sub β]
[SMul ℕ β]
[SMul ℤ β]
[Sup β]
[Inf β]
(f : β → α)
(hf : Function.Injective f)
(one : f 0 = 0)
(mul : ∀ (x y : β), f (x + y) = f x + f y)
(inv : ∀ (x : β), f (-x) = -f x)
(div : ∀ (x y : β), f (x - y) = f x - f y)
(npow : ∀ (x : β) (n : ℕ), f (n • x) = n • f x)
(zpow : ∀ (x : β) (n : ℤ), f (n • x) = n • f x)
(sup : ∀ (x y : β), f (x ⊔ y) = max (f x) (f y))
(inf : ∀ (x y : β), f (x ⊓ y) = min (f x) (f y))
 :
Pullback a LinearOrderedAddCommGroup under an injective map.
Equations
- One or more equations did not get rendered due to their size.
Instances For
@[reducible]
def
Function.Injective.linearOrderedCommGroup
{α : Type u_1}
[LinearOrderedCommGroup α]
{β : Type u_3}
[One β]
[Mul β]
[Inv β]
[Div β]
[Pow β ℕ]
[Pow β ℤ]
[Sup β]
[Inf β]
(f : β → α)
(hf : Function.Injective f)
(one : f 1 = 1)
(mul : ∀ (x y : β), f (x * y) = f x * f y)
(inv : ∀ (x : β), f x⁻¹ = (f x)⁻¹)
(div : ∀ (x y : β), f (x / y) = f x / f y)
(npow : ∀ (x : β) (n : ℕ), f (x ^ n) = f x ^ n)
(zpow : ∀ (x : β) (n : ℤ), f (x ^ n) = f x ^ n)
(sup : ∀ (x y : β), f (x ⊔ y) = max (f x) (f y))
(inf : ∀ (x y : β), f (x ⊓ y) = min (f x) (f y))
 :
Pullback a LinearOrderedCommGroup under an injective map.
See note [reducible non-instances].
Equations
- One or more equations did not get rendered due to their size.