Skip to content

Commit

Permalink
merge
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em committed Aug 9, 2024
2 parents 7f481b2 + 71f5442 commit 61cc015
Showing 1 changed file with 6 additions and 1 deletion.
7 changes: 6 additions & 1 deletion examples/hoMatching.lean
Original file line number Diff line number Diff line change
@@ -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)

0 comments on commit 61cc015

Please sign in to comment.