Skip to content

Commit

Permalink
fix: avoid with in Finsupp.module (#6189)
Browse files Browse the repository at this point in the history
  • Loading branch information
kbuzzard committed Jul 28, 2023
1 parent 284442f commit d60c218
Show file tree
Hide file tree
Showing 3 changed files with 6 additions and 9 deletions.
3 changes: 1 addition & 2 deletions Mathlib/Data/Finsupp/Basic.lean
Expand Up @@ -1535,8 +1535,7 @@ instance isCentralScalar [Zero M] [SMulZeroClass R M] [SMulZeroClass Rᵐᵒᵖ
#align finsupp.is_central_scalar Finsupp.isCentralScalar

instance module [Semiring R] [AddCommMonoid M] [Module R M] : Module R (α →₀ M) :=
{ Finsupp.distribMulAction α M with
smul := (· • ·)
{ toDistribMulAction := Finsupp.distribMulAction α M
zero_smul := fun _ => ext fun _ => zero_smul _ _
add_smul := fun _ _ _ => ext fun _ => add_smul _ _ _ }
#align finsupp.module Finsupp.module
Expand Down
6 changes: 3 additions & 3 deletions Mathlib/RepresentationTheory/GroupCohomology/Basic.lean
Expand Up @@ -117,7 +117,7 @@ def d [Monoid G] (n : ℕ) (A : Rep k G) : ((Fin n → G) → A) →ₗ[k] (Fin
variable [Group G] (n) (A : Rep k G)

/- Porting note: linter says the statement doesn't typecheck, so we add `@[nolint checkType]` -/
set_option maxHeartbeats 1600000 in
set_option maxHeartbeats 800000 in
/-- The theorem that our isomorphism `Fun(Gⁿ, A) ≅ Hom(k[Gⁿ⁺¹], A)` (where the righthand side is
morphisms in `Rep k G`) commutes with the differentials in the complex of inhomogeneous cochains
and the homogeneous `linearYonedaObjResolution`. -/
Expand Down Expand Up @@ -172,7 +172,7 @@ variable [Group G] (n) (A : Rep k G)

open InhomogeneousCochains

set_option maxHeartbeats 6400000 in
set_option maxHeartbeats 3200000 in
/-- Given a `k`-linear `G`-representation `A`, this is the complex of inhomogeneous cochains
$$0 \to \mathrm{Fun}(G^0, A) \to \mathrm{Fun}(G^1, A) \to \mathrm{Fun}(G^2, A) \to \dots$$
which calculates the group cohomology of `A`. -/
Expand All @@ -199,7 +199,7 @@ noncomputable abbrev inhomogeneousCochains : CochainComplex (ModuleCat k) ℕ :=
exact map_zero _
#align group_cohomology.inhomogeneous_cochains GroupCohomology.inhomogeneousCochains

set_option maxHeartbeats 6400000 in
set_option maxHeartbeats 3200000 in
/-- Given a `k`-linear `G`-representation `A`, the complex of inhomogeneous cochains is isomorphic
to `Hom(P, A)`, where `P` is the standard resolution of `k` as a trivial `G`-representation. -/
def inhomogeneousCochainsIso : inhomogeneousCochains A ≅ linearYonedaObjResolution A := by
Expand Down
6 changes: 2 additions & 4 deletions Mathlib/RepresentationTheory/GroupCohomology/Resolution.lean
Expand Up @@ -342,7 +342,7 @@ theorem diagonalHomEquiv_apply (f : Rep.ofMulAction k G (Fin (n + 1) → G) ⟶
set_option linter.uppercaseLean3 false in
#align Rep.diagonal_hom_equiv_apply Rep.diagonalHomEquiv_apply

set_option maxHeartbeats 800000 in
set_option maxHeartbeats 400000 in
/-- Given a `k`-linear `G`-representation `A`, `diagonalHomEquiv` is a `k`-linear isomorphism of
the set of representation morphisms `Hom(k[Gⁿ⁺¹], A)` with `Fun(Gⁿ, A)`. This lemma says that the
inverse map sends a function `f : Gⁿ → A` to the representation morphism sending
Expand Down Expand Up @@ -701,9 +701,7 @@ def GroupCohomology.extIso (V : Rep k G) (n : ℕ) :
((Ext k (Rep k G) n).obj (Opposite.op <| Rep.trivial k G k)).obj V ≅
(((((linearYoneda k (Rep k G)).obj V).rightOp.mapHomologicalComplex _).obj
(GroupCohomology.resolution k G)).homology
n).unop := by
let E := (((linearYoneda k (Rep k G)).obj V).rightOp.leftDerivedObjIso n
n).unop := (((linearYoneda k (Rep k G)).obj V).rightOp.leftDerivedObjIso n
(GroupCohomology.projectiveResolution k G)).unop.symm
exact E
set_option linter.uppercaseLean3 false in
#align group_cohomology.Ext_iso GroupCohomology.extIso

0 comments on commit d60c218

Please sign in to comment.