Skip to content

Commit

Permalink
Bump to Lean v4.10.0
Browse files Browse the repository at this point in the history
One of the new core linters crashes on this test, so for now we disable it.
Since we're touching the test anyway, let's improve the output checking.
  • Loading branch information
eric-wieser committed Aug 9, 2024
1 parent 01ad339 commit 8e20e08
Show file tree
Hide file tree
Showing 2 changed files with 7 additions and 2 deletions.
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)
2 changes: 1 addition & 1 deletion lean-toolchain
Original file line number Diff line number Diff line change
@@ -1 +1 @@
leanprover/lean4:v4.9.0-rc1
leanprover/lean4:v4.10.0

0 comments on commit 8e20e08

Please sign in to comment.