Skip to content

Commit e4d2652

Browse files
bolluluisacicolini
andauthored
Update src/Init/Data/BitVec/Bitblast.lean
Co-authored-by: Luisa Cicolini <[email protected]>
1 parent 92770de commit e4d2652

File tree

1 file changed

+1
-2
lines changed

1 file changed

+1
-2
lines changed

src/Init/Data/BitVec/Bitblast.lean

Lines changed: 1 addition & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -1798,8 +1798,7 @@ theorem msb_sdiv_eq_decide {x y : BitVec w} :
17981798
· simp only [hy₁, decide_false, Bool.not_false, Bool.and_true]
17991799
by_cases hxy₁ : (- x / y) = 0#w
18001800
· simp only [hxy₁, neg_zero, msb_zero, false_eq_decide_iff, BitVec.not_le]
1801-
simp only [udiv_eq_zero_iff_eq_zero_or_lt] at hxy₁
1802-
simp only [hy₁, _root_.false_or] at hxy₁
1801+
simp only [udiv_eq_zero_iff_eq_zero_or_lt, hy₁, _root_.false_or] at hxy₁
18031802
bv_omega
18041803
· simp only [udiv_eq_zero_iff_eq_zero_or_lt, _root_.not_or, BitVec.not_lt,
18051804
hy₁, not_false_eq_true, _root_.true_and] at hxy₁

0 commit comments

Comments
 (0)