Results #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
derivation_to_square_zero_equiv_lift
: TheR
-derivations fromA
into a square-zero idealI
ofB
corresponds to the liftsA →ₐ[R] B
of the mapA →ₐ[R] B ⧸ I
.
If f₁ f₂ : A →ₐ[R] B
are two lifts of the same A →ₐ[R] B ⧸ I
,
we may define a map f₁ - f₂ : A →ₗ[R] I
.
Equations
- diff_to_ideal_of_quotient_comp_eq I f₁ f₂ e = linear_map.cod_restrict (submodule.restrict_scalars R I) (f₁.to_linear_map - f₂.to_linear_map) _
Given a tower of algebras R → A → B
, and a square-zero I : ideal B
, each lift A →ₐ[R] B
of the canonical map A →ₐ[R] B ⧸ I
corresponds to a R
-derivation from A
to I
.
Equations
- derivation_to_square_zero_of_lift I hI f e = {to_linear_map := {to_fun := (diff_to_ideal_of_quotient_comp_eq I f (is_scalar_tower.to_alg_hom R A B) _).to_fun, map_add' := _, map_smul' := _}, map_one_eq_zero' := _, leibniz' := _}
Given a tower of algebras R → A → B
, and a square-zero I : ideal B
, each R
-derivation
from A
to I
corresponds to a lift A →ₐ[R] B
of the canonical map A →ₐ[R] B ⧸ I
.
Given a tower of algebras R → A → B
, and a square-zero I : ideal B
,
there is a 1-1 correspondance between R
-derivations from A
to I
and
lifts A →ₐ[R] B
of the canonical map A →ₐ[R] B ⧸ I
.
Equations
- derivation_to_square_zero_equiv_lift I hI = {to_fun := λ (d : derivation R A ↥I), ⟨lift_of_derivation_to_square_zero I hI d, _⟩, inv_fun := λ (f : {f // (ideal.quotient.mkₐ R I).comp f = is_scalar_tower.to_alg_hom R A (B ⧸ I)}), derivation_to_square_zero_of_lift I hI f.val _, left_inv := _, right_inv := _}