Cast of naturals into fields #
This file concerns the canonical homomorphism ℕ → F
, where F
is a field.
Main results #
Nat.cast_div
: ifn
dividesm
, then↑(m / n) = ↑m / ↑n
@[simp]
@[simp]
theorem
Nat.cast_div_charZero
{K : Type u_1}
[DivisionSemiring K]
{m n : ℕ}
[CharZero K]
(hnm : n ∣ m)
: