mathlib4 icon indicating copy to clipboard operation
mathlib4 copied to clipboard

feat: port `itauto` from lean 3

Open digama0 opened this issue 1 year ago • 0 comments

This tactic solves problems in intuitionistic propositional logic. It also produces nice proofs when doing so, so it is useful even for proving classical theorems (using the itauto! variant to enable EM) and observing the results with #explode.

example (p : Prop) : ¬(p ↔ ¬p) := by itauto

Open in Gitpod

digama0 avatar Jan 02 '24 05:01 digama0