Documentation

BrauerGroup.MoritaEquivalence

instance instModuleMatrixForall_brauerGroup (R : Type u) [Ring R] (ι : Type w) [Fintype ι] [DecidableEq ι] (M : Type u_1) [AddCommGroup M] [Module R M] :
Module (Matrix ι ι R) (ιM)
Equations
theorem matrix_smul_vec_def (R : Type u) [Ring R] (ι : Type w) [Fintype ι] [DecidableEq ι] {M : Type u_1} [AddCommGroup M] [Module R M] (N : Matrix ι ι R) (v : ιM) :
N v = fun (i : ι) => j : ι, N i j v j
theorem matrix_smul_vec_def' (R : Type u) [Ring R] (ι : Type w) [Fintype ι] [DecidableEq ι] {M : Type u_1} [AddCommGroup M] [Module R M] (N : Matrix ι ι R) (v : ιM) :
N v = j : ι, fun (i : ι) => N i j v j
theorem matrix_smul_vec_apply (R : Type u) [Ring R] (ι : Type w) [Fintype ι] [DecidableEq ι] {M : Type u_1} [AddCommGroup M] [Module R M] (N : Matrix ι ι R) (v : ιM) (i : ι) :
(N v) i = j : ι, N i j v j
Equations
  • One or more equations did not get rendered due to their size.
Instances For
    @[simp]
    theorem toModuleCatOverMatrix_map_hom_apply (R : Type u) [Ring R] (ι : Type w) [Fintype ι] [DecidableEq ι] {X✝ Y✝ : ModuleCat R} (f : X✝ Y✝) (v : ιX✝) (i : ι) :
    ((toModuleCatOverMatrix R ι).map f).hom v i = f.hom (v i)
    @[simp]
    theorem toModuleCatOverMatrix_obj_isAddCommGroup (R : Type u) [Ring R] (ι : Type w) [Fintype ι] [DecidableEq ι] (M : ModuleCat R) :
    ((toModuleCatOverMatrix R ι).obj M).isAddCommGroup = Pi.addCommGroup
    @[simp]
    theorem toModuleCatOverMatrix_obj_carrier (R : Type u) [Ring R] (ι : Type w) [Fintype ι] [DecidableEq ι] (M : ModuleCat R) :
    ((toModuleCatOverMatrix R ι).obj M) = (ιM)
    @[simp]
    theorem toModuleCatOverMatrix_obj_isModule (R : Type u) [Ring R] (ι : Type w) [Fintype ι] [DecidableEq ι] (M : ModuleCat R) :
    def fromModuleCatOverMatrix.α (R : Type u) [Ring R] (ι : Type w) [Fintype ι] [DecidableEq ι] [Inhabited ι] (M : Type u_1) [AddCommGroup M] [Module (Matrix ι ι R) M] :
    Equations
    Instances For
      @[simp]
      theorem fromModuleCatOverMatrix.coe_α (R : Type u) [Ring R] (ι : Type w) [Fintype ι] [DecidableEq ι] [Inhabited ι] (M : Type u_1) [AddCommGroup M] [Module (Matrix ι ι R) M] :
      (α R ι M) = Set.range fun (x : M) => Matrix.stdBasisMatrix default default 1 x
      instance fromModuleCatOverMatrix.module_α (R : Type u) [Ring R] (ι : Type w) [Fintype ι] [Inhabited ι] [DecidableEq ι] (M : Type u_1) [AddCommGroup M] [Module (Matrix ι ι R) M] :
      Module R (α R ι M)
      Equations
      @[simp]
      theorem fromModuleCatOverMatrix.smul_α_coe (R : Type u) [Ring R] (ι : Type w) [Fintype ι] [Inhabited ι] [DecidableEq ι] {M : Type u_1} [AddCommGroup M] [Module (Matrix ι ι R) M] (x : R) (y : (α R ι M)) :
      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        @[simp]
        theorem fromModuleCatOverMatrix_obj_carrier (R : Type u) [Ring R] (ι : Type w) [Fintype ι] [Inhabited ι] [DecidableEq ι] (M : ModuleCat (Matrix ι ι R)) :
        ((fromModuleCatOverMatrix R ι).obj M) = (fromModuleCatOverMatrix.α R ι M)
        @[simp]
        theorem fromModuleCatOverMatrix_map_hom_apply_coe (R : Type u) [Ring R] (ι : Type w) [Fintype ι] [Inhabited ι] [DecidableEq ι] {X✝ Y✝ : ModuleCat (Matrix ι ι R)} (f : X✝ Y✝) (x : (fromModuleCatOverMatrix.α R ι X✝)) :
        (((fromModuleCatOverMatrix R ι).map f).hom x) = f.hom x
        @[simp]
        theorem fromModuleCatOverMatrix_obj_isModule (R : Type u) [Ring R] (ι : Type w) [Fintype ι] [Inhabited ι] [DecidableEq ι] (M : ModuleCat (Matrix ι ι R)) :
        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          @[simp]
          theorem matrix.unitIsoHom_app_hom_apply (R : Type u) [Ring R] (ι : Type w) [Fintype ι] [Inhabited ι] [DecidableEq ι] (X : ModuleCat R) (x : (fromModuleCatOverMatrix.α R ι ((toModuleCatOverMatrix R ι).obj X))) :
          ((unitIsoHom R ι).app X).hom x = i : ι, x i
          Equations
          • One or more equations did not get rendered due to their size.
          Instances For
            @[simp]
            theorem matrix.unitIsoInv_app_hom_apply_coe (R : Type u) [Ring R] (ι : Type w) [Fintype ι] [Inhabited ι] [DecidableEq ι] (X : ModuleCat R) (x : X) (a : ι) :
            (((unitIsoInv R ι).app X).hom x) a = Function.update 0 default x a
            Equations
            Instances For
              @[simp]
              theorem matrix.unitIso_inv (R : Type u) [Ring R] (ι : Type w) [Fintype ι] [Inhabited ι] [DecidableEq ι] :
              (unitIso R ι).inv = unitIsoInv R ι
              @[simp]
              theorem matrix.unitIso_hom (R : Type u) [Ring R] (ι : Type w) [Fintype ι] [Inhabited ι] [DecidableEq ι] :
              (unitIso R ι).hom = unitIsoHom R ι
              noncomputable def matrix.counitIsoHomMap (R : Type u) [Ring R] (ι : Type w) [Fintype ι] [Inhabited ι] [DecidableEq ι] (M : ModuleCat (Matrix ι ι R)) :
              Equations
              Instances For
                @[simp]
                theorem matrix.counitIsoHomMap_hom_hom_apply_coe (R : Type u) [Ring R] (ι : Type w) [Fintype ι] [Inhabited ι] [DecidableEq ι] (M : ModuleCat (Matrix ι ι R)) (a✝ : M) (a✝¹ : ι) :
                ((counitIsoHomMap R ι M).hom.hom a✝ a✝¹) = Matrix.stdBasisMatrix default a✝¹ 1 a✝
                @[simp]
                theorem matrix.counitIsoHomMap_inv_hom_apply (R : Type u) [Ring R] (ι : Type w) [Fintype ι] [Inhabited ι] [DecidableEq ι] (M : ModuleCat (Matrix ι ι R)) (a : ι((fromModuleCatOverMatrix R ι).obj M)) :
                (counitIsoHomMap R ι M).inv.hom a = ((↑(LinearEquiv.ofBijective { toFun := fun (m : M) (i : ι) => Matrix.stdBasisMatrix default i 1 m, , map_add' := , map_smul' := } )).inverse (LinearEquiv.ofBijective { toFun := fun (m : M) (i : ι) => Matrix.stdBasisMatrix default i 1 m, , map_add' := , map_smul' := } ).symm ) a
                noncomputable def matrix.counitIsoHom (R : Type u) [Ring R] (ι : Type w) [Fintype ι] [Inhabited ι] [DecidableEq ι] :
                Equations
                Instances For
                  @[simp]
                  theorem matrix.counitIsoHom_app (R : Type u) [Ring R] (ι : Type w) [Fintype ι] [Inhabited ι] [DecidableEq ι] (M : ModuleCat (Matrix ι ι R)) :
                  (counitIsoHom R ι).app M = (counitIsoHomMap R ι M).inv
                  noncomputable def matrix.counitIsoInv (R : Type u) [Ring R] (ι : Type w) [Fintype ι] [Inhabited ι] [DecidableEq ι] :
                  Equations
                  Instances For
                    @[simp]
                    theorem matrix.counitIsoInv_app (R : Type u) [Ring R] (ι : Type w) [Fintype ι] [Inhabited ι] [DecidableEq ι] (M : ModuleCat (Matrix ι ι R)) :
                    (counitIsoInv R ι).app M = (counitIsoHomMap R ι M).hom
                    noncomputable def matrix.counitIso (R : Type u) [Ring R] (ι : Type w) [Fintype ι] [Inhabited ι] [DecidableEq ι] :
                    Equations
                    Instances For
                      @[simp]
                      theorem matrix.counitIso_inv (R : Type u) [Ring R] (ι : Type w) [Fintype ι] [Inhabited ι] [DecidableEq ι] :
                      (counitIso R ι).inv = counitIsoInv R ι
                      @[simp]
                      theorem matrix.counitIso_hom (R : Type u) [Ring R] (ι : Type w) [Fintype ι] [Inhabited ι] [DecidableEq ι] :
                      (counitIso R ι).hom = counitIsoHom R ι
                      noncomputable def moritaEquivalentToMatrix (R : Type u) [Ring R] (ι : Type w) [Fintype ι] [Inhabited ι] [DecidableEq ι] :
                      Equations
                      • One or more equations did not get rendered due to their size.
                      Instances For
                        @[simp]
                        theorem moritaEquivalentToMatrix_unitIso (R : Type u) [Ring R] (ι : Type w) [Fintype ι] [Inhabited ι] [DecidableEq ι] :
                        (moritaEquivalentToMatrix R ι).unitIso = (matrix.unitIso R ι).symm
                        @[simp]
                        @[simp]
                        theorem moritaEquivalentToMatrix_counitIso (R : Type u) [Ring R] (ι : Type w) [Fintype ι] [Inhabited ι] [DecidableEq ι] :
                        class IsMoritaEquivalent (R : Type u) (S : Type u') [Ring R] [Ring S] :
                        Instances
                          noncomputable def IsMoritaEquivalent.equiv (R : Type u) (S : Type u') [Ring R] [Ring S] [IsMoritaEquivalent R S] :
                          Equations
                          Instances For
                            instance IsMoritaEquivalent.instAdditiveModuleCatFunctorEquiv (R : Type u) (S : Type u') [Ring R] [Ring S] [IsMoritaEquivalent R S] :
                            (equiv R S).functor.Additive
                            instance IsMoritaEquivalent.instAdditiveModuleCatInverseEquiv (R : Type u) (S : Type u') [Ring R] [Ring S] [IsMoritaEquivalent R S] :
                            (equiv R S).inverse.Additive
                            theorem IsMoritaEquivalent.trans (R : Type u) (S : Type u') (T : Type u'') [Ring R] [Ring S] [Ring T] [IsMoritaEquivalent R S] [IsMoritaEquivalent S T] :
                            instance IsMoritaEquivalent.matrix (R : Type u) [Ring R] (n : ) :
                            IsMoritaEquivalent R (Matrix (Fin (n + 1)) (Fin (n + 1)) R)
                            theorem IsMoritaEquivalent.matrix' (R : Type u) [Ring R] (n : ) [hn : NeZero n] :
                            @[reducible, inline]
                            abbrev IsMoritaEquivalent.ofIsoApp1 (R : Type u) (S : Type u') [Ring R] [Ring S] (e : R ≃+* S) (X : ModuleCat R) :
                            X ((ModuleCat.restrictScalars e.symm.toRingHom).comp (ModuleCat.restrictScalars e.toRingHom)).obj X
                            Equations
                            Instances For
                              @[reducible, inline]
                              abbrev IsMoritaEquivalent.ofIsoApp2 (R : Type u) (S : Type u') [Ring R] [Ring S] (e : R ≃+* S) (X : ModuleCat R) :
                              ((ModuleCat.restrictScalars e.symm.toRingHom).comp (ModuleCat.restrictScalars e.toRingHom)).obj X X
                              Equations
                              Instances For
                                theorem IsMoritaEquivalent.ofIso (R : Type u) (S : Type u') [Ring R] [Ring S] (e : R ≃+* S) :
                                instance CategoryTheory.Equivalence.nontrivial {R S : Type u} [Ring R] [Ring S] (e : ModuleCat R ModuleCat S) (M : ModuleCat R) [h : Nontrivial M] :
                                Nontrivial (e.functor.obj M)
                                theorem IsMoritaEquivalent.division_ring.IsSimpleModule.functor (R S : Type u) [Ring R] [Ring S] (e : ModuleCat R ModuleCat S) (M : ModuleCat R) [simple_module : IsSimpleModule R M] :
                                IsSimpleModule S (e.functor.obj M)
                                Equations
                                • One or more equations did not get rendered due to their size.
                                Instances For
                                  Equations
                                  • One or more equations did not get rendered due to their size.
                                  Instances For
                                    noncomputable def IsMoritaEquivalent.division_ring.aux20 (R S : Type u) [DivisionRing R] [DivisionRing S] (e : ModuleCat R ModuleCat S) :
                                    e.functor.obj (ModuleCat.of R R) ModuleCat.of S S
                                    Equations
                                    Instances For
                                      Equations
                                      • One or more equations did not get rendered due to their size.
                                      Instances For
                                        Equations
                                        • One or more equations did not get rendered due to their size.
                                        Instances For
                                          Equations
                                          • One or more equations did not get rendered due to their size.
                                          Instances For