Files
NNG/Game/Tactic/Ne.lean
2023-10-28 22:01:03 +02:00

16 lines
478 B
Lean4

import Lean
/-!
A pretty-printer that displays `¬ (a = b)` as `a ≠ b`.
-/
open Lean PrettyPrinter Delaborator SubExpr
@[delab app.Not] def delab_not_mem :=
whenPPOption Lean.getPPNotation do
let #[f] := ( SubExpr.getExpr).getAppArgs | failure
unless f.getAppFn matches .const `Eq _ do failure
let stx₁ SubExpr.withAppArg <| SubExpr.withNaryArg 1 delab
let stx₂ SubExpr.withAppArg <| SubExpr.withNaryArg 2 delab
return `($stx₁ $stx₂)