Skip to content
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

chore: update/remove heart beat bumps #6370

Closed
wants to merge 27 commits into from
Closed
Show file tree
Hide file tree
Changes from all commits
Commits
Show all changes
27 commits
Select commit Hold shift + click to select a range
2637c7e
type _ -> type*
mattrobball Aug 4, 2023
0c9345f
remove
mattrobball Aug 4, 2023
b1dfc8c
fix some files
mattrobball Aug 4, 2023
9095a38
fix more
mattrobball Aug 4, 2023
8064173
build
mattrobball Aug 4, 2023
ced8c9b
long lines
mattrobball Aug 4, 2023
466a8a7
lint
mattrobball Aug 4, 2023
00d53f8
Merge remote-tracking branch 'refs/remotes/origin/mrb/universes' into…
mattrobball Aug 6, 2023
3c0e5c2
Merge branch 'mrb/universes_2' into mrb/universes
mattrobball Aug 7, 2023
75c10e6
Merge remote-tracking branch 'refs/remotes/origin/mrb/universes' into…
mattrobball Aug 6, 2023
c06e819
comment out all bumps
mattrobball Aug 7, 2023
e02809f
restore necessary bumps
mattrobball Aug 7, 2023
79c6822
revisit all places where Type* fails
mattrobball Aug 7, 2023
5e7bd9a
move Type* and Sort* and set imports
mattrobball Aug 8, 2023
914e9e1
Sort _ -> Sort*
mattrobball Aug 8, 2023
cde37ba
fix errors
mattrobball Aug 8, 2023
b5ec8c8
lint
mattrobball Aug 8, 2023
6fbf296
comment out bumps again
mattrobball Aug 8, 2023
29fa063
restore bumps
mattrobball Aug 8, 2023
9c65527
Merge branch 'master' into mrb/universes
mattrobball Aug 9, 2023
43a7236
remove notes and update author
mattrobball Aug 9, 2023
c17ce8b
Merge branch 'master' (early part) into mrb/universes
eric-wieser Aug 10, 2023
51e3570
Merge branch 'master' into mrb/universes
eric-wieser Aug 10, 2023
60486c5
Merge branch 'master' into mrb/universes
mattrobball Aug 29, 2023
4a33a0e
restore
mattrobball Aug 30, 2023
1e47611
remove comments
mattrobball Aug 30, 2023
ce8dea4
remove comments
mattrobball Aug 30, 2023
File filter

Filter by extension

Filter by extension

Conversations
Failed to load comments.
Loading
Jump to
Jump to file
Failed to load files.
Loading
Diff view
Diff view
4 changes: 2 additions & 2 deletions Mathlib/Algebra/Category/FGModuleCat/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -265,15 +265,15 @@ theorem FGModuleCatEvaluation_apply (f : FGModuleCatDual K V) (x : V) :

-- Porting note: extremely slow, was fast in mathlib3.
-- I tried many things using `dsimp` and `change`, but couldn't find anything faster than this.
set_option maxHeartbeats 1600000 in
set_option maxHeartbeats 1500000 in
private theorem coevaluation_evaluation :
letI V' : FGModuleCat K := FGModuleCatDual K V
(𝟙 V' ⊗ FGModuleCatCoevaluation K V) ≫ (α_ V' V V').inv ≫ (FGModuleCatEvaluation K V ⊗ 𝟙 V') =
(ρ_ V').hom ≫ (λ_ V').inv := by
apply contractLeft_assoc_coevaluation K V

-- Porting note: extremely slow, was fast in mathlib3.
set_option maxHeartbeats 1600000 in
set_option maxHeartbeats 400000 in
private theorem evaluation_coevaluation :
(FGModuleCatCoevaluation K V ⊗ 𝟙 V) ≫
(α_ V (FGModuleCatDual K V) V).hom ≫ (𝟙 V ⊗ FGModuleCatEvaluation K V) =
Expand Down
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/Category/ModuleCat/Monoidal/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -135,7 +135,7 @@ theorem associator_naturality {X₁ X₂ X₃ Y₁ Y₂ Y₃ : ModuleCat R} (f
#align Module.monoidal_category.associator_naturality ModuleCat.MonoidalCategory.associator_naturality

-- Porting note: very slow!
set_option maxHeartbeats 1600000 in
set_option maxHeartbeats 1200000 in
theorem pentagon (W X Y Z : ModuleCat R) :
tensorHom (associator W X Y).hom (𝟙 Z) ≫
(associator W (tensorObj X Y) Z).hom ≫ tensorHom (𝟙 W) (associator X Y Z).hom =
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
2 changes: 1 addition & 1 deletion Mathlib/Algebra/Homology/DifferentialObject.lean
Original file line number Diff line number Diff line change
Expand Up @@ -82,7 +82,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
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/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
6 changes: 3 additions & 3 deletions Mathlib/AlgebraicGeometry/AffineScheme.lean
Original file line number Diff line number Diff line change
Expand Up @@ -498,7 +498,7 @@ instance basicOpenSectionsToAffine_isIso {X : Scheme} {U : Opens X} (hU : IsAffi
rw [hU.fromSpec_range]
exact RingedSpace.basicOpen_le _ _

set_option maxHeartbeats 310000 in
set_option maxHeartbeats 300000 in
theorem isLocalization_basicOpen {X : Scheme} {U : Opens X} (hU : IsAffineOpen U)
(f : X.presheaf.obj (op U)) : IsLocalization.Away f (X.presheaf.obj (op <| X.basicOpen f)) := by
apply
Expand Down Expand Up @@ -626,7 +626,7 @@ theorem IsAffineOpen.isLocalization_stalk_aux {X : Scheme} (U : Opens X)
rw [eqToHom_trans]
#align algebraic_geometry.is_affine_open.is_localization_stalk_aux AlgebraicGeometry.IsAffineOpen.isLocalization_stalk_aux

set_option maxHeartbeats 3200000 in
set_option maxHeartbeats 1600000 in
theorem IsAffineOpen.isLocalization_stalk_aux' {X : Scheme} {U : Opens X} (hU : IsAffineOpen U)
(y : PrimeSpectrum (X.presheaf.obj <| op U)) (hy : hU.fromSpec.1.base y ∈ U) :
hU.fromSpec.val.c.app (op U) ≫ (Scheme.Spec.obj <| op (X.presheaf.obj <| op U)).presheaf.germ
Expand Down Expand Up @@ -657,7 +657,7 @@ theorem IsAffineOpen.isLocalization_stalk_aux' {X : Scheme} {U : Opens X} (hU :
rw [Category.id_comp]
rfl

set_option maxHeartbeats 800000 in
set_option maxHeartbeats 500000 in
theorem IsAffineOpen.isLocalization_stalk' {X : Scheme} {U : Opens X} (hU : IsAffineOpen U)
(y : PrimeSpectrum (X.presheaf.obj <| op U)) (hy : hU.fromSpec.1.base y ∈ U) :
haveI : IsAffine _ := hU
Expand Down
4 changes: 2 additions & 2 deletions Mathlib/AlgebraicGeometry/Morphisms/QuasiSeparated.lean
Original file line number Diff line number Diff line change
Expand Up @@ -310,7 +310,7 @@ theorem exists_eq_pow_mul_of_isAffineOpen (X : Scheme) (U : Opens X.carrier) (hU
simpa [mul_comm x] using d.symm
#align algebraic_geometry.exists_eq_pow_mul_of_is_affine_open AlgebraicGeometry.exists_eq_pow_mul_of_isAffineOpen

set_option maxHeartbeats 700000 in
set_option maxHeartbeats 500000 in
theorem exists_eq_pow_mul_of_is_compact_of_quasi_separated_space_aux (X : Scheme)
(S : X.affineOpens) (U₁ U₂ : Opens X.carrier) {n₁ n₂ : ℕ} {y₁ : X.presheaf.obj (op U₁)}
{y₂ : X.presheaf.obj (op U₂)} {f : X.presheaf.obj (op <| U₁ ⊔ U₂)}
Expand Down Expand Up @@ -372,7 +372,7 @@ theorem exists_eq_pow_mul_of_is_compact_of_quasi_separated_space_aux (X : Scheme
exact e
#align algebraic_geometry.exists_eq_pow_mul_of_is_compact_of_quasi_separated_space_aux AlgebraicGeometry.exists_eq_pow_mul_of_is_compact_of_quasi_separated_space_aux

set_option maxHeartbeats 7000000 in
set_option maxHeartbeats 700000 in
theorem exists_eq_pow_mul_of_isCompact_of_isQuasiSeparated (X : Scheme.{u}) (U : Opens X.carrier)
(hU : IsCompact U.1) (hU' : IsQuasiSeparated U.1) (f : X.presheaf.obj (op U))
(x : X.presheaf.obj (op <| X.basicOpen f)) :
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/AlgebraicGeometry/Morphisms/RingHomProperties.lean
Original file line number Diff line number Diff line change
Expand Up @@ -283,7 +283,7 @@ theorem sourceAffineLocally_isLocal (h₁ : RingHom.RespectsIso @P)
variable (hP : RingHom.PropertyIsLocal @P)

-- Porting note: the terms here are getting huge ~ 1/2 Gb for the goal midway (with `pp.explicit`)
set_option maxHeartbeats 13000000 in
set_option maxHeartbeats 4000000 in
theorem sourceAffineLocally_of_source_open_cover_aux (h₁ : RingHom.RespectsIso @P)
(h₃ : RingHom.OfLocalizationSpanTarget @P) {X Y : Scheme} (f : X ⟶ Y) (U : X.affineOpens)
(s : Set (X.presheaf.obj (op U.1))) (hs : Ideal.span s = ⊤)
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/AlgebraicGeometry/OpenImmersion/Scheme.lean
Original file line number Diff line number Diff line change
Expand Up @@ -1073,7 +1073,7 @@ def morphismRestrictEq {X Y : Scheme} (f : X ⟶ Y) {U V : Opens Y} (e : U = V)

-- Porting note : this does not compile under 200000 heart beats. The proof is more or less
-- preserved with some morphisms named so that instances about them can be made manually.
set_option maxHeartbeats 350000 in
set_option maxHeartbeats 300000 in
/-- Restricting a morphism twice is isomorphic to one restriction. -/
def morphismRestrictRestrict {X Y : Scheme} (f : X ⟶ Y) (U : Opens Y) (V : Opens U) :
Arrow.mk (f ∣_ U ∣_ V) ≅ Arrow.mk (f ∣_ U.openEmbedding.isOpenMap.functor.obj V) := by
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/AlgebraicGeometry/Properties.lean
Original file line number Diff line number Diff line change
Expand Up @@ -89,7 +89,7 @@ theorem isReducedOfOpenImmersion {X Y : Scheme} (f : X ⟶ Y) [H : IsOpenImmersi
Y.presheaf.obj _ ≅ _).symm.commRingCatIsoToRingEquiv.injective
#align algebraic_geometry.is_reduced_of_open_immersion AlgebraicGeometry.isReducedOfOpenImmersion

set_option maxHeartbeats 300000 in
set_option maxHeartbeats 250000 in
instance {R : CommRingCat} [H : _root_.IsReduced R] : IsReduced (Scheme.Spec.obj <| op R) := by
apply (config := { allowSynthFailures := true }) isReducedOfStalkIsReduced
intro x; dsimp
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
3 changes: 1 addition & 2 deletions Mathlib/Analysis/Calculus/ContDiff.lean
Original file line number Diff line number Diff line change
Expand Up @@ -2345,7 +2345,7 @@ theorem ContinuousLinearMap.norm_iteratedFDerivWithin_le_of_bilinear_aux {Du Eu
(fun i j => ‖iteratedFDerivWithin 𝕜 i f s x‖ * ‖iteratedFDerivWithin 𝕜 j g s x‖) n).symm
#align continuous_linear_map.norm_iterated_fderiv_within_le_of_bilinear_aux ContinuousLinearMap.norm_iteratedFDerivWithin_le_of_bilinear_aux

set_option maxHeartbeats 900000 in -- 4.5× the default limit
set_option maxHeartbeats 700000 in -- 3.5× the default limit
/-- Bounding the norm of the iterated derivative of `B (f x) (g x)` within a set in terms of the
iterated derivatives of `f` and `g` when `B` is bilinear:
`‖D^n (x ↦ B (f x) (g x))‖ ≤ ‖B‖ ∑_{k ≤ n} n.choose k ‖D^k f‖ ‖D^{n-k} g‖` -/
Expand Down 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
2 changes: 1 addition & 1 deletion Mathlib/Analysis/Convolution.lean
Original file line number Diff line number Diff line change
Expand Up @@ -1198,7 +1198,7 @@ variable [IsROrC 𝕜] [NormedSpace 𝕜 E] [NormedSpace 𝕜 E'] [NormedSpace
(L : E →L[𝕜] E' →L[𝕜] F)

-- porting note: the lemma is slow, added `set_option maxHeartbeats 300000 in`
set_option maxHeartbeats 300000 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 @@ -222,7 +222,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
1 change: 0 additions & 1 deletion Mathlib/Analysis/InnerProductSpace/Spectrum.lean
Original file line number Diff line number Diff line change
Expand Up @@ -139,7 +139,6 @@ theorem 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
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 @@ -819,8 +819,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 @@ -836,21 +834,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 @@ -871,7 +866,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 @@ -1017,7 +1011,7 @@ variable (M₁ : Type u₁) [SeminormedAddCommGroup M₁] [NormedSpace 𝕜 M₁

variable {Eₗ} (𝕜)

set_option maxHeartbeats 750000 in
set_option maxHeartbeats 500000 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 @@ -253,8 +253,6 @@ theorem elementalStarAlgebra.bijective_characterSpaceToSpectrum :
exact ⟨φ, rfl⟩
#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
/-- 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 :
Expand All @@ -265,8 +263,6 @@ noncomputable def elementalStarAlgebra.characterSpaceHomeo :
(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
/-- **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
2 changes: 1 addition & 1 deletion Mathlib/Combinatorics/SimpleGraph/Regularity/Chunk.lean
Original file line number Diff line number Diff line change
Expand Up @@ -470,7 +470,7 @@ private theorem edgeDensity_star_not_uniform [Nonempty α]
left; linarith
right; linarith

set_option maxHeartbeats 350000 in
set_option maxHeartbeats 300000 in
/-- Lower bound on the edge densities between non-uniform parts of `SzemerediRegularity.increment`.
-/
theorem edgeDensity_chunk_not_uniform [Nonempty α] (hPα : P.parts.card * 16 ^ P.parts.card ≤ card α)
Expand Down
Loading
Loading