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 3fd8de6 commit c19d3b3Copy full SHA for c19d3b3
src/Init/Data/Dyadic/Round.lean
@@ -28,7 +28,7 @@ theorem roundDown_le {x : Dyadic} {prec : Int} : roundDown x prec ≤ x :=
28
match h : k - prec with
29
| .ofNat l =>
30
dsimp
31
- rw [ofOdd_eq_ofIntWithPrec, le_iff_toRat]
+ rw [ofOdd_eq_ofIntWithPrec, ← toRat_le_toRat_iff]
32
replace h : k = Int.ofNat l + prec := by omega
33
subst h
34
simp only [toRat_ofIntWithPrec_eq_mul_two_pow]
0 commit comments