Documentation

Mathlib.Data.Rat.Cast.Lemmas

Some exiled lemmas about casting #

These lemmas have been removed from Mathlib.Data.Rat.Cast.Defs to avoiding needing to import Mathlib.Algebra.Field.Basic there.

In fact, these lemmas don't appear to be used anywhere in Mathlib, so perhaps this file can simply be deleted.

@[simp]
theorem Rat.cast_inv_nat {α : Type u_1} [DivisionRing α] (n : ) :
(n)⁻¹ = (n)⁻¹
@[simp]
theorem Rat.cast_inv_int {α : Type u_1} [DivisionRing α] (n : ) :
(n)⁻¹ = (n)⁻¹
@[simp]
theorem Rat.cast_nnratCast {K : Type u_2} [DivisionRing K] (q : ℚ≥0) :
q = q
@[simp]
theorem Rat.cast_ofScientific {K : Type u_2} [DivisionRing K] (m : ) (s : Bool) (e : ) :

Casting a scientific literal via is the same as casting directly.