File tree Expand file tree Collapse file tree 1 file changed +1
-2
lines changed
src/Lean/Elab/Tactic/BVDecide/Frontend/Normalize Expand file tree Collapse file tree 1 file changed +1
-2
lines changed Original file line number Diff line number Diff line change @@ -240,7 +240,7 @@ construct and return a proof of `x = y`.
240240
241241Uses `grind`'s CommRing theory solver internally to construct said proof. -/
242242def proveEqualityByGrindCommRing (x y : Expr) : MetaM Expr := do
243- trace[Meta.Tactic.bv] m!"Proving equality by AC : {indentD x} = {indentD y}"
243+ trace[Meta.Tactic.bv] m!"Proving equality by grind : {indentD x} = {indentD y}"
244244 let expectedType ← mkEq x y
245245 let mvar ← mkFreshExprMVar expectedType
246246 let config := {}
@@ -250,7 +250,6 @@ def proveEqualityByGrindCommRing (x y : Expr) : MetaM Expr := do
250250 else
251251 instantiateMVars mvar
252252
253-
254253/--
255254Given an expression `P lhs rhs`, where `lhs, rhs : ty` and `P : $ty → $ty → _`,
256255canonicalize top-level applications of a recognized associative and commutative
You can’t perform that action at this time.
0 commit comments