Releases: leanprover/lean4-nightly
Releases · leanprover/lean4-nightly
nightly-2024-10-16
Changes since nightly-2024-10-15:
Full commit log
- a04b476 chore: remove instBEqNat, which is redundant with instBEqOfDecidableEq but not defeq (#5694)
- eea953b feat: push/pop tactic API (#5720)
- dec1262 chore: upstream
classical
tactic (#5730) - 487c2a9 feat: Expr helper functions (#5729)
- 831fa08 chore: upstream String.dropPrefix? (#5728)
- 94053c9 chore: make getIntrosize public (#5727)
- 94b1e51 fix: simpproc to reduce Fin literals consistently (#5632)
- 5a87b10 refactor: remove mkRecursorInfoForKernelRec (#5681)
- dc83a60 fix: List.drop_drop addition order (#5716)
- 7234ab7 feat: add BitVec.sdiv_[zero|one|self] theorems (#5718)
- c27e671 chore: rename
instDecidableEqQuotientOfDecidableEquiv
toQuotient.decidableEq
(#5722) - 94dd1d6 feat: bv_decide inequality regression tests (#5714)
- 4409e39 chore: upstream List.sum, planning to later deprecate Nat.sum (#5703)
nightly-2024-10-15
Changes since nightly-2024-10-14:
Full commit log
- 0bfe1a8 chore: better default value for Array.swapAt! (#5705)
- a026bc7 feat: let dot notation see through
CoeFun
instances (#5692) - 36c2511 feat: options
pp.mvars.anonymous
andpp.mvars.levels
(#5711) - adfbc56 chore: disable ac_nf by default (#5673)
- 9f8ce47 feat: add BitVec.[udiv|umod]_[zero|one|self] theorems (#5712)
- 3d175ab fix: the
⋯
elaboration warning did not mentionpp.maxSteps
(#5710) - 9b6696b feat: use libuv for tempfiles (#5135)
- 057482e feat: denote deprecations in completion items (#5707)
- 16e2a78 chore: remove @[simp] from Option.isSome_eq_isSome (#5704)
- 2580694 chore: mark prefix_append_right_inj as simp lemma (#5706)
- 9ec29b4 chore: update stage0
- aa2360a chore: rename List.join to List.flatten
- 65637b7 feat: lemmas about BitVector arithmetic inequalities (#5646)
- 20ea855 feat: upstream List.mapIdx, and add lemmas (#5696)
nightly-2024-10-14
Changes since nightly-2024-10-13:
Full commit log
nightly-2024-10-13
nightly-2024-10-12
Changes since nightly-2024-10-11:
Full commit log
- a3bc4d2 fix: make IO-bound tasks dedicated (#5678)
- 087219b feat: make bv_decide error when the LRAT proof is invalid (#5676)
- e5bbda1 fix: context tracking in bv_decide counter example (#5675)
- 742ca6a feat: support
let rec
in#eval
(#5663) - fe0fbc6 feat:
decide!
tactic for using kernel reduction (#5665)
nightly-2024-10-11
Changes since nightly-2024-10-10:
Full commit log
nightly-2024-10-10
nightly-2024-10-09
Changes since nightly-2024-10-08:
Full commit log
- b814be6 fix: use
MessageData.tagged
to mark maxHeartbeat exceptions (#5566) - feb8185 fix: upgrade instance synth order issues to hard errors (#5399)
- 7942b9e fix: lake: make package
extraDep
intransitive (#5641) - 15bb8a2 fix: have
simpa ... using ...
doexact
-like checks (#5648) - a35e6f4 feat: infer
Prop
forinductive
/structure
when defining syntactic subsingletons (#5517) - fdd5aec feat: better
#eval
command (#5627) - 81743d8 chore: reduce error on bv_check to warning (#5655)
- 248864c perf: benchmark for modulo on bv_decide (#5653)
- bd46319 feat: add option
pp.mvars.delayed
(#5643) - 6cdede3 fix: make sure name literals use escaping when pretty printing (#5639)
- f1d3527 fix: have
Lean.Meta.ppGoal
use hard newlines (#5640) - b2b450d fix: now linters in general do not run on
#guard_msgs
itself (#5644) - abae95e feat: support umod in bv_decide (#5652)
- e9ea99f feat: support udiv in bv_decide (#5628)
- 2ed7924 chore: define udiv normal form to be /, resp. umod and % (#5645)
- 4415a81 chore: add Siddharth to authors list of BitVec (#5647)
nightly-2024-10-08
Changes since nightly-2024-10-07:
Full commit log
- 3e75d8f fix: FunInd: avoid over-eta-expanding in preprocessing step (#5619)
- f1ff9ce feat: more getLsbD bitblaster theory (#5637)
- 99a9d9b doc: remarks about multiplication (#5636)
- 1914a2b feat: add auxiliary bitblasters for negation and subtraction (#5635)
- 6312787 feat: lemmas for Bitvector division when denominator is zero (#5609)
- ec5f206 fix: shutdown deadlock and crash desync (#5340)
- d835616 chore: fix MSYS2 build instructions (#5617)
nightly-2024-10-07
Changes since nightly-2024-10-03:
Full commit log
- 9dac514 feat: Document Bitblasting in a documentation comment (#5620)
- c0617da feat: support
at
inac_nf
and use it inbv_normalize
(#5618) - a3ee111 chore: update stage0
- 13e3a38 fix: Lake: brittle dependency on env ext name
- 0178f2b chore: update stage0
- 4f5f392 chore: update stage0
- d4fdb5d fix: getFunInfo, inferType to use withAtLeastTransparency, not withTransparency (#5563)
- f9048c1 chore: add bv_toNat tag for toNat_ofInt (#5608)
- 53c5470 perf: remove List.redLength (#5605)
- 3584a62 fix: call hierarchy into
(builtin_)initialize
(#5560)