Documentation

Mathlib.Tactic.NormNum.OfScientific

norm_num plugin for scientific notation. #

theorem Mathlib.Meta.NormNum.isRat_ofScientific_of_true {α : Type u_1} [DivisionRing α] {m e : } {n : } {d : } :
IsRat (↑(mkRat (↑m) (10 ^ e))) n dIsRat (OfScientific.ofScientific m true e) n d
theorem Mathlib.Meta.NormNum.isNat_ofScientific_of_false {α : Type u_1} [DivisionRing α] {m e nm ne n : } :
IsNat m nmIsNat e nen = nm.mul (10 ^ ne)IsNat (OfScientific.ofScientific m false e) n

The norm_num extension which identifies expressions in scientific notation, normalizing them to rat casts if the scientific notation is inherited from the one for rationals.

Equations
  • One or more equations did not get rendered due to their size.
Instances For