Skip to content

Commit

Permalink
Attempt tweaking defeq heuristic
Browse files Browse the repository at this point in the history
  • Loading branch information
Command-Master committed Dec 8, 2024
1 parent 6e60d13 commit 937190f
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion src/Lean/Meta/ExprDefEq.lean
Original file line number Diff line number Diff line change
Expand Up @@ -1364,7 +1364,7 @@ private def unfoldBothDefEq (fn : Name) (t s : Expr) : MetaM LBool := do
unfold s (pure .undef) fun s =>
isDefEqLeftRight fn t s
| .app _ _, .app _ _ =>
if (← tryHeuristic t s) then
if (← getProjectionFnInfo? fn).isNone && (← tryHeuristic t s) then
return .true
else
unfold t
Expand Down

0 comments on commit 937190f

Please sign in to comment.