Commit
This commit does not belong to any branch on this repository, and may belong to a fork outside of the repository.
chore: change BitVec.intMin/Max from abbrev to def (#5252)
I don't think we gain anything from having them as `abbrev` here, and the simpNF linter complains: ``` -- Init.Data.BitVec.Lemmas #check @BitVec.toNat_intMin /- simp can prove this: by simp only [BitVec.toNat_twoPow] One of the lemmas above could be a duplicate. If that's not the case try reordering lemmas or adding @[priority]. -/ #check @BitVec.toNat_intMax /- Left-hand side simplifies from (BitVec.intMax w).toNat to (2 ^ w - 1 % 2 ^ w + 2 ^ (w - 1)) % 2 ^ w using simp only [@BitVec.toNat_sub, @BitVec.ofNat_eq_ofNat, BitVec.toNat_ofNat, BitVec.toNat_twoPow, Nat.add_mod_mod] Try to change the left-hand side to the simplified term! -/ ```
- Loading branch information