Documentation

Mathlib.Algebra.Ring.Int

The integers are a ring #

This file contains the commutative ring instance on .

See note [foundational algebra order theory].

@[simp]
theorem Int.cast_mul {α : Type u_1} [NonAssocRing α] (m : ) (n : ) :
(m * n) = m * n
@[simp]
theorem Int.cast_pow {R : Type u_1} [Ring R] (n : ) (m : ) :
(n ^ m) = n ^ m

Extra instances to short-circuit type class resolution #

These also prevent non-computable instances like Int.normedCommRing being used to construct these instances non-computably.

Equations
Equations
Equations