Skip to content

Commit

Permalink
fix bad comments
Browse files Browse the repository at this point in the history
  • Loading branch information
eric-wieser committed Dec 5, 2024
1 parent 7da5ecf commit d6671db
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions Mathlib/Data/Rat/Floor.lean
Original file line number Diff line number Diff line change
Expand Up @@ -142,7 +142,7 @@ def evalIntFloor : NormNumExt where eval {u αZ} e := do
let _i ← synthInstanceQ q(LinearOrderedField $α)
assertInstancesCommute
have z : Q(ℤ) := mkRawIntLit ⌊q⌋
letI : $z =Q $n / $d := ⟨⟩
letI : $z =Q $n / $d := ⟨⟩
return .isInt q(inferInstance) z ⌊q⌋ q(isInt_intFloor_ofIsRat _ $n $d $h)
| _, _, _ => failure

Expand Down Expand Up @@ -172,7 +172,7 @@ def evalIntCeil : NormNumExt where eval {u αZ} e := do
return .isNat q(inferInstance) _ q(isNat_intCeil $x _ $pb)
| .isNegNat _ _ pb => do
assertInstancesCommute
-- floor always keeps naturals negative, so we can shortcut `.isInt`
-- ceil always keeps naturals negative, so we can shortcut `.isInt`
return .isNegNat q(inferInstance) _ q(isInt_intCeil _ _ $pb)
| .isRat _ q n d h => do
let _i ← synthInstanceQ q(LinearOrderedField $α)
Expand Down

0 comments on commit d6671db

Please sign in to comment.