-
Notifications
You must be signed in to change notification settings - Fork 367
New issue
Have a question about this project? Sign up for a free GitHub account to open an issue and contact its maintainers and the community.
By clicking “Sign up for GitHub”, you agree to our terms of service and privacy statement. We’ll occasionally send you account related emails.
Already on GitHub? Sign in to your account
[Merged by Bors] - chore: adaptations for nightly-2024-11-14 #19059
Changes from all commits
ca56307
2361f93
783e37d
afadc60
ea3e578
41dcf04
d9ad7e8
b831286
03f7ab6
336cd6a
3d52276
14ecc17
250bb15
5883eb2
0b56c17
7018874
abb3bda
2e937f9
65c3efc
fab6ff3
e5c238b
2cbf446
72854cf
b0a9ae3
bc60566
19f952e
2b2c002
3080ea2
f7cb8ad
764642e
3b9cb77
e76e277
134d8af
889a393
c310f98
6ff59b9
22c9339
5d03a2c
2895654
File filter
Filter by extension
Conversations
Jump to
Diff view
Diff view
There are no files selected for viewing
Original file line number | Diff line number | Diff line change |
---|---|---|
|
@@ -212,7 +212,7 @@ lemma finitelyAtomistic : ∀ s : Finset (LieIdeal R L), ↑s ⊆ {I : LieIdeal | |
set K := s'.sup id | ||
suffices I ≤ K by | ||
obtain ⟨t, hts', htI⟩ := finitelyAtomistic s' hs'S I this | ||
exact ⟨t, hts'.trans hs'.subset, htI⟩ | ||
exact ⟨t, Finset.Subset.trans hts' hs'.subset, htI⟩ | ||
There was a problem hiding this comment. Choose a reason for hiding this commentThe reason will be displayed to describe this comment to others. Learn more. Do we understand this regression? This makes me moderately sad... |
||
-- Since `I` is contained in the supremum of `J` with the supremum of `s'`, | ||
-- any element `x` of `I` can be written as `y + z` for some `y ∈ J` and `z ∈ K`. | ||
intro x hx | ||
|
Original file line number | Diff line number | Diff line change |
---|---|---|
|
@@ -63,14 +63,14 @@ theorem sigmaCurry_zero [∀ i j, Zero (δ i j)] : | |
|
||
@[simp] | ||
theorem sigmaCurry_add [∀ i j, AddZeroClass (δ i j)] (f g : Π₀ (i : Σ _, _), δ i.1 i.2) : | ||
sigmaCurry (f + g) = sigmaCurry f + sigmaCurry g := by | ||
sigmaCurry (f + g) = (sigmaCurry f + sigmaCurry g : Π₀ (i) (j), δ i j) := by | ||
There was a problem hiding this comment. Choose a reason for hiding this commentThe reason will be displayed to describe this comment to others. Learn more. This makes me a little bit sad, but I guess it's not too bad. |
||
ext (i j) | ||
rfl | ||
|
||
@[simp] | ||
theorem sigmaCurry_smul [Monoid γ] [∀ i j, AddMonoid (δ i j)] [∀ i j, DistribMulAction γ (δ i j)] | ||
(r : γ) (f : Π₀ (i : Σ _, _), δ i.1 i.2) : | ||
sigmaCurry (r • f) = r • sigmaCurry f := by | ||
sigmaCurry (r • f) = (r • sigmaCurry f : Π₀ (i) (j), δ i j) := by | ||
ext (i j) | ||
rfl | ||
|
||
|
Original file line number | Diff line number | Diff line change |
---|---|---|
|
@@ -35,11 +35,13 @@ variable {E : Type v} [Field E] {L : Type w} [Field L] | |
|
||
variable (A B C : Subfield E) | ||
|
||
set_option synthInstance.maxHeartbeats 400000 in | ||
There was a problem hiding this comment. Choose a reason for hiding this commentThe reason will be displayed to describe this comment to others. Learn more. Can we add some adaptation notes here? Or is this just a fact of life that we have to live with until we debug/speedup? |
||
/-- `Subfield.relrank A B` is defined to be `[B : A ⊓ B]` as a `Cardinal`, in particular, | ||
when `A ≤ B` it is `[B : A]`, the degree of the field extension `B / A`. | ||
This is similar to `Subgroup.relindex` but it is `Cardinal` valued. -/ | ||
noncomputable def relrank := Module.rank ↥(A ⊓ B) (extendScalars (inf_le_right : A ⊓ B ≤ B)) | ||
|
||
set_option synthInstance.maxHeartbeats 400000 in | ||
/-- The `Nat` version of `Subfield.relrank`. | ||
If `B / A ⊓ B` is an infinite extension, then it is zero. -/ | ||
noncomputable def relfinrank := finrank ↥(A ⊓ B) (extendScalars (inf_le_right : A ⊓ B ≤ B)) | ||
|
@@ -55,12 +57,14 @@ theorem relrank_eq_of_inf_eq (h : A ⊓ C = B ⊓ C) : relrank A C = relrank B C | |
theorem relfinrank_eq_of_inf_eq (h : A ⊓ C = B ⊓ C) : relfinrank A C = relfinrank B C := | ||
congr(toNat $(relrank_eq_of_inf_eq h)) | ||
|
||
set_option synthInstance.maxHeartbeats 400000 in | ||
/-- If `A ≤ B`, then `Subfield.relrank A B` is `[B : A]` -/ | ||
theorem relrank_eq_rank_of_le (h : A ≤ B) : relrank A B = Module.rank A (extendScalars h) := by | ||
rw [relrank] | ||
have := inf_of_le_left h | ||
congr! | ||
|
||
set_option synthInstance.maxHeartbeats 400000 in | ||
/-- If `A ≤ B`, then `Subfield.relfinrank A B` is `[B : A]` -/ | ||
theorem relfinrank_eq_finrank_of_le (h : A ≤ B) : relfinrank A B = finrank A (extendScalars h) := | ||
congr(toNat $(relrank_eq_rank_of_le h)) | ||
|
@@ -112,6 +116,7 @@ theorem relrank_top_left : relrank ⊤ A = 1 := relrank_eq_one_of_le le_top | |
@[simp] | ||
theorem relfinrank_top_left : relfinrank ⊤ A = 1 := relfinrank_eq_one_of_le le_top | ||
|
||
set_option synthInstance.maxHeartbeats 400000 in | ||
@[simp] | ||
theorem relrank_top_right : relrank A ⊤ = Module.rank A E := by | ||
rw [relrank_eq_rank_of_le (show A ≤ ⊤ from le_top), extendScalars_top, | ||
|
Original file line number | Diff line number | Diff line change |
---|---|---|
|
@@ -764,7 +764,7 @@ nonrec theorem _root_.MulEquiv.isHaarMeasure_map [BorelSpace G] [TopologicalGrou | |
[TopologicalGroup H] (e : G ≃* H) (he : Continuous e) (hesymm : Continuous e.symm) : | ||
IsHaarMeasure (Measure.map e μ) := | ||
let f : G ≃ₜ H := .mk e | ||
isHaarMeasure_map μ e he e.surjective f.isClosedEmbedding.tendsto_cocompact | ||
isHaarMeasure_map μ e.toMonoidHom he e.surjective f.isClosedEmbedding.tendsto_cocompact | ||
There was a problem hiding this comment. Choose a reason for hiding this commentThe reason will be displayed to describe this comment to others. Learn more. Why do we need this now? Makes me mildly sad. |
||
|
||
/-- A convenience wrapper for MeasureTheory.Measure.isAddHaarMeasure_map`. -/ | ||
instance _root_.ContinuousLinearEquiv.isAddHaarMeasure_map | ||
|
Original file line number | Diff line number | Diff line change |
---|---|---|
|
@@ -507,8 +507,10 @@ def arrowProdEquivProdArrow (α β γ : Type*) [MeasurableSpace α] [MeasurableS | |
measurable_toFun _ h := by | ||
simp_rw [Equiv.arrowProdEquivProdArrow, coe_fn_mk] | ||
exact MeasurableSet.preimage h (Measurable.prod_mk | ||
(measurable_pi_lambda (fun a c ↦ (a c).1) fun a ↦ (measurable_pi_apply a).fst) | ||
(measurable_pi_lambda (fun a c ↦ (a c).2) fun a ↦ (measurable_pi_apply a).snd )) | ||
(measurable_pi_lambda (fun (a : γ → α × β) c ↦ (a c).1) | ||
There was a problem hiding this comment. Choose a reason for hiding this commentThe reason will be displayed to describe this comment to others. Learn more. This becomes quite a bit more unreadable... mildly sad... |
||
fun a ↦ (measurable_pi_apply a).fst) | ||
(measurable_pi_lambda (fun (a : γ → α × β) c ↦ (a c).2) | ||
fun a ↦ (measurable_pi_apply a).snd)) | ||
measurable_invFun _ h := by | ||
simp_rw [Equiv.arrowProdEquivProdArrow, coe_fn_symm_mk] | ||
exact MeasurableSet.preimage h (by measurability) | ||
|
Original file line number | Diff line number | Diff line change |
---|---|---|
|
@@ -704,7 +704,7 @@ lemma finite_of_finite_type_of_isJacobsonRing (R S : Type*) [CommRing R] [Field | |
obtain ⟨ι, hι, f, hf⟩ := Algebra.FiniteType.iff_quotient_mvPolynomial'.mp ‹_› | ||
have : (algebraMap R S).IsIntegral := by | ||
rw [← f.comp_algebraMap] | ||
exact MvPolynomial.comp_C_integral_of_surjective_of_isJacobsonRing f hf | ||
exact MvPolynomial.comp_C_integral_of_surjective_of_isJacobsonRing f.toRingHom hf | ||
There was a problem hiding this comment. Choose a reason for hiding this commentThe reason will be displayed to describe this comment to others. Learn more. Why do we need this now? |
||
have : Algebra.IsIntegral R S := Algebra.isIntegral_def.mpr this | ||
exact Algebra.IsIntegral.finite | ||
|
||
|
Original file line number | Diff line number | Diff line change |
---|---|---|
@@ -1 +1 @@ | ||
leanprover/lean4:nightly-2024-11-13 | ||
leanprover/lean4:nightly-2024-11-14 |
There was a problem hiding this comment.
Choose a reason for hiding this comment
The reason will be displayed to describe this comment to others. Learn more.
This makes me a little bit sad, but we can certainly live with this.