Releases: leanprover/lean4-nightly
Releases · leanprover/lean4-nightly
nightly-2024-12-20
Changes since nightly-2024-12-19:
Full commit log
- 9a53c88 chore: temporarily disable Web Assembly build in CI (#6424)
- e06673e feat: lemmas about List/Array/Vector lexicographic order (#6423)
- 7b0b190 feat: lake: local package overrides (#6411)
- 759da5d fix: lake:
afterBuildCache*
traces (#6422) - 9fca337 fix: multiple bugs in
grind
(#6419) - 12cadda fix: process delayed assignment metavariables correctly in
Lean.Meta.Closure
(#6414) - b4ff545 feat: lemmas about lexicographic order on Array and Vector (#6399)
- 5dd3536 chore: protect Nat.div_eq_iff (#6417)
nightly-2024-12-19
nightly-2024-12-18
nightly-2024-12-17
Changes since nightly-2024-12-16:
Full commit log
- 64d3e9a chore: in
#print
for structures, mention 'field notation' (#6406) - 1880c61 feat: support erasure of Decidable.decide in new code generator (#6405)
- 5fcd42d chore: remove old language manual (#6401)
- 1b15a0f fix: add missing fields in the profiler datastructures (#6363)
- 0340f90 fix:
check
must check projections (#6398)
nightly-2024-12-16
Changes since nightly-2024-12-15:
Full commit log
- 791bea0 feat: lemmas about Std.Range (#6396)
- 5c2ef51 chore: add gitpod configuration (#6382)
- a8656c5 feat: generalize
panic
toSort
(#6333) - a8dc619 doc: split the docstring of
LocalContext
(#6340) - 80fb404 chore: require
0 < Range.step
(#6391) - 474adc8 feat: redefine Range.forIn' (#6390)
- 6893913 feat: replace
List.lt
withList.Lex
(#6379)
nightly-2024-12-15
Changes since nightly-2024-12-14:
Full commit log
- a8a160b fix:
revertAll
must clear auxiliary declarations (#6386) - e08d35c fix: type incorrect term produced by
contradiction
(#6387) - 94641e8 fix:
simp_all?
local declarations (#6385) - b721c0f test: add test for issue #4585 (#6384)
- f790b19 fix: new code generator must generate code for opaque declarations that are not
@[extern]
(#6383) - 6571bc0 fix:
withTrackingZetaDelta
must reset cache (#6381) - 37122c3 chore: move implementation details of
mergeSort
into namespace (#6380)
nightly-2024-12-14
Changes since nightly-2024-12-13:
Full commit log
- 280fcc9 feat:
lean --error=kind
(#6362) - 19eac5f fix: propagate
Simp.Config
when reducing terms and checking definitional equality insimp
(#6123) - aa00725 chore: stop running compiler twice during tests (#6321)
- 7530fd6 chore: remove Lean.Compiler.LCNF.ForEachExpr (#6313)
- 58ffd15 doc: fix typo reference in doc of lazy discrimination tree (#6377)
nightly-2024-12-13
nightly-2024-12-12
nightly-2024-12-11
Changes since nightly-2024-12-10:
Full commit log
- 8709ca3 chore: DecidableRel allows a heterogeneous relation (#6341)
- 19fb1fb feat: do not propagate pretty printer errors through messages (#3696)
- cb31ddc feat: lemmas about indexing and membership for Vector (#6367)
- 633c825 feat: add
Float32
support (#6366) - c83ce02 feat: alignment of Array.set lemmas with List lemmas (#6365)
- cd909b0 fix: when pretty printing constant names, do not use aliases from "non-API
export
s" (#5689) - d27c5af refactor: ArgsPacker.unpack to return
Option
(#6359) - 9386511 refactor: elabWFRel to take names, not
PreDefinition
(#6358) - a9b6a9a refactor: WF.EqnInfo.hasInduct (#6357)
- d5b565e refactor: make
mkInhabitantFor
error message configurable (#6356) - 27c2323 chore: alignment of Array.any/all lemmas with List (#6353)
- 1786539 feat: BitVec.[toInt|toFin|getMsbD]_ofBool (#6317)
- a805946 chore: adjust CODEOWNERS (#6327)