Properties of the ZNum
representation of integers #
This file was split from Mathlib.Data.Num.Lemmas
to keep the former under 1500 lines.
@[simp]
@[simp]
@[simp]
@[simp]
@[simp]
@[simp]
@[simp]
@[simp]
@[simp]
theorem
ZNum.cast_lt
{α : Type u_1}
[Ring α]
[PartialOrder α]
[IsStrictOrderedRing α]
{m n : ZNum}
:
@[simp]
@[simp]
theorem
ZNum.cast_inj
{α : Type u_1}
[Ring α]
[PartialOrder α]
[IsStrictOrderedRing α]
{m n : ZNum}
:
This tactic tries to turn an (in)equality about ZNum
s to one about Int
s by rewriting.
example (n : ZNum) (m : ZNum) : n ≤ n + m * m := by
transfer_rw
exact le_add_of_nonneg_right (mul_self_nonneg _)
Equations
- ZNum.transfer_rw = Lean.ParserDescr.node `ZNum.transfer_rw 1024 (Lean.ParserDescr.nonReservedSymbol "transfer_rw" false)
Instances For
This tactic tries to prove (in)equalities about ZNum
s by transferring them to the Int
world and
then trying to call simp
.
example (n : ZNum) (m : ZNum) : n ≤ n + m * m := by
transfer
exact mul_self_nonneg _
Equations
- ZNum.transfer = Lean.ParserDescr.node `ZNum.transfer 1024 (Lean.ParserDescr.nonReservedSymbol "transfer" false)
Instances For
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
@[simp]
Equations
- x✝¹.decidableDvd x✝ = decidable_of_iff' (x✝ % x✝¹ = 0) ⋯
Equations
- x✝¹.decidableDvd x✝ = (Num.pos x✝¹).decidableDvd (Num.pos x✝)
Equations
- x✝¹.decidableDvd x✝ = decidable_of_iff' (x✝ % x✝¹ = 0) ⋯