Instances for concrete types #
Equations
- Lean.Grind.instToIntIntIi = { toInt := id, toInt_inj := Lean.Grind.instToIntIntIi._proof_1, toInt_mem := Lean.Grind.instToIntIntIi._proof_2 }
Equations
- Lean.Grind.instToIntNatCiOfNatInt = { toInt := Nat.cast, toInt_inj := Lean.Grind.instToIntNatCiOfNatInt._proof_2, toInt_mem := Lean.Grind.instToIntNatCiOfNatInt._proof_1 }
Equations
- Lean.Grind.instToIntFinCoOfNatIntCast = { toInt := fun (x : Fin n) => ↑↑x, toInt_inj := ⋯, toInt_mem := ⋯ }
instance
Lean.Grind.instZeroFinCoOfNatIntCast
{n : Nat}
[NeZero n]
:
ToInt.Zero (Fin n) (IntInterval.co 0 ↑n)
instance
Lean.Grind.instOfNatFinCoOfNatIntCast
{n : Nat}
[NeZero n]
:
ToInt.OfNat (Fin n) (IntInterval.co 0 ↑n)
Equations
- Lean.Grind.instToIntUInt8UintOfNatNat = { toInt := fun (x : UInt8) => ↑x.toNat, toInt_inj := Lean.Grind.instToIntUInt8UintOfNatNat._proof_2, toInt_mem := ⋯ }
Equations
- Lean.Grind.instToIntUInt16UintOfNatNat = { toInt := fun (x : UInt16) => ↑x.toNat, toInt_inj := Lean.Grind.instToIntUInt16UintOfNatNat._proof_2, toInt_mem := ⋯ }
Equations
- Lean.Grind.instToIntUInt32UintOfNatNat = { toInt := fun (x : UInt32) => ↑x.toNat, toInt_inj := Lean.Grind.instToIntUInt32UintOfNatNat._proof_2, toInt_mem := ⋯ }
Equations
- Lean.Grind.instToIntUInt64UintOfNatNat = { toInt := fun (x : UInt64) => ↑x.toNat, toInt_inj := Lean.Grind.instToIntUInt64UintOfNatNat._proof_2, toInt_mem := ⋯ }
Equations
- Lean.Grind.instToIntUSizeUintNumBits = { toInt := fun (x : USize) => ↑x.toNat, toInt_inj := Lean.Grind.instToIntUSizeUintNumBits._proof_1, toInt_mem := ⋯ }
Equations
- Lean.Grind.instToIntInt8SintOfNatNat = { toInt := fun (x : Int8) => x.toInt, toInt_inj := Lean.Grind.instToIntInt8SintOfNatNat._proof_2, toInt_mem := ⋯ }
Equations
- Lean.Grind.instToIntInt16SintOfNatNat = { toInt := fun (x : Int16) => x.toInt, toInt_inj := Lean.Grind.instToIntInt16SintOfNatNat._proof_2, toInt_mem := ⋯ }
Equations
- Lean.Grind.instToIntInt32SintOfNatNat = { toInt := fun (x : Int32) => x.toInt, toInt_inj := Lean.Grind.instToIntInt32SintOfNatNat._proof_2, toInt_mem := ⋯ }
Equations
- Lean.Grind.instToIntInt64SintOfNatNat = { toInt := fun (x : Int64) => x.toInt, toInt_inj := Lean.Grind.instToIntInt64SintOfNatNat._proof_2, toInt_mem := ⋯ }
Equations
- Lean.Grind.instToIntISizeSintNumBits = { toInt := fun (x : ISize) => x.toInt, toInt_inj := Lean.Grind.instToIntISizeSintNumBits._proof_2, toInt_mem := ⋯ }