Documentation
Mathlib
.
Algebra
.
GroupWithZero
.
Int
Search
return to top
source
Imports
Init
Mathlib.Algebra.GroupWithZero.WithZero
Mathlib.Algebra.Group.Int.TypeTags
Imported by
WithZero
.
ofAdd_zpow
WithZero
.
ofAdd_neg_one_pow_comm
Lemmas about
ℤₘ₀
.
#
source
theorem
WithZero
.
ofAdd_zpow
(a :
ℤ
)
:
↑
(
Multiplicative.ofAdd
a
)
=
↑
(
Multiplicative.ofAdd
1
)
^
a
source
theorem
WithZero
.
ofAdd_neg_one_pow_comm
(a :
ℤ
)
(n :
ℕ
)
:
(
↑
(
Multiplicative.ofAdd
(-
1
)
)
^
(
-
a
))
^
n
=
↑
(
Multiplicative.ofAdd
↑
n
)
^
a