Skip to content

Commit 490d2d4

Browse files
kim-emeric-wiesernomeata
committed
chore: move to v4.6.0-rc1, merging adaptations from bump/v4.6.0 (#10176)
Co-authored-by: Scott Morrison <scott.morrison@gmail.com> Co-authored-by: Eric Wieser <wieser.eric@gmail.com> Co-authored-by: Joachim Breitner <mail@joachim-breitner.de>
1 parent 86ecbac commit 490d2d4

File tree

161 files changed

+485
-481
lines changed

Some content is hidden

Large Commits have some content hidden by default. Use the searchbox below for content that may be hidden.

161 files changed

+485
-481
lines changed

.github/workflows/bors.yml

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -284,7 +284,7 @@ jobs:
284284
run: |
285285
git clone https://github.com/leanprover/lean4checker
286286
cd lean4checker
287-
git checkout toolchain/v4.5.0-rc1
287+
git checkout toolchain/v4.6.0-rc1
288288
# Now that the git hash is embedded in each olean,
289289
# we need to compile lean4checker on the same toolchain
290290
cp ../lean-toolchain .

.github/workflows/build.yml

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -291,7 +291,7 @@ jobs:
291291
run: |
292292
git clone https://github.com/leanprover/lean4checker
293293
cd lean4checker
294-
git checkout toolchain/v4.5.0-rc1
294+
git checkout toolchain/v4.6.0-rc1
295295
# Now that the git hash is embedded in each olean,
296296
# we need to compile lean4checker on the same toolchain
297297
cp ../lean-toolchain .

.github/workflows/build.yml.in

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -270,7 +270,7 @@ jobs:
270270
run: |
271271
git clone https://github.com/leanprover/lean4checker
272272
cd lean4checker
273-
git checkout toolchain/v4.5.0-rc1
273+
git checkout toolchain/v4.6.0-rc1
274274
# Now that the git hash is embedded in each olean,
275275
# we need to compile lean4checker on the same toolchain
276276
cp ../lean-toolchain .

.github/workflows/build_fork.yml

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -288,7 +288,7 @@ jobs:
288288
run: |
289289
git clone https://github.com/leanprover/lean4checker
290290
cd lean4checker
291-
git checkout toolchain/v4.5.0-rc1
291+
git checkout toolchain/v4.6.0-rc1
292292
# Now that the git hash is embedded in each olean,
293293
# we need to compile lean4checker on the same toolchain
294294
cp ../lean-toolchain .

Archive/Examples/IfNormalization/Result.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -99,7 +99,7 @@ def normalize (l : AList (fun _ : ℕ => Bool)) :
9999
by_cases w = v <;> ◾⟩
100100
| some b =>
101101
have i' := normalize l (.ite (lit b) t e); ⟨i'.1, ◾⟩
102-
termination_by normalize e => e.normSize
102+
termination_by e => e.normSize
103103

104104
/-
105105
We recall the statement of the if-normalization problem.

Archive/Examples/IfNormalization/WithoutAesop.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -116,7 +116,7 @@ def normalize' (l : AList (fun _ : ℕ => Bool)) :
116116
| some b =>
117117
have ⟨e', he'⟩ := normalize' l (.ite (lit b) t e)
118118
⟨e', by simp_all⟩
119-
termination_by normalize' e => e.normSize'
119+
termination_by e' => e'.normSize'
120120

121121
example : IfNormalization :=
122122
fun e => (normalize' ∅ e).1,

Archive/Wiedijk100Theorems/BallotProblem.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -171,7 +171,7 @@ theorem countedSequence_finite : ∀ p q : ℕ, (countedSequence p q).Finite
171171
rw [counted_succ_succ, Set.finite_union, Set.finite_image_iff (List.cons_injective.injOn _),
172172
Set.finite_image_iff (List.cons_injective.injOn _)]
173173
exact ⟨countedSequence_finite _ _, countedSequence_finite _ _⟩
174-
termination_by _ p q => p + q -- Porting note: Added `termination_by`
174+
termination_by p q => p + q -- Porting note: Added `termination_by`
175175
#align ballot.counted_sequence_finite Ballot.countedSequence_finite
176176

177177
theorem countedSequence_nonempty : ∀ p q : ℕ, (countedSequence p q).Nonempty
@@ -215,7 +215,7 @@ theorem count_countedSequence : ∀ p q : ℕ, count (countedSequence p q) = (p
215215
count_injective_image List.cons_injective, count_countedSequence _ _]
216216
· norm_cast
217217
rw [add_assoc, add_comm 1 q, ← Nat.choose_succ_succ, Nat.succ_eq_add_one, add_right_comm]
218-
termination_by _ p q => p + q -- Porting note: Added `termination_by`
218+
termination_by p q => p + q -- Porting note: Added `termination_by`
219219
#align ballot.count_counted_sequence Ballot.count_countedSequence
220220

221221
theorem first_vote_pos :

Counterexamples/CharPZeroNeCharZero.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -34,7 +34,7 @@ theorem withZero_unit_charP_zero : CharP (WithZero Unit) 0 :=
3434
#align counterexample.with_zero_unit_char_p_zero Counterexample.withZero_unit_charP_zero
3535

3636
theorem withZero_unit_not_charZero : ¬CharZero (WithZero Unit) := fun ⟨h⟩ =>
37-
h.ne (by simp : 1 + 10 + 1) (by simp)
37+
h.ne (by simp : 1 + 10 + 1) (by set_option simprocs false in simp)
3838
#align counterexample.with_zero_unit_not_char_zero Counterexample.withZero_unit_not_charZero
3939

4040
end Counterexample

Mathlib/Algebra/Category/GroupCat/Basic.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -491,7 +491,7 @@ end CategoryTheory.Aut
491491
instance GroupCat.forget_reflects_isos : ReflectsIsomorphisms (forget GroupCat.{u}) where
492492
reflects {X Y} f _ := by
493493
let i := asIso ((forget GroupCat).map f)
494-
let e : X ≃* Y := { i.toEquiv with map_mul' := by aesop }
494+
let e : X ≃* Y := { i.toEquiv with map_mul' := map_mul _ }
495495
exact IsIso.of_iso e.toGroupCatIso
496496
set_option linter.uppercaseLean3 false in
497497
#align Group.forget_reflects_isos GroupCat.forget_reflects_isos
@@ -502,7 +502,7 @@ set_option linter.uppercaseLean3 false in
502502
instance CommGroupCat.forget_reflects_isos : ReflectsIsomorphisms (forget CommGroupCat.{u}) where
503503
reflects {X Y} f _ := by
504504
let i := asIso ((forget CommGroupCat).map f)
505-
let e : X ≃* Y := { i.toEquiv with map_mul' := by aesop }
505+
let e : X ≃* Y := { i.toEquiv with map_mul' := map_mul _}
506506
exact IsIso.of_iso e.toCommGroupCatIso
507507
set_option linter.uppercaseLean3 false in
508508
#align CommGroup.forget_reflects_isos CommGroupCat.forget_reflects_isos

Mathlib/Algebra/DirectLimit.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -719,7 +719,7 @@ theorem of.zero_exact_aux [Nonempty ι] [IsDirected ι (· ≤ ·)] {x : FreeCom
719719
have := DirectedSystem.map_map (fun i j h => f' i j h) hij (le_refl j : j ≤ j)
720720
rw [this]
721721
exact sub_self _
722-
exacts [Or.inr rfl, Or.inl rfl]
722+
exacts [Or.inl rfl, Or.inr rfl]
723723
· refine' ⟨i, {⟨i, 1⟩}, _, isSupported_sub (isSupported_of.2 rfl) isSupported_one, _⟩
724724
· rintro k (rfl | h)
725725
rfl

0 commit comments

Comments
 (0)