diff --git a/examples/hoMatching.lean b/examples/hoMatching.lean index db8faf2..871b39c 100644 --- a/examples/hoMatching.lean +++ b/examples/hoMatching.lean @@ -1,8 +1,13 @@ import Qq open Qq Lean +-- TODO: this linter crashes on the `def` below +set_option linter.constructorNameAsVariable false in def turnExistsIntoForall : Q(Prop) → MetaM Q(Prop) | ~q(∃ x y, $p x y) => return q(∀ x y, $p x y) | e => return e -#eval turnExistsIntoForall q(∃ a b, String.length a ≤ b + 42) +/-- info: ∀ (x : String) (y : Nat), x.length ≤ y + 42 -/ +#guard_msgs in +run_cmd Elab.Command.liftTermElabM do + Lean.logInfo <| ← turnExistsIntoForall q(∃ a b, String.length a ≤ b + 42)