Skip to content

Commit 2b1f0ce

Browse files
committed
Stash
1 parent 7567f7d commit 2b1f0ce

File tree

1 file changed

+1
-2
lines changed
  • src/Lean/Elab/Tactic/BVDecide/Frontend/Normalize

1 file changed

+1
-2
lines changed

src/Lean/Elab/Tactic/BVDecide/Frontend/Normalize/AC.lean

Lines changed: 1 addition & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -240,7 +240,7 @@ construct and return a proof of `x = y`.
240240
241241
Uses `grind`'s CommRing theory solver internally to construct said proof. -/
242242
def 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
/--
255254
Given an expression `P lhs rhs`, where `lhs, rhs : ty` and `P : $ty → $ty → _`,
256255
canonicalize top-level applications of a recognized associative and commutative

0 commit comments

Comments
 (0)