Documentation

Mathlib.Data.Int.Cast.Basic

Cast of integers (additional theorems) #

This file proves additional properties about the canonical homomorphism from the integers into an additive group with a one (Int.cast).

There is also Data.Int.Cast.Lemmas, which includes lemmas stated in terms of algebraic homomorphisms, and results involving the order structure of .

By contrast, this file's only import beyond Data.Int.Cast.Defs is Algebra.Group.Basic.

theorem Nat.cast_sub {R : Type u} [AddGroupWithOne R] {m n : Nat} (h : LE.le m n) :
theorem Nat.cast_pred {R : Type u} [AddGroupWithOne R] {n : Nat} :
LT.lt 0 nEq (HSub.hSub n 1).cast (HSub.hSub n.cast 1)
theorem Int.cast_neg {R : Type u} [AddGroupWithOne R] (n : Int) :
theorem Int.cast_add {R : Type u} [AddGroupWithOne R] (m n : Int) :
theorem Int.cast_sub {R : Type u} [AddGroupWithOne R] (m n : Int) :
theorem zsmul_one {R : Type u_1} [AddGroupWithOne R] (n : Int) :