Skip to content

Commit fdafdd4

Browse files
committed
no need to go through tmod
1 parent e1fb65f commit fdafdd4

File tree

1 file changed

+3
-3
lines changed

1 file changed

+3
-3
lines changed

src/Init/Data/BitVec/Bitblast.lean

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -1846,9 +1846,9 @@ theorem toInt_smod {x y : BitVec w} :
18461846
have hynonpos := toInt_neg_of_msb_true hymsb
18471847
have := (@toInt_dvd_toInt_iff_of_msb_false_msb_true (w + 1) x y hxmsb hymsb)
18481848
simp only [hx_dvd_y, false_iff] at this
1849-
simp only [this, Int.fmod_eq_tmod, Int.tmod_eq_emod_of_nonneg hxnonneg]
1850-
simp [hx_dvd_y, hxnonneg, hymsb, hxmsb, show ¬0 ≤ y.toInt by omega,
1851-
toInt_umod_neg_add hx_dvd_y]
1849+
simp only [this]
1850+
simp only [Int.fmod_eq_emod, show ¬0 ≤ y.toInt by omega]
1851+
simp [hx_dvd_y, hymsb, hxmsb, toInt_umod_neg_add hx_dvd_y]
18521852
· have hynonneg := toInt_nonneg_of_msb_false hymsb
18531853
rw [Int.fmod_eq_emod_of_nonneg x.toInt (b := y.toInt) (by omega)]
18541854
have hdvd := toInt_dvd_toInt_iff_of_msb_true_msb_false hxmsb hymsb

0 commit comments

Comments
 (0)