Skip to content

Commit

Permalink
chore: use hasNoConfusionDecl in grind
Browse files Browse the repository at this point in the history
  • Loading branch information
jrr6 committed Jan 21, 2025
1 parent 57e7693 commit 6fcce8f
Showing 1 changed file with 1 addition and 2 deletions.
3 changes: 1 addition & 2 deletions src/Lean/Meta/Tactic/Grind/Ctor.lean
Original file line number Diff line number Diff line change
Expand Up @@ -46,8 +46,7 @@ def propagateCtor (a b : Expr) : GoalM Unit := do
propagateInjEqs (← inferType injLemma) injLemma
else
let .const declName _ := aType.getAppFn | return ()
let noConfusionDeclName := Name.mkStr declName "noConfusion"
unless (← getEnv).contains noConfusionDeclName do return ()
unless (← hasNoConfusionDecl declName) do return ()
closeGoal (← mkNoConfusion (← getFalseExpr) (← mkEqProof a b))

end Lean.Meta.Grind

0 comments on commit 6fcce8f

Please sign in to comment.