leanprover-community / aesop

White-box automation for Lean 4
Apache License 2.0
157 stars 25 forks source link

Builtin rules loop on simple goal with negation #54

Open JLimperg opened 1 year ago

JLimperg commented 1 year ago
import Aesop
theorem P Q : ¬ P → ¬ Q → False := by
  aesop

The loop happens because applyHyps transforms not P, not Q |- False into not P, not Q |- P and simp transforms this back into not P, not Q |- False.