Skip to content

Commit c19d3b3

Browse files
committed
fix
1 parent 3fd8de6 commit c19d3b3

File tree

1 file changed

+1
-1
lines changed

1 file changed

+1
-1
lines changed

src/Init/Data/Dyadic/Round.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -28,7 +28,7 @@ theorem roundDown_le {x : Dyadic} {prec : Int} : roundDown x prec ≤ x :=
2828
match h : k - prec with
2929
| .ofNat l =>
3030
dsimp
31-
rw [ofOdd_eq_ofIntWithPrec, le_iff_toRat]
31+
rw [ofOdd_eq_ofIntWithPrec, ← toRat_le_toRat_iff]
3232
replace h : k = Int.ofNat l + prec := by omega
3333
subst h
3434
simp only [toRat_ofIntWithPrec_eq_mul_two_pow]

0 commit comments

Comments
 (0)