Skip to content

Commit

Permalink
chore: remove TODO
Browse files Browse the repository at this point in the history
  • Loading branch information
leodemoura committed Jan 13, 2025
1 parent ca1790c commit 339d12f
Showing 1 changed file with 1 addition and 2 deletions.
3 changes: 1 addition & 2 deletions src/Lean/Meta/Tactic/Grind/Arith/Offset.lean
Original file line number Diff line number Diff line change
Expand Up @@ -213,8 +213,7 @@ def internalizeCnstr (e : Expr) : GoalM Unit := do
return ()
if let some k ← getDist? v u then
if (← propagateFalse v u k c e) then
-- TODO: constraint was assigned `False`, we don't need to register it
pure ()
return ()
trace[grind.offset.internalize] "{e} ↦ {c}"
modify' fun s => { s with
cnstrs := s.cnstrs.insert { expr := e } c
Expand Down

0 comments on commit 339d12f

Please sign in to comment.