Skip to content

Commit 667ad7e

Browse files
kim-emleanprover-community-mathlib4-botmathlib4-botjcommelingithub-actions
authored
chore: adaptations for nightly-2025-06-15 (#25940)
* Update lean-toolchain for testing leanprover/lean4#8584 * chore: adaptations for nightly-2025-06-02 * change phrasing of comments * chore(Geometry/Manifold): two simp-lemmas can be proven by simp * fix two lint problems * Trigger CI for leanprover/lean4#8519 * chore: bump to nightly-2025-06-03 * fix * fix * Update lean-toolchain for testing leanprover/lean4#8610 * fix * revert change in `Mathlib.Data.ZMOD.Basic` * fix Mathlib/Data/List/EditDistance/Estimator.lean * give specialized simp lemmas higher prio * simp can prove these * simp can prove these * chore: bump to nightly-2025-06-04 * bump toolchain * Adapt eqns * Revert "Adapt eqns" This reverts commit 34f1f7f. * Simply remove check for now * fix a bunch * fixes? * chore: adaptations for nightly-2025-06-04 * add `simp low` lemma `injOn_of_eq_iff_eq` * wip * wip * wip * fix * Trigger CI for leanprover-community/batteries#1220 * Merge master into nightly-testing * chore: bump to nightly-2025-06-05 * Kick CI * Bump lean4-cli * Bump import-graph * Kick CI * update lakefile * chore: use more robust syntax quotation in Shake * Trigger CI for leanprover/lean4#8419 * Revert "chore: use more robust syntax quotation in Shake" This reverts commit cd87328. * fix(Shake): fix import syntax @Kha this is deliberately using this approach because syntax quotations are also not robust but for a different reason: they fail to parse the new versions of the syntax (and do so at run time). And using all the optional doohickeys will not be future proof. The current setup is explicitly meant to ping me when there is a syntax change so I can evaluate the right way to handle it. In this case we want all the module options to be ignored (treated the same as a regular import for the purpose of dependency tracking), we don't want to fail. * cleanup lakefile * chore: bump to nightly-2025-06-06 * Update lean-toolchain for testing leanprover/lean4#8653 * fix * how did this get dropped?!?! * chore: bump to nightly-2025-06-07 * chore: bump to nightly-2025-06-08 * chore: bump to nightly-2025-06-09 * fix lakefile * fix lint-style for new Lean.Options API * chore: bump to nightly-2025-06-10 * chore: bump to nightly-2025-06-09 * merge lean-pr-testing-4 * chore: bump to nightly-2025-06-11 * chore: adaptations for nightly-2025-06-11 * Update Shake/Main.lean Co-authored-by: Johan Commelin <[email protected]> * Apply suggestions from code review * revert * chore: adaptations for nightly-2025-06-11 * 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 --------- Co-authored-by: leanprover-community-mathlib4-bot <[email protected]> Co-authored-by: mathlib4-bot <[email protected]> Co-authored-by: Johan Commelin <[email protected]> Co-authored-by: github-actions <[email protected]> Co-authored-by: Sebastian Ullrich <[email protected]> Co-authored-by: Jovan Gerbscheid <[email protected]> Co-authored-by: Joachim Breitner <[email protected]> Co-authored-by: Mario Carneiro <[email protected]> Co-authored-by: sgouezel <[email protected]> Co-authored-by: Kyle Miller <[email protected]>
1 parent c55fadb commit 667ad7e

File tree

18 files changed

+33
-36
lines changed

18 files changed

+33
-36
lines changed

Mathlib/Algebra/Group/Hom/Basic.lean

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -77,7 +77,6 @@ instance [Mul M] [CommSemigroup N] : Mul (M →ₙ* N) :=
7777
fun f g =>
7878
{ toFun := fun m => f m * g m,
7979
map_mul' := fun x y => by
80-
show f (x * y) * g (x * y) = f x * g x * (f y * g y)
8180
rw [f.map_mul, g.map_mul, ← mul_assoc, ← mul_assoc, mul_right_comm (f x)] }⟩
8281

8382
@[to_additive (attr := simp)]

Mathlib/Analysis/Normed/Module/Basic.lean

Lines changed: 0 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -512,18 +512,15 @@ abbrev PseudoMetricSpace.ofSeminormedSpaceCore {𝕜 E : Type*} [NormedField
512512
PseudoMetricSpace E where
513513
dist x y := ‖x - y‖
514514
dist_self x := by
515-
show ‖x - x‖ = 0
516515
simp only [sub_self]
517516
have : (0 : E) = (0 : 𝕜) • (0 : E) := by simp
518517
rw [this, core.norm_smul]
519518
simp
520519
dist_comm x y := by
521-
show ‖x - y‖ = ‖y - x‖
522520
have : y - x = (-1 : 𝕜) • (x - y) := by simp
523521
rw [this, core.norm_smul]
524522
simp
525523
dist_triangle x y z := by
526-
show ‖x - z‖ ≤ ‖x - y‖ + ‖y - z‖
527524
have : x - z = (x - y) + (y - z) := by abel
528525
rw [this]
529526
exact core.norm_triangle _ _

Mathlib/Analysis/SpecialFunctions/Log/Deriv.lean

Lines changed: 1 addition & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -251,8 +251,7 @@ theorem abs_log_sub_add_sum_range_le {x : ℝ} (h : |x| < 1) (n : ℕ) :
251251
theorem hasSum_pow_div_log_of_abs_lt_one {x : ℝ} (h : |x| < 1) :
252252
HasSum (fun n : ℕ => x ^ (n + 1) / (n + 1)) (-log (1 - x)) := by
253253
rw [Summable.hasSum_iff_tendsto_nat]
254-
· show Tendsto (fun n : ℕ => ∑ i ∈ range n, x ^ (i + 1) / (i + 1)) atTop (𝓝 (-log (1 - x)))
255-
rw [tendsto_iff_norm_sub_tendsto_zero]
254+
· rw [tendsto_iff_norm_sub_tendsto_zero]
256255
simp only [norm_eq_abs, sub_neg_eq_add]
257256
refine squeeze_zero (fun n => abs_nonneg _) (abs_log_sub_add_sum_range_le h) ?_
258257
suffices Tendsto (fun t : ℕ => |x| ^ (t + 1) / (1 - |x|)) atTop (𝓝 (|x| * 0 / (1 - |x|))) by

Mathlib/Data/List/Basic.lean

Lines changed: 0 additions & 11 deletions
Original file line numberDiff line numberDiff line change
@@ -548,19 +548,8 @@ theorem idxOf_of_notMem {l : List α} {a : α} : a ∉ l → idxOf a l = length
548548

549549
@[deprecated (since := "2025-01-30")] alias indexOf_of_not_mem := idxOf_of_notMem
550550

551-
theorem idxOf_le_length {a : α} {l : List α} : idxOf a l ≤ length l := by
552-
induction l with | nil => rfl | cons b l ih => ?_
553-
simp only [length, idxOf_cons, cond_eq_if, beq_iff_eq]
554-
by_cases h : b = a
555-
· rw [if_pos h]; exact Nat.zero_le _
556-
· rw [if_neg h]; exact succ_le_succ ih
557-
558551
@[deprecated (since := "2025-01-30")] alias indexOf_le_length := idxOf_le_length
559552

560-
theorem idxOf_lt_length_iff {a} {l : List α} : idxOf a l < length l ↔ a ∈ l :=
561-
fun h => Decidable.byContradiction fun al => Nat.ne_of_lt h <| idxOf_eq_length_iff.2 al,
562-
fun al => (lt_of_le_of_ne idxOf_le_length) fun h => idxOf_eq_length_iff.1 h al⟩
563-
564553
@[deprecated (since := "2025-01-30")] alias indexOf_lt_length_iff := idxOf_lt_length_iff
565554

566555
theorem idxOf_append_of_mem {a : α} (h : a ∈ l₁) : idxOf a (l₁ ++ l₂) = idxOf a l₁ := by

Mathlib/Data/Multiset/Fold.lean

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -90,7 +90,6 @@ theorem fold_dedup_idem [DecidableEq α] [hi : Std.IdempotentOp op] (s : Multise
9090
(dedup s).fold op b = s.fold op b :=
9191
Multiset.induction_on s (by simp) fun a s IH => by
9292
by_cases h : a ∈ s <;> simp [IH, h]
93-
show fold op b s = op a (fold op b s)
9493
rw [← cons_erase h, fold_cons_left, ← ha.assoc, hi.idempotent]
9594

9695
end Fold

Mathlib/Data/Nat/Pairing.lean

Lines changed: 2 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -59,11 +59,9 @@ alias pair_unpair' := pair_eq_of_unpair_eq
5959
@[simp]
6060
theorem unpair_pair (a b : ℕ) : unpair (pair a b) = (a, b) := by
6161
dsimp only [pair]; split_ifs with h
62-
· show unpair (b * b + a) = (a, b)
63-
have be : sqrt (b * b + a) = b := sqrt_add_eq _ (le_trans (le_of_lt h) (Nat.le_add_left _ _))
62+
· have be : sqrt (b * b + a) = b := sqrt_add_eq _ (le_trans (le_of_lt h) (Nat.le_add_left _ _))
6463
simp [unpair, be, Nat.add_sub_cancel_left, h]
65-
· show unpair (a * a + a + b) = (a, b)
66-
have ae : sqrt (a * a + (a + b)) = a := by
64+
· have ae : sqrt (a * a + (a + b)) = a := by
6765
rw [sqrt_add_eq]
6866
exact Nat.add_le_add_left (le_of_not_gt h) _
6967
simp [unpair, ae, Nat.not_lt_zero, Nat.add_assoc, Nat.add_sub_cancel_left]

Mathlib/Data/PFun.lean

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -439,7 +439,6 @@ theorem preimage_asSubtype (f : α →. β) (s : Set β) :
439439
f.asSubtype ⁻¹' s = Subtype.val ⁻¹' f.preimage s := by
440440
ext x
441441
simp only [Set.mem_preimage, Set.mem_setOf_eq, PFun.asSubtype, PFun.mem_preimage]
442-
show f.fn x.val _ ∈ s ↔ ∃ y ∈ s, y ∈ f x.val
443442
exact
444443
Iff.intro (fun h => ⟨_, h, Part.get_mem _⟩) fun ⟨y, ys, fxy⟩ =>
445444
have : f.fn x.val x.property ∈ f x.val := Part.get_mem _

Mathlib/FieldTheory/ChevalleyWarning.lean

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -139,7 +139,6 @@ theorem char_dvd_card_solutions_of_sum_lt {s : Finset ι} {f : ι → MvPolynomi
139139
-- We are now ready to apply the main machine, proven before.
140140
apply F.sum_eval_eq_zero
141141
-- It remains to verify the crucial assumption of this machine
142-
show F.totalDegree < (q - 1) * Fintype.card σ
143142
calc
144143
F.totalDegree ≤ ∑ i ∈ s, (1 - f i ^ (q - 1)).totalDegree := totalDegree_finset_prod s _
145144
_ ≤ ∑ i ∈ s, (q - 1) * (f i).totalDegree := sum_le_sum fun i _ => ?_

Mathlib/GroupTheory/CoprodI.lean

Lines changed: 2 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -1000,10 +1000,8 @@ theorem _root_.FreeGroup.injective_lift_of_ping_pong : Function.Injective (FreeG
10001000
let f : ∀ i, H i →* G := fun i => FreeGroup.lift fun _ => a i
10011001
let X' : ι → Set α := fun i => X i ∪ Y i
10021002
apply lift_injective_of_ping_pong f _ X'
1003-
· show ∀ i, (X' i).Nonempty
1004-
exact fun i => Set.Nonempty.inl (hXnonempty i)
1005-
· show Pairwise (Disjoint on X')
1006-
intro i j hij
1003+
· exact fun i => Set.Nonempty.inl (hXnonempty i)
1004+
· intro i j hij
10071005
simp only [X']
10081006
apply Disjoint.union_left <;> apply Disjoint.union_right
10091007
· exact hXdisj hij

Mathlib/GroupTheory/Coxeter/Inversion.lean

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -412,7 +412,6 @@ theorem prod_leftInvSeq (ω : List B) : prod (lis ω) = (π ω)⁻¹ := by
412412
theorem IsReduced.nodup_rightInvSeq {ω : List B} (rω : cs.IsReduced ω) : List.Nodup (ris ω) := by
413413
apply List.nodup_iff_getElem?_ne_getElem?.mpr
414414
intro j j' j_lt_j' j'_lt_length (dup : (rightInvSeq cs ω)[j]? = (rightInvSeq cs ω)[j']?)
415-
show False
416415
replace j'_lt_length : j' < List.length ω := by simpa using j'_lt_length
417416
rw [getElem?_eq_getElem (by simp; omega), getElem?_eq_getElem (by simp; omega)] at dup
418417
apply Option.some_injective at dup

0 commit comments

Comments
 (0)