Skip to content

Releases: leanprover/lean4

v4.25.2

25 Nov 14:40

Choose a tag to compare

chore: set(LEAN_VERSION_PATCH 2)

v4.25.1

25 Nov 12:52

Choose a tag to compare

chore: set(LEAN_VERSION_PATCH 1)

v4.24.1

25 Nov 12:16

Choose a tag to compare

chore: set(LEAN_VERSION_PATCH 1)

v4.26.0-rc2

21 Nov 02:01

Choose a tag to compare

v4.26.0-rc2 Pre-release
Pre-release
fix: bug `ite`/`dite` propagator used in `grind` (#11295)

This PR fixes a bug in the propagation rules for `ite` and `dite` used
in `grind`. The bug prevented equalities from being propagated to the
satellite solvers. Here is an example affected by this issue.

```lean
example
    [LE Ξ±] [LT Ξ±] [Std.IsLinearOrder Ξ±] [Std.LawfulOrderLT Ξ±]
    [Lean.Grind.CommRing Ξ±] [DecidableLE Ξ±] [Lean.Grind.OrderedRing Ξ±]
    (a b c : Ξ±) :
  (if a - b ≀ -(a - b) then -(a - b) else a - b) ≀
  ((if a - c ≀ -(a - c) then -(a - c) else a - c) + if c - d ≀ -(c - d) then -(c - d) else c - d) +
    if b - d ≀ -(b - d) then -(b - d) else b - d := by
  grind
```

v4.26.0-rc1

18 Nov 03:13

Choose a tag to compare

v4.26.0-rc1 Pre-release
Pre-release
chore: set LEAN_VERSION_IS_RELEASE

v4.25.0

14 Nov 06:02

Choose a tag to compare

fix: Meta.Closure: topologically sort abstracted vars (#10926)

This PR topologically sorts abstracted vars in
`Meta.Closure.mkValueTypeClosure` if MVars are being abstracted.
Fixes #10705

---------

Co-authored-by: Eric Wieser <[email protected]>
(cherry picked from commit a6d50a61b35b73576f5c4ceac08789d9517f3079)

v4.25.0-rc2

22 Oct 00:48

Choose a tag to compare

v4.25.0-rc2 Pre-release
Pre-release
chore: release_steps runs lake exe cache get when needed