Isomorphisms of R
-coalgebras #
This file defines bundled isomorphisms of R
-coalgebras. We simply mimic the early parts of
Mathlib/Algebra/Module/Equiv.lean
.
Main definitions #
CoalgEquiv R A B
: the type ofR
-coalgebra isomorphisms betweenA
andB
.
Notations #
A ≃ₗc[R] B
:R
-coalgebra equivalence fromA
toB
.
An equivalence of coalgebras is an invertible coalgebra homomorphism.
- toFun : A → B
- map_smul' : ∀ (m : R) (x : A), self.toFun (m • x) = (RingHom.id R) m • self.toFun x
- counit_comp : Coalgebra.counit ∘ₗ self.toLinearMap = Coalgebra.counit
- map_comp_comul : TensorProduct.map self.toLinearMap self.toLinearMap ∘ₗ Coalgebra.comul = Coalgebra.comul ∘ₗ self.toLinearMap
- invFun : B → A
- left_inv : Function.LeftInverse self.invFun self.toFun
- right_inv : Function.RightInverse self.invFun self.toFun
Instances For
An equivalence of coalgebras is an invertible coalgebra homomorphism.
Equations
- One or more equations did not get rendered due to their size.
Instances For
CoalgEquivClass F R A B
asserts F
is a type of bundled coalgebra equivalences
from A
to B
.
- map_smulₛₗ : ∀ (f : F) (c : R) (x : A), f (c • x) = (RingHom.id R) c • f x
- counit_comp : ∀ (f : F), Coalgebra.counit ∘ₗ ↑f = Coalgebra.counit
- map_comp_comul : ∀ (f : F), TensorProduct.map ↑f ↑f ∘ₗ Coalgebra.comul = Coalgebra.comul ∘ₗ ↑f
Instances
Reinterpret an element of a type of coalgebra equivalences as a coalgebra equivalence.
Equations
- ↑f = { toCoalgHom := ↑f, invFun := (↑f).invFun, left_inv := ⋯, right_inv := ⋯ }
Instances For
Reinterpret an element of a type of coalgebra equivalences as a coalgebra equivalence.
Equations
- CoalgEquivClass.instCoeToCoalgEquiv = { coe := fun (f : F) => ↑f }
The equivalence of types underlying a coalgebra equivalence.
Equations
- f.toEquiv = f.toLinearEquiv.toEquiv
Instances For
Equations
- CoalgEquiv.instFunLike = { coe := DFunLike.coe, coe_injective' := ⋯ }
Equations
- ⋯ = ⋯
See Note [custom simps projection]
Equations
- CoalgEquiv.Simps.apply f = ⇑f
Instances For
The identity map is a coalgebra equivalence.
Equations
- CoalgEquiv.refl R A = { toCoalgHom := CoalgHom.id R A, invFun := (LinearEquiv.refl R A).invFun, left_inv := ⋯, right_inv := ⋯ }
Instances For
Coalgebra equivalences are symmetric.
Equations
- e.symm = { toLinearMap := ↑(↑e).symm, counit_comp := ⋯, map_comp_comul := ⋯, invFun := (↑e).symm.invFun, left_inv := ⋯, right_inv := ⋯ }
Instances For
See Note [custom simps projection]
Equations
- CoalgEquiv.Simps.symm_apply e = ⇑e.symm
Instances For
Coalgebra equivalences are transitive.
Equations
- e₁₂.trans e₂₃ = { toCoalgHom := (↑e₂₃).comp ↑e₁₂, invFun := (e₁₂.toLinearEquiv.trans e₂₃.toLinearEquiv).invFun, left_inv := ⋯, right_inv := ⋯ }
Instances For
Let A
be an R
-coalgebra and let B
be an R
-module with a CoalgebraStruct
.
A linear equivalence A ≃ₗ[R] B
that respects the CoalgebraStruct
s defines an R
-coalgebra
structure on B
.
Equations
- f.toCoalgebra = Coalgebra.mk ⋯ ⋯ ⋯