Skip to content

Commit

Permalink
Merge remote-tracking branch 'refs/remotes/origin/mrb/universes' into…
Browse files Browse the repository at this point in the history
… mrb/universes
  • Loading branch information
mattrobball committed Aug 7, 2023
1 parent ced8c9b commit 00d53f8
Show file tree
Hide file tree
Showing 43 changed files with 40 additions and 99 deletions.
2 changes: 1 addition & 1 deletion Mathlib/Algebra/Category/ModuleCat/ChangeOfRings.lean
Original file line number Diff line number Diff line change
Expand Up @@ -333,7 +333,7 @@ namespace RestrictionCoextensionAdj
variable {R : Type u₁} {S : Type u₂} [Ring R] [Ring S] (f : R →+* S)

-- Porting note: too much time
set_option maxHeartbeats 600000 in
set_option maxHeartbeats 500000 in
/-- Given `R`-module X and `S`-module Y, any `g : (restrictScalars f).obj Y ⟶ X`
corresponds to `Y ⟶ (coextendScalars f).obj X` by sending `y ↦ (s ↦ g (s • y))`
-/
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Algebra/DirectLimit.lean
Original file line number Diff line number Diff line change
Expand Up @@ -733,7 +733,7 @@ protected theorem inv_mul_cancel {p : Ring.DirectLimit G f} (hp : p ≠ 0) : inv
#align field.direct_limit.inv_mul_cancel Field.DirectLimit.inv_mul_cancel

-- porting note: this takes some time, had to increase heartbeats
set_option maxHeartbeats 1000000 in
set_option maxHeartbeats 500000 in
/-- Noncomputable field structure on the direct limit of fields.
See note [reducible non-instances]. -/
@[reducible]
Expand Down
4 changes: 2 additions & 2 deletions Mathlib/Algebra/Homology/DifferentialObject.lean
Original file line number Diff line number Diff line change
Expand Up @@ -80,7 +80,7 @@ theorem d_eqToHom (X : HomologicalComplex V (ComplexShape.up' b)) {x y z : β} (
X.d x y ≫ eqToHom (congr_arg X.X h) = X.d x z := by cases h; simp
#align homological_complex.d_eq_to_hom HomologicalComplex.d_eqToHom

set_option maxHeartbeats 800000 in
set_option maxHeartbeats 400000 in
/-- The functor from differential graded objects to homological complexes.
-/
@[simps]
Expand Down Expand Up @@ -146,7 +146,7 @@ to the category of homological complexes in `V`.
-/
@[simps]
def dgoEquivHomologicalComplex :
DifferentialObject ℤ (GradedObjectWithShift b V) ≌
DifferentialObject ℤ (GradedObjectWithShift b V) ≌
HomologicalComplex V (ComplexShape.up' b) where
functor := dgoToHomologicalComplex b V
inverse := homologicalComplexToDGO b V
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Algebra/Homology/LocalCohomology.lean
Original file line number Diff line number Diff line change
Expand Up @@ -116,7 +116,7 @@ variable {R : Type max u v v'} [CommRing R] {D : Type v} [SmallCategory D]

variable {E : Type v'} [SmallCategory E] (I' : E ⥤ D) (I : D ⥤ Ideal R)

set_option maxHeartbeats 400000 in
set_option maxHeartbeats 250000 in
/-- Local cohomology along a composition of diagrams. -/
def diagramComp (i : ℕ) : diagram (I' ⋙ I) i ≅ I'.op ⋙ diagram I i :=
Iso.refl _
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Algebra/Homology/ModuleCat.lean
Original file line number Diff line number Diff line change
Expand Up @@ -92,7 +92,6 @@ theorem homology_ext' {M : ModuleCat R} (i : ι) {h k : C.homology i ⟶ M}
set_option linter.uppercaseLean3 false in
#align Module.homology_ext' ModuleCat.homology_ext'

set_option maxHeartbeats 400000 in
-- porting note: `erw` had to be used instead of `simp`
-- see https://github.com/leanprover-community/mathlib4/issues/5026
/-- We give an alternative proof of `homology_map_eq_of_homotopy`,
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Algebra/Module/PID.lean
Original file line number Diff line number Diff line change
Expand Up @@ -164,7 +164,6 @@ theorem exists_smul_eq_zero_and_mk_eq {z : M} (hz : Module.IsTorsionBy R M (p ^

open Finset Multiset

set_option maxHeartbeats 800000 in
/-- A finitely generated `p ^ ∞`-torsion module over a PID is isomorphic to a direct sum of some
`R ⧸ R ∙ (p ^ e i)` for some `e i`.-/
theorem torsion_by_prime_power_decomposition (hN : Module.IsTorsion' N (Submonoid.powers p))
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Algebra/MonoidAlgebra/Grading.lean
Original file line number Diff line number Diff line change
Expand Up @@ -120,7 +120,6 @@ instance grade.gradedMonoid [AddMonoid M] [CommSemiring R] :

variable [AddMonoid M] [DecidableEq ι] [AddMonoid ι] [CommSemiring R] (f : M →+ ι)

set_option maxHeartbeats 260000 in
/-- Auxiliary definition; the canonical grade decomposition, used to provide
`DirectSum.decompose`. -/
def decomposeAux : AddMonoidAlgebra R M →ₐ[R] ⨁ i : ι, gradeBy R f i :=
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Analysis/Analytic/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -1082,7 +1082,6 @@ section

variable (p : FormalMultilinearSeries 𝕜 E F) {x y : E} {r R : ℝ≥0}

set_option synthInstance.maxHeartbeats 100000 in
/-- A term of `FormalMultilinearSeries.changeOriginSeries`.
Given a formal multilinear series `p` and a point `x` in its ball of convergence,
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Analysis/Analytic/Composition.lean
Original file line number Diff line number Diff line change
Expand Up @@ -743,7 +743,7 @@ end FormalMultilinearSeries

open FormalMultilinearSeries

set_option maxHeartbeats 450000 in
set_option maxHeartbeats 300000 in
/-- If two functions `g` and `f` have power series `q` and `p` respectively at `f x` and `x`, then
`g ∘ f` admits the power series `q.comp p` at `x`. -/
theorem HasFPowerSeriesAt.comp {g : F → G} {f : E → F} {q : FormalMultilinearSeries 𝕜 F G}
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Analysis/Calculus/ContDiff.lean
Original file line number Diff line number Diff line change
Expand Up @@ -2542,7 +2542,6 @@ theorem norm_iteratedFDeriv_mul_le {f : E → A} {g : E → A} {N : ℕ∞} (hf

end

set_option maxHeartbeats 300000 in
/-- If the derivatives within a set of `g` at `f x` are bounded by `C`, and the `i`-th derivative
within a set of `f` at `x` is bounded by `D^i` for all `1 ≤ i ≤ n`, then the `n`-th derivative
of `g ∘ f` is bounded by `n! * C * D^n`.
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Analysis/Calculus/FDeriv/Symmetric.lean
Original file line number Diff line number Diff line change
Expand Up @@ -58,7 +58,6 @@ variable {E F : Type*} [NormedAddCommGroup E] [NormedSpace ℝ E] [NormedAddComm
{f'' : E →L[ℝ] E →L[ℝ] F} (hf : ∀ x ∈ interior s, HasFDerivAt f (f' x) x) {x : E} (xs : x ∈ s)
(hx : HasFDerivWithinAt f' f'' (interior s) x)

set_option maxHeartbeats 300000 in
/-- Assume that `f` is differentiable inside a convex set `s`, and that its derivative `f'` is
differentiable at a point `x`. Then, given two vectors `v` and `w` pointing inside `s`, one can
Taylor-expand to order two the function `f` on the segment `[x + h v, x + h (v + w)]`, giving a
Expand Down
4 changes: 2 additions & 2 deletions Mathlib/Analysis/Convex/Between.lean
Original file line number Diff line number Diff line change
Expand Up @@ -339,8 +339,8 @@ theorem sbtw_iff_mem_image_Ioo_and_ne [NoZeroSMulDivisors R V] {x y z : P} :
refine' ⟨⟨t, Set.mem_Icc_of_Ioo ht, rfl⟩, _⟩
rw [lineMap_apply, ← @vsub_ne_zero V, ← @vsub_ne_zero V _ _ _ _ z, vadd_vsub_assoc, vsub_self,
vadd_vsub_assoc, ← neg_vsub_eq_vsub_rev z x, ← @neg_one_smul R, ← add_smul, ← sub_eq_add_neg]
have : z -ᵥ x ≠ 0 := by simpa using hxz.symm
simp [smul_ne_zero, this, sub_eq_zero, ht.1.ne.symm, ht.2.ne, hxz.symm]
-- have : z -ᵥ x ≠ 0 := by simpa using hxz.symm
simp [smul_ne_zero, sub_eq_zero, ht.1.ne.symm, ht.2.ne, hxz.symm]
#align sbtw_iff_mem_image_Ioo_and_ne sbtw_iff_mem_image_Ioo_and_ne

variable (R)
Expand Down
4 changes: 2 additions & 2 deletions Mathlib/Analysis/Convolution.lean
Original file line number Diff line number Diff line change
Expand Up @@ -1196,8 +1196,8 @@ variable [IsROrC 𝕜] [NormedSpace 𝕜 E] [NormedSpace 𝕜 E'] [NormedSpace
[NormedSpace 𝕜 G] [NormedAddCommGroup P] [NormedSpace 𝕜 P] {μ : MeasureTheory.Measure G}
(L : E →L[𝕜] E' →L[𝕜] F)

-- porting note: the lemma is slow, added `set_option maxHeartbeats 300000 in`
set_option maxHeartbeats 300000 in
-- porting note: the lemma is slow, added `set_option maxHeartbeats 250000 in`
set_option maxHeartbeats 250000 in
/-- The derivative of the convolution `f * g` is given by `f * Dg`, when `f` is locally integrable
and `g` is `C^1` and compactly supported. Version where `g` depends on an additional parameter in an
open subset `s` of a parameter space `P` (and the compact support `k` is independent of the
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Analysis/InnerProductSpace/Adjoint.lean
Original file line number Diff line number Diff line change
Expand Up @@ -223,7 +223,6 @@ theorem isSelfAdjoint_iff' {A : E →L[𝕜] E} : IsSelfAdjoint A ↔ Continuous
Iff.rfl
#align continuous_linear_map.is_self_adjoint_iff' ContinuousLinearMap.isSelfAdjoint_iff'

set_option maxHeartbeats 300000 in -- Porting note: Added to prevent timeout.
instance : CstarRing (E →L[𝕜] E) :=
by
intro A
Expand Down
11 changes: 4 additions & 7 deletions Mathlib/Analysis/InnerProductSpace/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -1796,12 +1796,9 @@ theorem innerSL_apply_norm (x : E) : ‖innerSL 𝕜 x‖ = ‖x‖ := by
set_option linter.uppercaseLean3 false in
#align innerSL_apply_norm innerSL_apply_norm

set_option synthInstance.maxHeartbeats 80000 in
-- porting note: I'm not sure why the maxHeartbeats needed to be so high here
/-- The inner product as a continuous sesquilinear map, with the two arguments flipped. -/
def innerSLFlip : E →L[𝕜] E →L⋆[𝕜] 𝕜 :=
@ContinuousLinearMap.flipₗᵢ' 𝕜 𝕜 𝕜 E E 𝕜 _ _ _ _ _ _ _ _ _ (RingHom.id 𝕜) (starRingEnd 𝕜) _ _
(innerSL 𝕜)
ContinuousLinearMap.flipₗᵢ' E E 𝕜 (RingHom.id 𝕜) (starRingEnd 𝕜) (innerSL 𝕜)
set_option linter.uppercaseLean3 false in
#align innerSL_flip innerSLFlip

Expand All @@ -1817,11 +1814,11 @@ namespace ContinuousLinearMap

variable {E' : Type*} [NormedAddCommGroup E'] [InnerProductSpace 𝕜 E']

set_option maxHeartbeats 500000 in
set_option synthInstance.maxHeartbeats 100000 in
set_option synthInstance.maxHeartbeats 40000 in
-- Note: explicitly noncomputable due to strange compilation attempts by Lean
/-- Given `f : E →L[𝕜] E'`, construct the continuous sesquilinear form `fun x y ↦ ⟪x, A y⟫`, given
as a continuous linear map. -/
def toSesqForm : (E →L[𝕜] E') →L[𝕜] E' →L⋆[𝕜] E →L[𝕜] 𝕜 :=
noncomputable def toSesqForm : (E →L[𝕜] E') →L[𝕜] E' →L⋆[𝕜] E →L[𝕜] 𝕜 :=
(ContinuousLinearMap.flipₗᵢ' E E' 𝕜 (starRingEnd 𝕜) (RingHom.id 𝕜)).toContinuousLinearEquiv ∘L
ContinuousLinearMap.compSL E E' (E' →L⋆[𝕜] 𝕜) (RingHom.id 𝕜) (RingHom.id 𝕜) (innerSLFlip 𝕜)
#align continuous_linear_map.to_sesq_form ContinuousLinearMap.toSesqForm
Expand Down
2 changes: 0 additions & 2 deletions Mathlib/Analysis/InnerProductSpace/Spectrum.lean
Original file line number Diff line number Diff line change
Expand Up @@ -138,8 +138,6 @@ theorem orthogonalComplement_iSup_eigenspaces_eq_bot' :
rw [iSup_ne_bot_subtype, hT.orthogonalComplement_iSup_eigenspaces_eq_bot]
#align linear_map.is_symmetric.orthogonal_supr_eigenspaces_eq_bot' LinearMap.IsSymmetric.orthogonalComplement_iSup_eigenspaces_eq_bot'

-- porting note: a modest increast in the `synthInstance.maxHeartbeats`, but we should still fix it.
set_option synthInstance.maxHeartbeats 23000 in
/-- The eigenspaces of a self-adjoint operator on a finite-dimensional inner product space `E` gives
an internal direct sum decomposition of `E`.
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Analysis/NormedSpace/MazurUlam.lean
Original file line number Diff line number Diff line change
Expand Up @@ -39,7 +39,6 @@ noncomputable section

namespace IsometryEquiv

set_option maxHeartbeats 250000 in
/-- If an isometric self-homeomorphism of a normed vector space over `ℝ` fixes `x` and `y`,
then it fixes the midpoint of `[x, y]`. This is a lemma for a more general Mazur-Ulam theorem,
see below. -/
Expand Down
8 changes: 0 additions & 8 deletions Mathlib/Analysis/NormedSpace/Multilinear.lean
Original file line number Diff line number Diff line change
Expand Up @@ -1025,7 +1025,6 @@ theorem _root_.ContinuousLinearEquiv.compContinuousMultilinearMapL_apply (g : G
rfl
#align continuous_linear_equiv.comp_continuous_multilinear_mapL_apply ContinuousLinearEquiv.compContinuousMultilinearMapL_apply

set_option maxHeartbeats 250000 in
/-- Flip arguments in `f : G →L[𝕜] ContinuousMultilinearMap 𝕜 E G'` to get
`ContinuousMultilinearMap 𝕜 E (G →L[𝕜] G')` -/
@[simps! apply_apply]
Expand Down Expand Up @@ -1429,15 +1428,13 @@ def continuousMultilinearCurryLeftEquiv :

variable {𝕜 Ei G}

set_option synthInstance.maxHeartbeats 25000 in
@[simp]
theorem continuousMultilinearCurryLeftEquiv_apply
(f : Ei 0 →L[𝕜] ContinuousMultilinearMap 𝕜 (fun i : Fin n => Ei i.succ) G) (v : ∀ i, Ei i) :
continuousMultilinearCurryLeftEquiv 𝕜 Ei G f v = f (v 0) (tail v) :=
rfl
#align continuous_multilinear_curry_left_equiv_apply continuousMultilinearCurryLeftEquiv_apply

set_option synthInstance.maxHeartbeats 25000 in
@[simp]
theorem continuousMultilinearCurryLeftEquiv_symm_apply (f : ContinuousMultilinearMap 𝕜 Ei G)
(x : Ei 0) (v : ∀ i : Fin n, Ei i.succ) :
Expand Down Expand Up @@ -1866,15 +1863,13 @@ def curryFinFinset {k l n : ℕ} {s : Finset (Fin n)} (hk : s.card = k) (hl : s

variable {𝕜 G G'}

set_option synthInstance.maxHeartbeats 25000 in
@[simp]
theorem curryFinFinset_apply (hk : s.card = k) (hl : sᶜ.card = l) (f : G[×n]→L[𝕜] G')
(mk : Fin k → G) (ml : Fin l → G) : curryFinFinset 𝕜 G G' hk hl f mk ml =
f fun i => Sum.elim mk ml ((finSumEquivOfFinset hk hl).symm i) :=
rfl
#align continuous_multilinear_map.curry_fin_finset_apply ContinuousMultilinearMap.curryFinFinset_apply

set_option synthInstance.maxHeartbeats 25000 in
@[simp]
theorem curryFinFinset_symm_apply (hk : s.card = k) (hl : sᶜ.card = l)
(f : G[×k]→L[𝕜] G[×l]→L[𝕜] G') (m : Fin n → G) : (curryFinFinset 𝕜 G G' hk hl).symm f m =
Expand All @@ -1883,7 +1878,6 @@ theorem curryFinFinset_symm_apply (hk : s.card = k) (hl : sᶜ.card = l)
rfl
#align continuous_multilinear_map.curry_fin_finset_symm_apply ContinuousMultilinearMap.curryFinFinset_symm_apply

set_option synthInstance.maxHeartbeats 25000 in
-- @[simp] -- Porting note: simp removed: simp can reduce LHS
theorem curryFinFinset_symm_apply_piecewise_const (hk : s.card = k) (hl : sᶜ.card = l)
(f : G[×k]→L[𝕜] G[×l]→L[𝕜] G') (x y : G) :
Expand All @@ -1892,15 +1886,13 @@ theorem curryFinFinset_symm_apply_piecewise_const (hk : s.card = k) (hl : sᶜ.c
MultilinearMap.curryFinFinset_symm_apply_piecewise_const hk hl _ x y
#align continuous_multilinear_map.curry_fin_finset_symm_apply_piecewise_const ContinuousMultilinearMap.curryFinFinset_symm_apply_piecewise_const

set_option synthInstance.maxHeartbeats 25000 in
@[simp]
theorem curryFinFinset_symm_apply_const (hk : s.card = k) (hl : sᶜ.card = l)
(f : G[×k]→L[𝕜] G[×l]→L[𝕜] G') (x : G) :
((curryFinFinset 𝕜 G G' hk hl).symm f fun _ => x) = f (fun _ => x) fun _ => x :=
rfl
#align continuous_multilinear_map.curry_fin_finset_symm_apply_const ContinuousMultilinearMap.curryFinFinset_symm_apply_const

set_option synthInstance.maxHeartbeats 25000 in
-- @[simp] -- Porting note: simp removed: simp can reduce LHS
theorem curryFinFinset_apply_const (hk : s.card = k) (hl : sᶜ.card = l) (f : G[×n]→L[𝕜] G')
(x y : G) : (curryFinFinset 𝕜 G G' hk hl f (fun _ => x) fun _ => y) =
Expand Down
8 changes: 1 addition & 7 deletions Mathlib/Analysis/NormedSpace/OperatorNorm.lean
Original file line number Diff line number Diff line change
Expand Up @@ -815,8 +815,6 @@ theorem flip_smul (c : 𝕜₃) (f : E →SL[σ₁₃] F →SL[σ₂₃] G) : (c

variable (E F G σ₁₃ σ₂₃)

set_option maxHeartbeats 300000 in
set_option synthInstance.maxHeartbeats 25000 in
/-- Flip the order of arguments of a continuous bilinear map.
This is a version bundled as a `LinearIsometryEquiv`.
For an unbundled version see `ContinuousLinearMap.flip`. -/
Expand All @@ -832,21 +830,18 @@ def flipₗᵢ' : (E →SL[σ₁₃] F →SL[σ₂₃] G) ≃ₗᵢ[𝕜₃] F

variable {E F G σ₁₃ σ₂₃}

set_option synthInstance.maxHeartbeats 25000 in
@[simp]
theorem flipₗᵢ'_symm : (flipₗᵢ' E F G σ₂₃ σ₁₃).symm = flipₗᵢ' F E G σ₁₃ σ₂₃ :=
rfl
#align continuous_linear_map.flipₗᵢ'_symm ContinuousLinearMap.flipₗᵢ'_symm

set_option synthInstance.maxHeartbeats 75000 in
@[simp]
theorem coe_flipₗᵢ' : ⇑(flipₗᵢ' E F G σ₂₃ σ₁₃) = flip :=
rfl
#align continuous_linear_map.coe_flipₗᵢ' ContinuousLinearMap.coe_flipₗᵢ'

variable (𝕜 E Fₗ Gₗ)

set_option maxHeartbeats 250000 in
/-- Flip the order of arguments of a continuous bilinear map.
This is a version bundled as a `LinearIsometryEquiv`.
For an unbundled version see `ContinuousLinearMap.flip`. -/
Expand All @@ -867,7 +862,6 @@ theorem flipₗᵢ_symm : (flipₗᵢ 𝕜 E Fₗ Gₗ).symm = flipₗᵢ 𝕜 F
rfl
#align continuous_linear_map.flipₗᵢ_symm ContinuousLinearMap.flipₗᵢ_symm

set_option synthInstance.maxHeartbeats 60000 in
@[simp]
theorem coe_flipₗᵢ : ⇑(flipₗᵢ 𝕜 E Fₗ Gₗ) = flip :=
rfl
Expand Down Expand Up @@ -1013,7 +1007,7 @@ variable (M₁ : Type u₁) [SeminormedAddCommGroup M₁] [NormedSpace 𝕜 M₁

variable {Eₗ} (𝕜)

set_option maxHeartbeats 750000 in
set_option maxHeartbeats 600000 in
/-- `ContinuousLinearMap.prodMap` as a continuous linear map. -/
def prodMapL : (M₁ →L[𝕜] M₂) × (M₃ →L[𝕜] M₄) →L[𝕜] M₁ × M₃ →L[𝕜] M₂ × M₄ :=
ContinuousLinearMap.copy
Expand Down
Original file line number Diff line number Diff line change
Expand Up @@ -254,19 +254,19 @@ theorem elementalStarAlgebra.bijective_characterSpaceToSpectrum :
#align elemental_star_algebra.bijective_character_space_to_spectrum elementalStarAlgebra.bijective_characterSpaceToSpectrum

-- porting note: it would be good to understand why and where Lean is having trouble here
set_option synthInstance.maxHeartbeats 40000 in
-- set_option synthInstance.maxHeartbeats 40000 in
/-- The homeomorphism between the character space of the unital C⋆-subalgebra generated by a
single normal element `a : A` and `spectrum ℂ a`. -/
noncomputable def elementalStarAlgebra.characterSpaceHomeo :
characterSpace ℂ (elementalStarAlgebra ℂ a) ≃ₜ spectrum ℂ a :=
@Continuous.homeoOfEquivCompactToT2 _ _ _ _ _ _
(Equiv.ofBijective (elementalStarAlgebra.characterSpaceToSpectrum a)
Continuous.homeoOfEquivCompactToT2
(f := Equiv.ofBijective (elementalStarAlgebra.characterSpaceToSpectrum a)
(elementalStarAlgebra.bijective_characterSpaceToSpectrum a))
(elementalStarAlgebra.continuous_characterSpaceToSpectrum a)
#align elemental_star_algebra.character_space_homeo elementalStarAlgebra.characterSpaceHomeo

-- porting note: it would be good to understand why and where Lean is having trouble here
set_option maxHeartbeats 350000 in
-- set_option maxHeartbeats 350000 in
/-- **Continuous functional calculus.** Given a normal element `a : A` of a unital C⋆-algebra,
the continuous functional calculus is a `StarAlgEquiv` from the complex-valued continuous
functions on the spectrum of `a` to the unital C⋆-subalgebra generated by `a`. Moreover, this
Expand Down
2 changes: 0 additions & 2 deletions Mathlib/Analysis/SpecialFunctions/Pow/Deriv.lean
Original file line number Diff line number Diff line change
Expand Up @@ -204,7 +204,6 @@ theorem HasDerivWithinAt.cpow_const (hf : HasDerivWithinAt f f' s x)
(Complex.hasStrictDerivAt_cpow_const h0).hasDerivAt.comp_hasDerivWithinAt x hf
#align has_deriv_within_at.cpow_const HasDerivWithinAt.cpow_const

set_option maxHeartbeats 1000000 in
/-- Although `fun x => x ^ r` for fixed `r` is *not* complex-differentiable along the negative real
line, it is still real-differentiable, and the derivative is what one would formally expect. -/
theorem hasDerivAt_ofReal_cpow {x : ℝ} (hx : x ≠ 0) {r : ℂ} (hr : r ≠ -1) :
Expand Down Expand Up @@ -270,7 +269,6 @@ theorem hasStrictFDerivAt_rpow_of_pos (p : ℝ × ℝ) (hp : 0 < p.1) :
div_eq_mul_inv, smul_smul, smul_smul, mul_assoc, add_comm]
#align real.has_strict_fderiv_at_rpow_of_pos Real.hasStrictFDerivAt_rpow_of_pos

set_option maxHeartbeats 1000000 in
/-- `(x, y) ↦ x ^ y` is strictly differentiable at `p : ℝ × ℝ` such that `p.fst < 0`. -/
theorem hasStrictFDerivAt_rpow_of_neg (p : ℝ × ℝ) (hp : p.1 < 0) :
HasStrictFDerivAt (fun x : ℝ × ℝ => x.1 ^ x.2)
Expand Down
4 changes: 2 additions & 2 deletions Mathlib/FieldTheory/IsAlgClosed/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -299,8 +299,8 @@ AlgHom.comp
(AlgEquiv.adjoinSingletonEquivAdjoinRootMinpoly R x).toAlgHom

-- porting note: this was much faster in lean 3
set_option maxHeartbeats 800000 in
set_option synthInstance.maxHeartbeats 400000 in
set_option maxHeartbeats 600000 in
set_option synthInstance.maxHeartbeats 150000 in
theorem maximalSubfieldWithHom_eq_top : (maximalSubfieldWithHom K L M).carrier = ⊤ := by
rw [eq_top_iff]
intro x _
Expand Down
Original file line number Diff line number Diff line change
Expand Up @@ -139,15 +139,15 @@ instance : Add (LeftInvariantDerivation I G) where
⟨X + Y, fun g => by
simp only [map_add, Derivation.coe_add, left_invariant', Pi.add_apply]⟩

set_option maxHeartbeats 400000 in
-- set_option maxHeartbeats 400000 in
instance : Neg (LeftInvariantDerivation I G) where
neg X := ⟨-X, fun g => by
-- porting note: was simp [left_invariant']
-- `rw` fails without detailed type annotations too; also it needs a lot of time
rw [map_neg (Derivation.evalAt (𝕜 := 𝕜) (1 : G)), map_neg (𝒅ₕ (smoothLeftMul_one I g)),
left_invariant', map_neg (Derivation.evalAt (𝕜 := 𝕜) g)]⟩

set_option maxHeartbeats 400000 in
set_option maxHeartbeats 300000 in
instance : Sub (LeftInvariantDerivation I G) where
sub X Y := ⟨X - Y, fun g => by
-- porting note: was simp [left_invariant']
Expand Down Expand Up @@ -262,7 +262,7 @@ theorem comp_L : (X f).comp (𝑳 I g) = X (f.comp (𝑳 I g)) := by
set_option linter.uppercaseLean3 false in
#align left_invariant_derivation.comp_L LeftInvariantDerivation.comp_L

set_option maxHeartbeats 400000 in
-- set_option maxHeartbeats 400000 in
instance : Bracket (LeftInvariantDerivation I G) (LeftInvariantDerivation I G) where
bracket X Y :=
⟨⁅(X : Derivation 𝕜 C^∞⟮I, G; 𝕜⟯ C^∞⟮I, G; 𝕜⟯), Y⁆, fun g => by
Expand Down
5 changes: 2 additions & 3 deletions Mathlib/LinearAlgebra/AdicCompletion.lean
Original file line number Diff line number Diff line change
Expand Up @@ -85,7 +85,6 @@ def Hausdorffification : Type _ :=
M ⧸ (⨅ n : ℕ, I ^ n • ⊤ : Submodule R M)
#align Hausdorffification Hausdorffification

set_option maxHeartbeats 700000 in
/-- The completion of a module with respect to an ideal. This is not necessarily Hausdorff.
In fact, this is only complete if the ideal is finitely generated. -/
def adicCompletion : Submodule R (∀ n : ℕ, M ⧸ (I ^ n • ⊤ : Submodule R M)) where
Expand Down Expand Up @@ -213,7 +212,7 @@ def of : M →ₗ[R] adicCompletion I M where
map_smul' _ _ := rfl
#align adic_completion.of adicCompletion.of

set_option maxHeartbeats 700000 in
set_option maxHeartbeats 250000 in
@[simp]
theorem of_apply (x : M) (n : ℕ) : (of I M x).1 n = mkQ _ x :=
rfl
Expand All @@ -236,7 +235,7 @@ theorem eval_apply (n : ℕ) (f : adicCompletion I M) : eval I M n f = f.1 n :=
rfl
#align adic_completion.eval_apply adicCompletion.eval_apply

set_option maxHeartbeats 700000 in
set_option maxHeartbeats 250000 in
theorem eval_of (n : ℕ) (x : M) : eval I M n (of I M x) = mkQ _ x :=
rfl
#align adic_completion.eval_of adicCompletion.eval_of
Expand Down
Loading

0 comments on commit 00d53f8

Please sign in to comment.