Skip to content

Commit

Permalink
address comments
Browse files Browse the repository at this point in the history
  • Loading branch information
erdOne committed Jan 6, 2025
1 parent 9f5ff59 commit 8b7fa3b
Show file tree
Hide file tree
Showing 2 changed files with 3 additions and 2 deletions.
3 changes: 2 additions & 1 deletion Mathlib/RingTheory/Kaehler/CotangentComplex.lean
Original file line number Diff line number Diff line change
Expand Up @@ -353,7 +353,8 @@ lemma H1Cotangent.map_comp
map (g.comp f) = (map g).restrictScalars S ∘ₗ map f := by
ext; simp [Cotangent.map_comp]

/-- Maps `P₁ → P₂` and `P₂ → P₁` between extensions induce an isomorphism of `H¹(L)`. -/
/-- Maps `P₁ → P₂` and `P₂ → P₁` between extensions
induce an isomorphism between `H¹(L_P₁)` and `H¹(L_P₂)`. -/
@[simps! apply]
noncomputable
def H1Cotangent.equiv {P₁ P₂ : Extension R S} (f₁ : P₁.Hom P₂) (f₂ : P₂.Hom P₁) :
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/RingTheory/Smooth/Kaehler.lean
Original file line number Diff line number Diff line change
Expand Up @@ -527,7 +527,7 @@ def homInfinitesimal (P₁ P₂ : Extension R S) [FormallySmooth R P₁.Ring] :
exact FormallySmooth.liftOfSurjective_apply _
(IsScalarTower.toAlgHom R P₂.infinitesimal.Ring S) _ _ x }

/-- Formally smooth extensions have isomorphic `H¹(L)`. -/
/-- Formally smooth extensions have isomorphic `H¹(L_P)`. -/
noncomputable
def H1Cotangent.equivOfFormallySmooth (P₁ P₂ : Extension R S)
[FormallySmooth R P₁.Ring] [FormallySmooth R P₂.Ring] :
Expand Down

0 comments on commit 8b7fa3b

Please sign in to comment.