Skip to content

Releases: leanprover/lean4-nightly

nightly-2024-11-20

20 Nov 12:41
7fbe8e3
Compare
Choose a tag to compare
nightly-2024-11-20 Pre-release
Pre-release

Changes since nightly-2024-11-19:

Full commit log

  • 7fbe8e3 fix: Inhabited Float produced a bogus run-time value (#6136)
  • 2fbc466 fix: trace.profiler pretty-printing (#6138)
  • 17419ac feat: thread support for trace.profiler.output (#6137)
  • f85c667 feat: Array.insertIdx/eraseIdx take a tactic-provided proof (#6133)
  • c8b4f6b feat: duplicate List.attach/attachWith/pmap API for Array (#6132)
  • 3c75551 feat: add BitVec.(msb, getMsbD)_(rotateLeft, rotateRight) (#6120)
  • 5eef3d2 feat: have #print show precise fields of structures (#6096)
  • 75d1504 fix: isDefEq for constants with different universe parameters (#6131)
  • a00cf63 fix: add a missing case to Level.geq (#2689)
  • 1f32477 fix: isDefEq when zetaDelta := false (#6129)
  • 91c14c7 fix: only consider salient bytes in sharecommon eq, hash (#5840)
  • 69530af chore: update stage0
  • b7667c1 fix: don't issue atomic id completions when there is a dangling dot (#5837)
  • d6f8980 chore: generalize List.get_mem (#6095)
  • a385666 test: fix brittle structure instance completion test (#6127)
  • 4bef358 chore: update stage0
  • 64538cf chore: prepare for bootstrap
  • aadf3f1 feat: use new structInstFields parser to tag structure instance fields
  • 95bf45f refactor: split Completion.lean
  • 2a02c12 feat: structure auto-completion & partial InfoTrees

nightly-2024-11-19

19 Nov 08:31
4600bb1
Compare
Choose a tag to compare
nightly-2024-11-19 Pre-release
Pre-release

Changes since nightly-2024-11-18:

Full commit log

  • 4600bb1 feat: use BaseIO at IO.rand (#6102)
  • 7ccdfc3 chore: turn off pp.mvars in apply? results (#6108)
  • 7f0bdef chore: fix apply? error reporting when out of heartbeats (#6121)
  • 799b2b6 fix: handle reordered indices in structural recursion (#6116)
  • b8d6e44 fix: liberalize rules for atoms by allowing leading '' (#6114)

nightly-2024-11-18

18 Nov 08:31
5a99cb3
Compare
Choose a tag to compare
nightly-2024-11-18 Pre-release
Pre-release

Changes since nightly-2024-11-15:

Full commit log

  • 5a99cb3 chore: make Lean.Elab.Command.mkMetaContext public (#6113)
  • e10fac9 feat: lemmas for Array.findSome? and find? (#6111)
  • 62ae320 chore: document Lean.Elab.StructInst, refactor (#6110)
  • 98b1edf fix: backtrack at injection failure (#6109)
  • ab162b3 fix: isDefEq, whnf, simp caching and configuration (#6053)
  • b8a13ab chore: fix naming of left/right injectivity lemmas (#6106)
  • 405593e chore: avoid stack overflow in debug tests (#6103)
  • 24f305c chore: fix canonicalizer handling over forall/lambda (#6082)
  • 5d553d6 fix: circular assignment at structure instance elaborator (#6105)
  • a449e3f feat: IO.getTID (#6049)
  • 7643867 fix: improvements to change tactic (#6022)
  • 7f1d7a5 fix: use Expr.equal instead of == in MVarId.replaceTargetDefEq and MVarId.replaceLocalDeclDefEq (#6098)
  • f13e5ca chore: naming convention and NaN normalization (#6097)
  • ecbaeff feat: add Float.toBits and Float.fromBits (#6094)
  • 691acde feat: pp.parens option to pretty print with all parentheses (#2934)
  • b1e0c1b chore: remove decide! tactic (#6016)
  • 93b4ec0 refactor: use mkFreshUserName in ArgsPacker (#6093)
  • f06fc30 perf: remove @[specialize] from mkBinding (#6019)
  • 64b35a8 perf: add LEAN_ALWAYS_INLINE to some functions (#6045)
  • 688ee4c fix: constant folding for Nat.ble and Nat.blt (#6087)
  • 9a3dd61 chore: bv_decide remove noop rewrites (#6080)
  • 7e6363d chore: join → flatten in docstring (#6040)

nightly-2024-11-15

15 Nov 08:27
a074bd9
Compare
Choose a tag to compare
nightly-2024-11-15 Pre-release
Pre-release

Changes since nightly-2024-11-14:

Full commit log

  • a074bd9 feat: implementation of Array.pmap (#6052)
  • 498d416 fix: pretty print .coeFun with terminfo of coercee (#6085)
  • e0d7c3a feat: add date and time functionality (#4904)
  • 6a5b122 perf: use RArray in simp_arith meta code (#6068 part 2)
  • bf9ddf2 chore: update stage0
  • 3f47871 perf: use RArray in simp_arith meta code (#6068 part 1)
  • 85f2596 feat: Lean.RArray (#6070)
  • 8e1ddbc fix: validate atoms modulo leading and trailing whitespace (#6012)
  • e6e39f5 feat: add options to configure all of bv_decide's preprocessing (#6077)
  • debb82b perf: make andFlattening work on deeply nested hyps in one pass (#6075)

nightly-2024-11-14

14 Nov 08:24
9a85433
Compare
Choose a tag to compare
nightly-2024-11-14 Pre-release
Pre-release

Changes since nightly-2024-11-13:

Full commit log

  • 9a85433 refactor: allow Sort u in Squash (#6074)
  • 4616c0a refactor: lake: avoid v! in builtin code (#6073)
  • e55b681 feat: add Context.setConfig (#6072)
  • 6313210 feat: lemmas about for loops over Array (#6055)
  • 350b364 chore: upstream some NameMap functions (#6056)
  • 1c30c76 chore: remove >6 month old deprecations (#6057)
  • d5adadc chore: add newline at end of file for lake new templates (#6026)
  • f08805e feat: message kinds (#5945)
  • 256b49b perf: optimize Nat.Linear.Poly.norm (#6064)
  • 28cf146 fix: make sure monad lift coercion elaborator has no side effects (#6024)
  • 970261b perf: optimize Nat.Linear.Expr.toPoly (#6062)
  • 6b811f8 test: synthetic simp_arith benchmark (#6061)
  • f721f94 feat: Bool.to(U)IntX (#6060)
  • 86524d5 fix: line break in simp? output (#6048)
  • f18d9e0 refactor: omega: avoid MVar machinery (#5991)
  • fa33423 chore: pr-body: run as part of merge_group, but do not do anything (#6069)

nightly-2024-11-13

13 Nov 08:25
Compare
Choose a tag to compare
nightly-2024-11-13 Pre-release
Pre-release

Changes since nightly-2024-11-12:

Full commit log

  • 1315266 refactor: mark the Simp.Context constructor as private
  • b1e52f1 chore: mark Meta.Context.config as private (#6051)
  • 985600f chore: update stage0
  • ace6248 chore: deprecate Array.sequenceMap
  • 9f42368 chore: update stage0
  • a401368 feat: various minor changes to List/Array API (#6044)

nightly-2024-11-12

12 Nov 08:23
5e01e62
Compare
Choose a tag to compare
nightly-2024-11-12 Pre-release
Pre-release

Changes since nightly-2024-11-11:

Full commit log

  • 5e01e62 chore: review Array operations argument order (#6041)
  • 3a408e0 feat: change Array.get to take a Nat and a proof (#6032)
  • 675d2d5 feat: only direct parents of classes create projections (#5920)
  • 281c07c fix: bv_decide embedded constraint substitution changes models (#6037)
  • 004430b fix: avoid new term info around def bodies (#6031)
  • 61f7dcb feat: bv_decide and flattening (#6035)
  • 5c611f7 fix: simp only [· ∈ ·] (#6030)
  • 722cb73 feat: BitVec normalization rule for udiv by twoPow (#6029)
  • 258d372 feat: change Array.set to take a Nat and a tactic provided bound (#5988)

nightly-2024-11-11

11 Nov 08:27
456e6d2
Compare
Choose a tag to compare
nightly-2024-11-11 Pre-release
Pre-release

Changes since nightly-2024-11-10:

Full commit log

  • 456e6d2 chore: deprecate duplicated Fin.size_pos (#6025)
  • 48e3d76 feat: variants of List.forIn_eq_foldlM (#6023)
  • 78fe925 feat: BitVec lemmas for smtUDiv, smtSDiv when denominator is zero (#5616)

nightly-2024-11-10

10 Nov 08:25
811d8fb
Compare
Choose a tag to compare
nightly-2024-11-10 Pre-release
Pre-release

Changes since nightly-2024-11-09:

Full commit log

nightly-2024-11-09

09 Nov 13:05
f55a9a7
Compare
Choose a tag to compare
nightly-2024-11-09 Pre-release
Pre-release

Changes since nightly-2024-11-08:

Full commit log

  • f55a9a7 chore: CI: do not run check-pr-body in merge group
  • d12df6c fix: bv_decide benchmarks (#6017)
  • d1a99d8 fix: avoid delaborating with field notation if object is a metavariable (#6014)
  • c10e4c2 feat: prop instance yields theorems (#5856)
  • e3420c0 feat: decide +revert and improvements to native_decide (#5999)
  • 4f7aa8c chore: CI: exempt drafts from PR body check (#6002)
  • dac73c1 perf: avoid negative environment lookup (#5429)
  • cb40dda fix: avoid max heartbeat error in completion (#5996)
  • fc0529b fix: ensure instantiateMVarsProfiling adds a trace node (#5501)
  • 837a67b feat: change bv_decide to an elaborated config (#6010)
  • 85f2213 fix: unset trailing for simpa? "try this" suggestion (#5907)
  • 9b167e2 feat: verify keys method on HashMaps (#5866)
  • 1870c00 chore: missing @[ext] attribute on monad transformer ext lemmas (#6008)