Skip to content

Commit df47d57

Browse files
kim-emleanprover-community-mathlib4-botgithub-actionsjcommelinmathlib4-bot
authored
chore: adaptations for nightly-2025-06-30 (#8)
* cleanup grind tests * chore: bump to nightly-2025-06-12 * merge lean-pr-testing-8419 * chore: bump to nightly-2025-06-12 * merge lean-pr-testing-8653 * adaptation note * oops * chore: adaptations for nightly-2025-06-12 * remove nolint simpNF * remove spurious file * Update lean-toolchain for testing leanprover/lean4#8751 * fix * chore: bump to nightly-2025-06-13 * Merge master into nightly-testing * fix * remove upstreamed * drop no-op `show` * chore: bump to nightly-2025-06-14 * chore: bump to nightly-2025-06-15 * intentionally left blank * fix tests * chore: bump to nightly-2025-06-16 * fix upstream * fix * fix * fixes * chore: adaptations for nightly-2025-06-16 * chore: bump to nightly-2025-06-17 * fixes * more fixes * fixes! * more fixes! * hmm * chore: adaptations for nightly-2025-06-17 * chore: adaptations for nightly-2025-06-17 * chore: lint `show` (adaptation for leanprover/lean4#7395) (leanprover-community#25749) Adds `show` as an exception to the unused tactic linter and adds a separate linter for `show`s that should be replaced by `change`. Context: https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/unused.20tactic.20linter.20for.20.60show.60/with/523701633 Co-authored-by: Christian Merten <[email protected]> Co-authored-by: Kenny Lau <[email protected]> Co-authored-by: Fabrizio Barroero <[email protected]> Co-authored-by: Rob23oba <[email protected]> Co-authored-by: leanprover-community-mathlib4-bot <[email protected]> Co-authored-by: Rob23oba <[email protected]> Co-authored-by: Kim Morrison <[email protected]> * Update lean-toolchain for testing leanprover/lean4#8577 * chore: bump to nightly-2025-06-18 * chore: adaptations for nightly-2025-06-18 * Merge master into nightly-testing * Update lean-toolchain for testing leanprover/lean4#8804 * Update lean-toolchain for testing leanprover/lean4#8699 * bump Qq and batteries * meta adaptations * bump aesop * fix * fix (adaptation note) * Update lean-toolchain for leanprover/lean4#8699 * shake * chore: bump to nightly-2025-06-19 * fix * Update lean-toolchain for leanprover/lean4#8699 * fix: correct memoFix's use of unsafe code * fix: adjust noncomputable annotations for new compiler * fix: replace use of `open private _ in` with `open private _ from` The implementation of `open private _ from` relies on specific internals of the old compiler and will no longer work. * remove mul_hmul * chore: adjust one maxHeartbeats for the new compiler * linter * chore: bump to nightly-2025-06-20 * chore: adaptations for nightly-2025-06-20 * Update lean-toolchain for testing leanprover/lean4#8914 * chore: bump to nightly-2025-06-21 * fix * fixes * fixes * fixes * updated lake manifest * comment out tests * chore: fix for nightly-testing (leanprover-community#26246) * fix * fix * fix grind typeclasses * chore: adaptations for nightly-2025-06-20 * lake update * Update lean-toolchain for leanprover/lean4#8914 * fix grind instance * chore: bump to nightly-2025-06-22 * chore: bump to nightly-2025-06-23 * chore: rm unused `Lean.Util.Paths` import & use updated batteries * Ensure we checkout mathlib4 master, not nightly-testing master (which does not exist) * merge lean-pr-testing-8804 * Bump dependencies and silence linter. * Fixes (Now `elabSimpArgs` already handles `*`, so we can delete the associated code.) * lake update; disable unusedSimpArgs in Batteries * lkae update aesop * disable unusedSimpArgs in MathlibTest * fix grind instance priorities * comment out MathlibTest/zmod with adaptation note * touch for CI * chore: bump to nightly-2025-06-24 * Kick CI * Bump batteries * Guessing adaption for leanprover/lean4#8929 * chore: bump to nightly-2025-06-25 * fix: workflow merging master into nightly-testing * fix * chore: cache get uses tracking remote * touch for new CI * restart CI * chore: bump to nightly-2025-06-26 * Update lean-toolchain for testing leanprover/lean4#8928 * Teach Mathlib about `mrefine` * Merge master into nightly-testing * Update lean-toolchain for testing leanprover/lean4#8980 * chore: update linter warning test outputs * chore: remove excess line break in deprecation lint now that notes add their own line breaks * chore: more test cleanup * . * cleanup adaptation notes * fix * fix * chore: bump to nightly-2025-06-27 * Merge master into nightly-testing * Merge master into nightly-testing * re-enable unusedSimpArgs * re-enable unusedSimpArgs * re-enable unusedSimpArgs * re-enable unusedSimpArgs * re-enable unusedSimpArgs * fix tests * chore: bump to nightly-2025-06-28 * Merge master into nightly-testing * lintining * Merge master into nightly-testing * unused simp args * chore: bump to nightly-2025-06-29 * chore: adaptations for nightly-2025-06-29 * Merge master into nightly-testing * chore: robustify `open Mathlib` benchmark * deprecations * Update lean-toolchain for testing leanprover/lean4#9086 * Merge master into nightly-testing * fixes * chore: bump to nightly-2025-06-30 * lake update * lake update * lake update * lake update * lake update * . --------- Co-authored-by: leanprover-community-mathlib4-bot <[email protected]> Co-authored-by: github-actions <[email protected]> Co-authored-by: Johan Commelin <[email protected]> Co-authored-by: mathlib4-bot <[email protected]> Co-authored-by: sgouezel <[email protected]> Co-authored-by: Kyle Miller <[email protected]> Co-authored-by: Sebastian Ullrich <[email protected]> Co-authored-by: Rob23oba <[email protected]> Co-authored-by: Rob23oba <[email protected]> Co-authored-by: Christian Merten <[email protected]> Co-authored-by: Kenny Lau <[email protected]> Co-authored-by: Fabrizio Barroero <[email protected]> Co-authored-by: Rob23oba <[email protected]> Co-authored-by: Cameron Zwarich <[email protected]> Co-authored-by: Mac Malone <[email protected]> Co-authored-by: Anne C.A. Baanen <[email protected]> Co-authored-by: Joachim Breitner <[email protected]> Co-authored-by: Sebastian Graf <[email protected]> Co-authored-by: Joseph Rotella <[email protected]>
1 parent 9715c1d commit df47d57

File tree

9 files changed

+18
-21
lines changed

9 files changed

+18
-21
lines changed

Mathlib/Algebra/PresentedMonoid/Basic.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -122,7 +122,7 @@ def lift : PresentedMonoid rels →* M :=
122122
@[to_additive]
123123
theorem toMonoid.unique (g : MonoidHom (conGen rels).Quotient M)
124124
(hg : ∀ a : α, g (of rels a) = f a) : g = lift f h :=
125-
Con.lift_unique (Con.conGen_le h) g (FreeMonoid.hom_eq fun x ↦ let_fun this := hg x; this)
125+
Con.lift_unique (Con.conGen_le h) g (FreeMonoid.hom_eq hg)
126126

127127
@[to_additive (attr := simp)]
128128
theorem lift_of {x : α} : lift f h (of rels x) = f x := rfl

Mathlib/Analysis/Normed/Lp/PiLp.lean

Lines changed: 1 addition & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -818,8 +818,7 @@ protected def _root_.LinearIsometryEquiv.piLpCongrRight (e : ∀ i, α i ≃ₗ
818818
≪≫ₗ (LinearEquiv.piCongrRight fun i => (e i).toLinearEquiv)
819819
≪≫ₗ (WithLp.linearEquiv _ _ _).symm
820820
norm_map' := (WithLp.linearEquiv p 𝕜 _).symm.surjective.forall.2 fun x => by
821-
simp only [LinearEquiv.trans_apply,
822-
WithLp.linearEquiv_symm_apply, WithLp.linearEquiv_apply]
821+
simp only [LinearEquiv.trans_apply, WithLp.linearEquiv_symm_apply, WithLp.linearEquiv_apply]
823822
obtain rfl | hp := p.dichotomy
824823
· simp_rw [PiLp.norm_toLp, Pi.norm_def, LinearEquiv.piCongrRight_apply,
825824
LinearIsometryEquiv.coe_toLinearEquiv, LinearIsometryEquiv.nnnorm_map,

Mathlib/RingTheory/ZMod/UnitsCyclic.lean

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -139,7 +139,7 @@ lemma exists_one_add_mul_pow_prime_pow_eq {u v : R}
139139
(mul_dvd_mul_left _ hvu)
140140
(by
141141
rw [mul_pow]
142-
simp only [← mul_assoc, mul_comm _ p]
142+
simp only [← mul_assoc]
143143
rw [mul_assoc, mul_assoc, ← mul_assoc u, mul_comm u]
144144
apply mul_dvd_mul _ hpuv
145145
rw [← pow_two]
@@ -170,7 +170,7 @@ theorem orderOf_one_add_mul_prime_pow {p : ℕ} (hp : p.Prime) (m : ℕ) (hm0 :
170170
pow_succ, Nat.cast_mul, Int.mul_dvd_mul_iff_left (by simp [hp.ne_zero])]
171171
· obtain ⟨y, hy⟩ := this (n + 1)
172172
rw [hy, ← pow_add, ← Nat.cast_pow]
173-
simp [ZMod.natCast_self]
173+
simp
174174
· rw [← pow_succ', ← pow_succ, ← pow_mul, mul_comm]
175175
exact pow_dvd_pow _ hpm
176176

@@ -331,7 +331,7 @@ theorem isCyclic_units_iff (n : ℕ) :
331331
· rw [h2]; simp [isCyclic_units_two]
332332
by_cases h4 : n = 4
333333
· rw [h4]; simp [isCyclic_units_four]
334-
simp only [h0, h1, h2, h4, exists_and_left, false_or, and_or_left, exists_or, ← exists_and_left]
334+
simp only [h0, h1, h2, h4, false_or, and_or_left, exists_or]
335335
rcases (n.even_or_odd).symm with hn | hn
336336
· rw [isCyclic_units_iff_of_odd hn, or_iff_left]
337337
· congr! with p m

Mathlib/Tactic/Clean.lean

Lines changed: 3 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -23,15 +23,13 @@ def cleanConsts : List Name :=
2323
[``id]
2424

2525
/-- Clean an expression by eliminating identify functions listed in `cleanConsts`.
26-
Also eliminates `fun x => x` applications and tautological `let_fun` bindings. -/
26+
Also eliminates `fun x => x` applications and tautological `let`/`have` bindings. -/
2727
def clean (e : Expr) : Expr :=
2828
e.replace fun
2929
| .app (.app (.const n _) _) e' => if n ∈ cleanConsts then some e' else none
3030
| .app (.lam _ _ (.bvar 0) _) e' => some e'
31-
| e =>
32-
match e.letFun? with
33-
| some (_n, _t, v, .bvar 0) => some v
34-
| _ => none
31+
| .letE _ _ v (.bvar 0) _ => some v
32+
| _ => none
3533

3634
end Lean.Expr
3735

Mathlib/Tactic/HaveI.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -23,7 +23,7 @@ macro_rules
2323
| `(assert! haveIDummy $hd:letDecl; $body) => `(haveI $hd:letDecl; $body)
2424

2525
/--
26-
`haveI'` behaves like `have`, but inlines the value instead of producing a `let_fun` term.
26+
`haveI'` behaves like `have`, but inlines the value instead of producing a `have` term.
2727
2828
(This is the do-notation version of the term-mode `haveI`.)
2929
-/
@@ -35,7 +35,7 @@ macro_rules
3535
| `(assert! letIDummy $hd:letDecl; $body) => `(letI $hd:letDecl; $body)
3636

3737
/--
38-
`letI` behaves like `let`, but inlines the value instead of producing a `let_fun` term.
38+
`letI` behaves like `let`, but inlines the value instead of producing a `let` term.
3939
4040
(This is the do-notation version of the term-mode `haveI`.)
4141
-/

MathlibTest/Clean.lean

Lines changed: 4 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -42,13 +42,13 @@ example : True := by
4242
guard_hyp x' :ₛ id Nat := (1 : Nat)
4343

4444
let y := show Nat from 1
45-
guard_hyp y :ₛ Nat := let_fun this := 1; this
45+
guard_hyp y :ₛ Nat := have this := 1; this
4646
let y' := clean% show Nat from 1
4747
guard_hyp y' :ₛ Nat := 1
4848

49-
-- Not a tautological let_fun:
50-
let z := clean% let_fun x := 1; x + x
51-
guard_hyp z :ₛ Nat := let_fun x := 1; x + x
49+
-- Not a tautological have:
50+
let z := clean% have x := 1; x + x
51+
guard_hyp z :ₛ Nat := have x := 1; x + x
5252

5353
trivial
5454

lake-manifest.json

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -65,7 +65,7 @@
6565
"type": "git",
6666
"subDir": null,
6767
"scope": "leanprover-community",
68-
"rev": "95fdabf0825b787a865d266139bbc4f86e138cbc",
68+
"rev": "2eb4ccfc2628c4f68451cd73403ee2f9f29e2a9f",
6969
"name": "batteries",
7070
"manifestFile": "lake-manifest.json",
7171
"inputRev": "nightly-testing",

lean-toolchain

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1 +1 @@
1-
leanprover/lean4:nightly-2025-06-28
1+
leanprover/lean4:nightly-2025-06-30

scripts/bench/temci-config.run.yml

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -27,8 +27,8 @@
2727
properties: ['wall-clock', 'task-clock', 'instructions:u']
2828
rusage_properties: ['maxrss']
2929
cmd: |
30-
# run lake+lean like the file worker would
31-
LEAN_PATH=$(lake setup-file --no-build Mathlib Mathlib | jq -r '.paths.oleanPath | join(":")') lean Mathlib.lean
30+
# approximate `import Mathlib` in the editor
31+
lake lean Mathlib.lean
3232
runs: 5
3333
- attributes:
3434
description: size

0 commit comments

Comments
 (0)