Documentation

Mathlib.Data.Int.Cast.Pi

Cast of integers to function types #

This file provides a (pointwise) cast from to function types.

Main declarations #

instance Pi.instIntCast {ι : Type u_1} {π : ιType u_2} [(i : ι) → IntCast (π i)] :
IntCast ((i : ι) → π i)
Equations
  • Pi.instIntCast = { intCast := fun (n : ) (x : ι) => n }
theorem Pi.intCast_apply {ι : Type u_1} {π : ιType u_2} [(i : ι) → IntCast (π i)] (n : ) (i : ι) :
n i = n
@[simp]
theorem Pi.intCast_def {ι : Type u_1} {π : ιType u_2} [(i : ι) → IntCast (π i)] (n : ) :
n = fun (x : ι) => n
@[deprecated Pi.intCast_apply]
theorem Pi.int_apply {ι : Type u_1} {π : ιType u_2} [(i : ι) → IntCast (π i)] (n : ) (i : ι) :
n i = n

Alias of Pi.intCast_apply.

@[deprecated Pi.intCast_def]
theorem Pi.coe_int {ι : Type u_1} {π : ιType u_2} [(i : ι) → IntCast (π i)] (n : ) :
n = fun (x : ι) => n

Alias of Pi.intCast_def.

theorem Sum.elim_intCast_intCast {α : Type u_1} {β : Type u_2} {γ : Type u_3} [IntCast γ] (n : ) :
Sum.elim n n = n