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

Commit 60e279b

Browse files
ericrbgurkud
andcommitted
chore(*): update to lean 3.36.0 (#11253)
The main breaking change is the change in elaboration of double membership binders into x hx y hy, from x y hx hy. Co-authored-by: Yury G. Kudryashov <urkud@urkud.name>
1 parent dd1242d commit 60e279b

File tree

79 files changed

+267
-264
lines changed

Some content is hidden

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

79 files changed

+267
-264
lines changed

archive/imo/imo1994_q1.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -85,7 +85,7 @@ begin
8585
rcases hx with ⟨i, ⟨hi, rfl⟩⟩,
8686
have h1 : a i + a (fin.last m - k) ≤ n,
8787
{ linarith only [h, a.monotone hi.2] },
88-
have h2 : a i + a (fin.last m - k) ∈ A := hadd _ _ (ha _) (ha _) h1,
88+
have h2 : a i + a (fin.last m - k) ∈ A := hadd _ (ha _) _ (ha _) h1,
8989
rw [←mem_coe, ←range_order_emb_of_fin A hm, set.mem_range] at h2,
9090
cases h2 with j hj,
9191
use j,

archive/imo/imo2021_q1.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -143,7 +143,7 @@ begin
143143
{ rw [finset.mem_insert, finset.mem_singleton, finset.mem_singleton],
144144
push_neg,
145145
exact ⟨⟨hab.ne, (hab.trans hbc).ne⟩, hbc.ne⟩ } },
146-
{ intros x y hx hy hxy,
146+
{ intros x hx y hy hxy,
147147
simp only [finset.mem_insert, finset.mem_singleton] at hx hy,
148148
rcases hx with rfl|rfl|rfl; rcases hy with rfl|rfl|rfl,
149149
all_goals { contradiction <|> assumption <|> simpa only [add_comm x y], } },
@@ -177,5 +177,5 @@ begin
177177
simp only [finset.subset_iff, finset.mem_inter] at hCA,
178178
-- Now we split into the two cases C ⊆ [n, 2n] \ A and C ⊆ A, which can be dealt with identically.
179179
cases hCA; [right, left];
180-
exact ⟨a, b, (hCA ha).2, (hCA hb).2, hab, h₁ a b (hCA ha).1 (hCA hb).1 hab⟩,
180+
exact ⟨a, (hCA ha).2, b, (hCA hb).2, hab, h₁ a (hCA ha).1 b (hCA hb).1 hab⟩,
181181
end

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.35.1"
4+
lean_version = "leanprover-community/lean:3.36.0"
55
path = "src"
66

77
[dependencies]

src/algebra/lie/solvable.lean

Lines changed: 4 additions & 8 deletions
Original file line numberDiff line numberDiff line change
@@ -261,19 +261,15 @@ instance radical_is_solvable [is_noetherian R L] : is_solvable R (radical R L) :
261261
begin
262262
have hwf := lie_submodule.well_founded_of_noetherian R L L,
263263
rw ← complete_lattice.is_sup_closed_compact_iff_well_founded at hwf,
264-
refine hwf { I : lie_ideal R L | is_solvable R I } _ _,
265-
{ use ⊥, exact lie_algebra.is_solvable_bot R L, },
266-
{ intros I J hI hJ, apply lie_algebra.is_solvable_add R L; [exact hI, exact hJ], },
264+
refine hwf { I : lie_ideal R L | is_solvable R I } ⟨⊥, _⟩ (λ I hI J hJ, _),
265+
{ exact lie_algebra.is_solvable_bot R L, },
266+
{ apply lie_algebra.is_solvable_add R L, exacts [hI, hJ] },
267267
end
268268

269269
/-- The `→` direction of this lemma is actually true without the `is_noetherian` assumption. -/
270270
lemma lie_ideal.solvable_iff_le_radical [is_noetherian R L] (I : lie_ideal R L) :
271271
is_solvable R I ↔ I ≤ radical R L :=
272-
begin
273-
split; intros h,
274-
{ exact le_Sup h, },
275-
{ apply le_solvable_ideal_solvable h, apply_instance, },
276-
end
272+
⟨λ h, le_Sup h, λ h, le_solvable_ideal_solvable h infer_instance⟩
277273

278274
lemma center_le_radical : center R L ≤ radical R L :=
279275
have h : is_solvable R (center R L), { apply_instance, }, le_Sup h

src/algebraic_geometry/prime_spectrum/basic.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -349,7 +349,7 @@ topological_space.of_closed (set.range prime_spectrum.zero_locus)
349349
simp only [hf],
350350
exact ⟨_, zero_locus_Union _⟩
351351
end
352-
(by { rintro _ _ ⟨s, rfl⟩ ⟨t, rfl⟩, exact ⟨_, (union_zero_locus s t).symm⟩ })
352+
(by { rintro _ ⟨s, rfl⟩ _ ⟨t, rfl⟩, exact ⟨_, (union_zero_locus s t).symm⟩ })
353353

354354
lemma is_open_iff (U : set (prime_spectrum R)) :
355355
is_open U ↔ ∃ s, Uᶜ = zero_locus s :=

src/algebraic_geometry/properties.lean

Lines changed: 3 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -207,7 +207,9 @@ begin
207207
exact H } },
208208
{ intros R hX s hs x,
209209
erw [basic_open_eq_of_affine', prime_spectrum.basic_open_eq_bot_iff] at hs,
210-
replace hs := (hs.map (Spec_Γ_identity.app R).inv).eq_zero,
210+
replace hs := (hs.map (Spec_Γ_identity.app R).inv),
211+
-- what the hell?!
212+
replace hs := @is_nilpotent.eq_zero _ _ _ _ (show _, from _) hs,
211213
rw coe_hom_inv_id at hs,
212214
rw [hs, map_zero],
213215
exact @@is_reduced.component_reduced hX ⊤ }

src/algebraic_geometry/structure_sheaf.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -694,7 +694,7 @@ begin
694694
refine ⟨(λ i, a i * (h i) ^ N), (λ i, (h i) ^ (N + 1)),
695695
(λ i, eq_to_hom (basic_opens_eq i) ≫ iDh i), _, _, _⟩,
696696
{ simpa only [basic_opens_eq] using h_cover },
697-
{ intros i j hi hj,
697+
{ intros i hi j hj,
698698
-- Here we need to show that our new fractions `a i / h i` satisfy the normalization condition
699699
-- Of course, the power `N` we used to expand the fractions might be bigger than the power
700700
-- `n (i, j)` which was originally chosen. We denote their difference by `k`
@@ -795,7 +795,7 @@ begin
795795
rw [← hb, finset.sum_mul, finset.mul_sum],
796796
apply finset.sum_congr rfl,
797797
intros j hj,
798-
rw [mul_assoc, ah_ha j i hj hi],
798+
rw [mul_assoc, ah_ha j hj i hi],
799799
ring
800800
end
801801

src/analysis/ODE/gronwall.lean

Lines changed: 5 additions & 6 deletions
Original file line numberDiff line numberDiff line change
@@ -165,9 +165,8 @@ begin
165165
assume t ht,
166166
have := dist_triangle4_right (f' t) (g' t) (v t (f t)) (v t (g t)),
167167
rw [dist_eq_norm] at this,
168-
apply le_trans this,
169-
apply le_trans (add_le_add (add_le_add (f_bound t ht) (g_bound t ht))
170-
(hv t (f t) (g t) (hfs t ht) (hgs t ht))),
168+
refine this.trans ((add_le_add (add_le_add (f_bound t ht) (g_bound t ht))
169+
(hv t (f t) (hfs t ht) (g t) (hgs t ht))).trans _),
171170
rw [dist_eq_norm, add_comm]
172171
end
173172

@@ -188,7 +187,7 @@ theorem dist_le_of_approx_trajectories_ODE {v : ℝ → E → E}
188187
(ha : dist (f a) (g a) ≤ δ) :
189188
∀ t ∈ Icc a b, dist (f t) (g t) ≤ gronwall_bound δ K (εf + εg) (t - a) :=
190189
have hfs : ∀ t ∈ Ico a b, f t ∈ (@univ E), from λ t ht, trivial,
191-
dist_le_of_approx_trajectories_ODE_of_mem_set (λ t x y hx hy, (hv t).dist_le_mul x y)
190+
dist_le_of_approx_trajectories_ODE_of_mem_set (λ t x hx y hy, (hv t).dist_le_mul x y)
192191
hf hf' f_bound hfs hg hg' g_bound (λ t ht, trivial) ha
193192

194193
/-- If `f` and `g` are two exact solutions of the same ODE, then the distance between them
@@ -234,7 +233,7 @@ theorem dist_le_of_trajectories_ODE {v : ℝ → E → E}
234233
(ha : dist (f a) (g a) ≤ δ) :
235234
∀ t ∈ Icc a b, dist (f t) (g t) ≤ δ * exp (K * (t - a)) :=
236235
have hfs : ∀ t ∈ Ico a b, f t ∈ (@univ E), from λ t ht, trivial,
237-
dist_le_of_trajectories_ODE_of_mem_set (λ t x y hx hy, (hv t).dist_le_mul x y)
236+
dist_le_of_trajectories_ODE_of_mem_set (λ t x hx y hy, (hv t).dist_le_mul x y)
238237
hf hf' hfs hg hg' (λ t ht, trivial) ha
239238

240239
/-- There exists only one solution of an ODE \(\dot x=v(t, x)\) in a set `s ⊆ ℝ × E` with
@@ -270,5 +269,5 @@ theorem ODE_solution_unique {v : ℝ → E → E}
270269
(ha : f a = g a) :
271270
∀ t ∈ Icc a b, f t = g t :=
272271
have hfs : ∀ t ∈ Ico a b, f t ∈ (@univ E), from λ t ht, trivial,
273-
ODE_solution_unique_of_mem_set (λ t x y hx hy, (hv t).dist_le_mul x y)
272+
ODE_solution_unique_of_mem_set (λ t x hx y hy, (hv t).dist_le_mul x y)
274273
hf hf' hfs hg hg' (λ t ht, trivial) ha

src/analysis/analytic/basic.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -565,7 +565,7 @@ lemma has_fpower_series_on_ball.image_sub_sub_deriv_le
565565
∃ C, ∀ (y z ∈ emetric.ball x r'),
566566
∥f y - f z - (p 1 (λ _, y - z))∥ ≤ C * (max ∥y - x∥ ∥z - x∥) * ∥y - z∥ :=
567567
by simpa only [is_O_principal, mul_assoc, normed_field.norm_mul, norm_norm, prod.forall,
568-
emetric.mem_ball, prod.edist_eq, max_lt_iff, and_imp]
568+
emetric.mem_ball, prod.edist_eq, max_lt_iff, and_imp, @forall_swap (_ < _) E]
569569
using hf.is_O_image_sub_image_sub_deriv_principal hr
570570

571571
/-- If `f` has formal power series `∑ n, pₙ` at `x`, then

src/analysis/box_integral/basic.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -658,7 +658,7 @@ begin
658658
have : 0 ≤ μ.to_box_additive J, from ennreal.to_real_nonneg,
659659
rw [norm_smul, real.norm_eq_abs, abs_of_nonneg this, ← dist_eq_norm],
660660
refine mul_le_mul_of_nonneg_left _ this,
661-
refine Hδ _ _ (tagged_prepartition.tag_mem_Icc _ _) (tagged_prepartition.tag_mem_Icc _ _) _,
661+
refine Hδ _ (tagged_prepartition.tag_mem_Icc _ _) _ (tagged_prepartition.tag_mem_Icc _ _) _,
662662
rw [← add_halves δ],
663663
refine (dist_triangle_left _ _ J.upper).trans (add_le_add (h₁.1 _ _ _) (h₂.1 _ _ _)),
664664
{ exact prepartition.bUnion_index_mem _ hJ },

0 commit comments

Comments
 (0)