Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit acbe099

Browse files
committed
feat(*): bump to lean 3.48.0 (#16292)
`fin n` is a structure now.
1 parent 87d8c4b commit acbe099

File tree

33 files changed

+173
-103
lines changed

33 files changed

+173
-103
lines changed

archive/imo/imo1987_q1.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -66,7 +66,7 @@ def fixed_points_equiv' :
6666
inv_fun := λ p,
6767
⟨⟨card (fixed_points p.1.2), (card_subtype_le _).trans_lt (nat.lt_succ_self _)⟩,
6868
⟨p.1.2, rfl⟩, ⟨p.1.1, p.2⟩⟩,
69-
left_inv := λ ⟨⟨k, hk⟩, ⟨σ, hσ⟩, ⟨x, hx⟩⟩, by { simp only [mem_fiber, subtype.coe_mk] at hσ,
69+
left_inv := λ ⟨⟨k, hk⟩, ⟨σ, hσ⟩, ⟨x, hx⟩⟩, by { simp only [mem_fiber, fin.coe_mk] at hσ,
7070
subst k, refl },
7171
right_inv := λ ⟨⟨x, σ⟩, h⟩, rfl }
7272

leanpkg.toml

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1,7 +1,7 @@
11
[package]
22
name = "mathlib"
33
version = "0.1"
4-
lean_version = "leanprover-community/lean:3.47.0"
4+
lean_version = "leanprover-community/lean:3.48.0"
55
path = "src"
66

77
[dependencies]

src/algebra/big_operators/fin.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -222,7 +222,7 @@ begin
222222
rw prod_take_succ _ _ this,
223223
have A : ((finset.univ : finset (fin n)).filter (λ j, j.val < i + 1))
224224
= ((finset.univ : finset (fin n)).filter (λ j, j.val < i)) ∪ {(⟨i, h⟩ : fin n)},
225-
by { ext j, simp [nat.lt_succ_iff_lt_or_eq, fin.ext_iff, - add_comm] },
225+
by { ext ⟨_, _⟩, simp [nat.lt_succ_iff_lt_or_eq] },
226226
have B : _root_.disjoint (finset.filter (λ (j : fin n), j.val < i) finset.univ)
227227
(singleton (⟨i, h⟩ : fin n)), by simp,
228228
rw [A, finset.prod_union B, IH],

src/algebra/char_zero/quotient.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -31,7 +31,7 @@ begin
3131
refine ⟨⟨(k % z).to_nat, _⟩, k / z, _⟩,
3232
{ rw [←int.coe_nat_lt, int.to_nat_of_nonneg (int.mod_nonneg _ hz)],
3333
exact (int.mod_lt _ hz).trans_eq (int.abs_eq_nat_abs _) },
34-
rw [subtype.coe_mk, int.to_nat_of_nonneg (int.mod_nonneg _ hz), int.div_add_mod] },
34+
rw [fin.coe_mk, int.to_nat_of_nonneg (int.mod_nonneg _ hz), int.div_add_mod] },
3535
{ rintro ⟨k, n, h⟩,
3636
exact ⟨_, h⟩, },
3737
end

src/algebraic_topology/simplex_category.lean

Lines changed: 6 additions & 6 deletions
Original file line numberDiff line numberDiff line change
@@ -193,7 +193,7 @@ begin
193193
rcases i with ⟨i, _⟩,
194194
rcases j with ⟨j, _⟩,
195195
rcases k with ⟨k, _⟩,
196-
simp only [subtype.mk_le_mk, fin.cast_succ_mk] at H,
196+
simp only [fin.mk_le_mk, fin.cast_succ_mk] at H,
197197
dsimp,
198198
split_ifs,
199199
-- Most of the goals can now be handled by `linarith`,
@@ -241,28 +241,28 @@ begin
241241
rcases i with ⟨i, _⟩,
242242
rcases j with ⟨j, _⟩,
243243
rcases k with ⟨k, _⟩,
244-
simp only [subtype.mk_lt_mk, fin.cast_succ_mk] at H,
244+
simp only [fin.mk_lt_mk, fin.cast_succ_mk] at H,
245245
suffices : ite (_ < ite (k < i + 1) _ _) _ _ =
246246
ite _ (ite (j < k) (k - 1) k) (ite (j < k) (k - 1) k + 1),
247247
{ simpa [apply_dite fin.cast_succ, fin.pred_above] with push_cast, },
248248
split_ifs,
249249
-- Most of the goals can now be handled by `linarith`,
250250
-- but we have to deal with three of them by hand.
251251
swap 2,
252-
{ simp only [subtype.mk_lt_mk] at h_1,
252+
{ simp only [fin.mk_lt_mk] at h_1,
253253
simp only [not_lt] at h_2,
254254
simp only [self_eq_add_right, one_ne_zero],
255255
exact lt_irrefl (k - 1) (lt_of_lt_of_le
256256
(nat.pred_lt (ne_of_lt (lt_of_le_of_lt (zero_le _) h_1)).symm)
257257
(le_trans (nat.le_of_lt_succ h) h_2)) },
258258
swap 4,
259-
{ simp only [subtype.mk_lt_mk] at h_1,
259+
{ simp only [fin.mk_lt_mk] at h_1,
260260
simp only [not_lt] at h,
261261
simp only [nat.add_succ_sub_one, add_zero],
262262
exfalso,
263263
exact lt_irrefl _ (lt_of_le_of_lt (nat.le_pred_of_lt (nat.lt_of_succ_le h)) h_3), },
264264
swap 4,
265-
{ simp only [subtype.mk_lt_mk] at h_1,
265+
{ simp only [fin.mk_lt_mk] at h_1,
266266
simp only [not_lt] at h_3,
267267
simp only [nat.add_succ_sub_one, add_zero],
268268
exact (nat.succ_pred_eq_of_pos (lt_of_le_of_lt (zero_le _) h_2)).symm, },
@@ -281,7 +281,7 @@ begin
281281
rcases i with ⟨i, _⟩,
282282
rcases j with ⟨j, _⟩,
283283
rcases k with ⟨k, _⟩,
284-
simp only [subtype.mk_le_mk] at H,
284+
simp only [fin.mk_le_mk] at H,
285285
-- At this point `simp with push_cast` makes good progress, but neither `simp?` nor `squeeze_simp`
286286
-- return usable sets of lemmas.
287287
-- To avoid using a non-terminal simp, we make a `suffices` statement indicating the shape

src/algebraic_topology/split_simplicial_object.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -89,7 +89,7 @@ begin
8989
induction Δ₁ using opposite.rec,
9090
induction Δ₂ using opposite.rec,
9191
simp only at h₁,
92-
have h₂ : Δ₁ = Δ₂ := by { ext1, simpa only [subtype.mk_eq_mk] using h₁.1, },
92+
have h₂ : Δ₁ = Δ₂ := by { ext1, simpa only [fin.mk_eq_mk] using h₁.1, },
9393
subst h₂,
9494
refine ext _ _ rfl _,
9595
ext : 2,

src/algebraic_topology/topological_simplex.lean

Lines changed: 1 addition & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -40,8 +40,7 @@ lemma to_Top_obj.ext {x : simplex_category} (f g : x.to_Top_obj) :
4040
def to_Top_map {x y : simplex_category} (f : x ⟶ y) : x.to_Top_obj → y.to_Top_obj :=
4141
λ g, ⟨λ i, ∑ j in (finset.univ.filter (λ k, f k = i)), g j,
4242
begin
43-
dsimp [to_Top_obj],
44-
simp only [finset.filter_congr_decidable, finset.sum_congr],
43+
simp only [finset.filter_congr_decidable, finset.sum_congr, to_Top_obj, set.mem_set_of],
4544
rw ← finset.sum_bUnion,
4645
convert g.2,
4746
{ rw finset.eq_univ_iff_forall,

src/analysis/complex/upper_half_plane/basic.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -154,7 +154,7 @@ begin
154154
change _ = (_ * (_ / _) + _) * _,
155155
field_simp [denom_ne_zero, -denom, -num],
156156
simp only [matrix.mul, dot_product, fin.sum_univ_succ, denom, num, coe_coe, subgroup.coe_mul,
157-
general_linear_group.coe_mul, fintype.univ_of_subsingleton, fin.mk_eq_subtype_mk, fin.mk_zero,
157+
general_linear_group.coe_mul, fintype.univ_of_subsingleton, fin.mk_zero,
158158
finset.sum_singleton, fin.succ_zero_eq_one, complex.of_real_add, complex.of_real_mul],
159159
ring
160160
end
@@ -167,7 +167,7 @@ begin
167167
rw denom_cocycle,
168168
field_simp [denom_ne_zero, -denom, -num],
169169
simp only [matrix.mul, dot_product, fin.sum_univ_succ, num, denom, coe_coe, subgroup.coe_mul,
170-
general_linear_group.coe_mul, fintype.univ_of_subsingleton, fin.mk_eq_subtype_mk, fin.mk_zero,
170+
general_linear_group.coe_mul, fintype.univ_of_subsingleton, fin.mk_zero,
171171
finset.sum_singleton, fin.succ_zero_eq_one, complex.of_real_add, complex.of_real_mul],
172172
ring
173173
end

src/analysis/convex/stone_separation.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -74,7 +74,7 @@ begin
7474
congr' 3,
7575
rw [←mul_smul, ←mul_rotate, mul_right_comm, mul_smul, ←mul_smul _ av, mul_rotate, mul_smul _ bz,
7676
←smul_add],
77-
simp only [list.map, list.pmap, nat.add_def, add_zero, fin.mk_eq_subtype_mk, fin.mk_bit0,
77+
simp only [list.map, list.pmap, nat.add_def, add_zero, fin.mk_bit0,
7878
fin.mk_one, list.foldr_cons, list.foldr_nil],
7979
refl,
8080
end

src/combinatorics/composition.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -719,7 +719,7 @@ def composition_as_set_equiv (n : ℕ) : composition_as_set n ≃ finset (fin (n
719719
erw [set.mem_set_of_eq],
720720
simp only [this, false_or, add_right_inj, add_eq_zero_iff, one_ne_zero, false_and, fin.coe_mk],
721721
split,
722-
{ rintros ⟨j, js, hj⟩, convert js, exact (fin.ext_iff _ _).2 hj },
722+
{ rintros ⟨j, js, hj⟩, convert js, exact fin.ext_iff.2 hj },
723723
{ assume h, exact ⟨i, h, rfl⟩ }
724724
end }
725725

0 commit comments

Comments
 (0)