Skip to content

Commit e9e777f

Browse files
committed
chore: mark TODO
1 parent 5fc1226 commit e9e777f

File tree

1 file changed

+3
-1
lines changed

1 file changed

+3
-1
lines changed

src/Lean/Meta/Tactic/Grind/Arith/CommRing/Internalize.lean

Lines changed: 3 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -94,7 +94,9 @@ private def processDiv (e inst a b : Expr) : RingM Unit := do
9494
pushNewFact <| mkExpectedPropHint
9595
(mkApp7 (mkConst ``Grind.CommRing.div_int_eqC [ring.u]) ring.type (mkNatLit c) fieldInst charInst a (mkIntLit k) reflBoolTrue)
9696
expected
97-
return ()
97+
else
98+
-- TODO
99+
return ()
98100

99101
/--
100102
Returns `true` if `e` is a term `a/b` or `a⁻¹`.

0 commit comments

Comments
 (0)