Skip to content

Commit d2cb56b

Browse files
committed
Add simp theorem
1 parent dfefd45 commit d2cb56b

File tree

1 file changed

+1
-0
lines changed

1 file changed

+1
-0
lines changed

src/Init/Data/BitVec/Bitblast.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -1810,6 +1810,7 @@ theorem toNat_pos_of_ne_zero {x : BitVec w} (hx : x ≠ 0#w) :
18101810
simp [toNat_eq] at hx
18111811
omega
18121812

1813+
@[simp]
18131814
theorem toInt_umod_neg_add {x y : BitVec w} (humod : ¬y.toInt ∣ x.toInt) (hymsb : y.msb = true) (hxmsb : x.msb = false) :
18141815
(x % -y + y).toInt = x.toInt % y.toInt + y.toInt := by
18151816
rcases w with _|w ; simp [of_length_zero]

0 commit comments

Comments
 (0)