We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent dfefd45 commit d2cb56bCopy full SHA for d2cb56b
src/Init/Data/BitVec/Bitblast.lean
@@ -1810,6 +1810,7 @@ theorem toNat_pos_of_ne_zero {x : BitVec w} (hx : x ≠ 0#w) :
1810
simp [toNat_eq] at hx
1811
omega
1812
1813
+@[simp]
1814
theorem toInt_umod_neg_add {x y : BitVec w} (humod : ¬y.toInt ∣ x.toInt) (hymsb : y.msb = true) (hxmsb : x.msb = false) :
1815
(x % -y + y).toInt = x.toInt % y.toInt + y.toInt := by
1816
rcases w with _|w ; simp [of_length_zero]
0 commit comments