Documentation

Init.Data.SInt.Lemmas

Equations
  • One or more equations did not get rendered due to their size.
Instances For
    @[simp]
    theorem Int8.lt_def {a b : Int8} :
    @[simp]
    @[simp]
    @[simp]
    @[simp]
    @[simp]
    @[simp]
    @[simp]
    theorem Int8.neg_zero :
    -0 = 0
    @[simp]
    theorem Int16.neg_zero :
    -0 = 0
    @[simp]
    theorem Int32.neg_zero :
    -0 = 0
    @[simp]
    theorem Int64.neg_zero :
    -0 = 0
    @[simp]
    theorem ISize.neg_zero :
    -0 = 0
    theorem ISize.toInt_ofInt {n : Int} (hn : -2 ^ 31 n) (hn' : n < 2 ^ 31) :
    (ofInt n).toInt = n
    theorem ISize.toNatClampNeg_ofInt_eq_zero {n : Int} (hn : -2 ^ 31 n) (hn' : n 0) :
    theorem ISize.neg_ofInt {n : Int} :
    theorem ISize.neg_ofNat {n : Nat} :
    -ofNat n = ofInt (-n)
    theorem ISize.toInt_ofNat_of_lt {n : Nat} (h : n < 2 ^ 31) :
    (ofNat n).toInt = n
    theorem ISize.toInt_neg_ofNat_of_le {n : Nat} (h : n 2 ^ 31) :
    (-ofNat n).toInt = -n