Documentation
Mathlib
.
Algebra
.
Group
.
Int
.
TypeTags
Search
return to top
source
Imports
Init
Mathlib.Algebra.Group.Int.Defs
Mathlib.Algebra.Group.TypeTags.Basic
Imported by
Int
.
toAdd_pow
Int
.
toAdd_zpow
Int
.
ofAdd_mul
Lemmas about
Multiplicative
ℤ
.
#
source
theorem
Int
.
toAdd_pow
(
a
:
Multiplicative
ℤ
)
(
b
:
ℕ
)
:
Multiplicative.toAdd
(
a
^
b
)
=
Multiplicative.toAdd
a
*
↑
b
source
theorem
Int
.
toAdd_zpow
(
a
:
Multiplicative
ℤ
)
(
b
:
ℤ
)
:
Multiplicative.toAdd
(
a
^
b
)
=
Multiplicative.toAdd
a
*
b
source
@[simp]
theorem
Int
.
ofAdd_mul
(
a
b
:
ℤ
)
:
Multiplicative.ofAdd
(
a
*
b
)
=
Multiplicative.ofAdd
a
^
b