Skip to content

Commit

Permalink
chore: bump to v4.4.0 (#26)
Browse files Browse the repository at this point in the history
* chore: bump to v4.4.0

* fixes
  • Loading branch information
kim-em authored Dec 22, 2023
1 parent 9c594e3 commit 29ff369
Show file tree
Hide file tree
Showing 7 changed files with 29 additions and 6 deletions.
6 changes: 5 additions & 1 deletion lake-manifest.json
Original file line number Diff line number Diff line change
@@ -1 +1,5 @@
{"version": 5, "packagesDir": "lake-packages", "packages": []}
{"version": 7,
"packagesDir": ".lake/packages",
"packages": [],
"name": "REPL",
"lakeDir": ".lake"}
2 changes: 1 addition & 1 deletion lean-toolchain
Original file line number Diff line number Diff line change
@@ -1 +1 @@
leanprover/lean4:v4.4.0-rc1
leanprover/lean4:v4.4.0
1 change: 1 addition & 0 deletions test/Mathlib/ReplMathlibTests.lean
Original file line number Diff line number Diff line change
@@ -0,0 +1 @@
import Mathlib
6 changes: 3 additions & 3 deletions test/Mathlib/lake-manifest.json
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@
[{"url": "https://github.com/leanprover/std4",
"type": "git",
"subDir": null,
"rev": "baf6defee1fe881ae535519c0776f37f6ef08603",
"rev": "af7f36db6e7e9e395710a70635f915e8e3a0e69b",
"name": "std",
"manifestFile": "lake-manifest.json",
"inputRev": "main",
Expand All @@ -22,7 +22,7 @@
{"url": "https://github.com/leanprover-community/aesop",
"type": "git",
"subDir": null,
"rev": "3141402ba5a5f0372d2378fd75a481bc79a74ecf",
"rev": "646be3a3604d0f2a3c1800cb4279a36493474b18",
"name": "aesop",
"manifestFile": "lake-manifest.json",
"inputRev": "master",
Expand All @@ -49,7 +49,7 @@
{"url": "https://github.com/leanprover-community/mathlib4",
"type": "git",
"subDir": null,
"rev": "561ab0981d6df710afb3d34423378152195e3440",
"rev": "cf8e23a62939ed7cc530fbb68e83539730f32f86",
"name": "mathlib",
"manifestFile": "lake-manifest.json",
"inputRev": "master",
Expand Down
2 changes: 2 additions & 0 deletions test/Mathlib/lakefile.lean
Original file line number Diff line number Diff line change
Expand Up @@ -5,5 +5,7 @@ package «repl-mathlib-tests» where
-- add package configuration options here
require mathlib from git "https://github.com/leanprover-community/mathlib4" @ "master"

@[default_target]
lean_lib «ReplMathlibTests» where
globs := #[.submodules `test]
-- add library configuration options here
2 changes: 1 addition & 1 deletion test/Mathlib/lean-toolchain
Original file line number Diff line number Diff line change
@@ -1 +1 @@
leanprover/lean4:v4.4.0-rc1
leanprover/lean4:v4.4.0
16 changes: 16 additions & 0 deletions test/Mathlib/test/H20231214.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,6 +3,22 @@ open Real
open Nat
open BigOperators

/--
error: type mismatch
h₀ x
has type
p x = 2 - x ^ 2 : Prop
but is expected to have type
p x = 6 / x * p x : Prop
---
error: unsolved goals
p q : ℝ → ℝ
h₀ : ∀ (x : ℝ), p x = 2 - x ^ 2
h₁ : ∀ (x : ℝ), x ≠ 0 → q x = 6 / x
hQ : ∀ (x : ℝ), p x = 6 / x
⊢ p (q 2) = -7
-/
#guard_msgs in
theorem mathd_algebra_35
(p q : ℝ → ℝ)
(h₀ : ∀ x, p x = 2 - x^2)
Expand Down

0 comments on commit 29ff369

Please sign in to comment.