Skip to content

Commit

Permalink
feat: port RingTheory.Kaehler (#4668)
Browse files Browse the repository at this point in the history
Co-authored-by: ART <anand.rao.art@gmail.com>
Co-authored-by: Xavier-François Roblot <46200072+xroblot@users.noreply.github.com>
Co-authored-by: Bulhwi Cha <chabulhwi@semmalgil.com>
Co-authored-by: Kevin Buzzard <k.buzzard@imperial.ac.uk>
Co-authored-by: Matthew Ballard <matt@mrb.email>
Co-authored-by: Kyle Miller <kmill31415@gmail.com>
Co-authored-by: Parcly Taxel <reddeloostw@gmail.com>
Co-authored-by: Scott Morrison <scott.morrison@gmail.com>
  • Loading branch information
9 people committed Jul 8, 2023
1 parent adca8e2 commit a3b66ec
Show file tree
Hide file tree
Showing 3 changed files with 698 additions and 1 deletion.
1 change: 1 addition & 0 deletions Mathlib.lean
Expand Up @@ -2725,6 +2725,7 @@ import Mathlib.RingTheory.IsAdjoinRoot
import Mathlib.RingTheory.IsTensorProduct
import Mathlib.RingTheory.Jacobson
import Mathlib.RingTheory.JacobsonIdeal
import Mathlib.RingTheory.Kaehler
import Mathlib.RingTheory.LaurentSeries
import Mathlib.RingTheory.LocalProperties
import Mathlib.RingTheory.Localization.AsSubring
Expand Down
3 changes: 2 additions & 1 deletion Mathlib/RingTheory/Ideal/Cotangent.lean
Expand Up @@ -50,13 +50,14 @@ instance Cotangent.moduleOfTower : Module S I.Cotangent :=
Submodule.Quotient.module' _
#align ideal.cotangent.module_of_tower Ideal.Cotangent.moduleOfTower

instance : IsScalarTower S S' I.Cotangent := by
instance Cotangent.isScalarTower : IsScalarTower S S' I.Cotangent := by
delta Cotangent
constructor
intro s s' x
rw [← @IsScalarTower.algebraMap_smul S' R, ← @IsScalarTower.algebraMap_smul S' R, ← smul_assoc, ←
IsScalarTower.toAlgHom_apply S S' R, map_smul]
rfl
#align ideal.cotangent.is_scalar_tower Ideal.Cotangent.isScalarTower

instance [IsNoetherian R I] : IsNoetherian R I.Cotangent := by delta Cotangent; infer_instance

Expand Down

0 comments on commit a3b66ec

Please sign in to comment.