Isomorphisms of R
-bialgebras #
This file defines bundled isomorphisms of R
-bialgebras. We simply mimic the early parts of
Mathlib/Algebra/Algebra/Equiv.lean
.
Main definitions #
BialgEquiv R A B
: the type ofR
-bialgebra isomorphisms betweenA
andB
.
Notations #
A ≃ₐc[R] B
:R
-bialgebra equivalence fromA
toB
.
An equivalence of bialgebras is an invertible bialgebra 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 bialgebras is an invertible bialgebra homomorphism.
Equations
- One or more equations did not get rendered due to their size.
Instances For
BialgEquivClass F R A B
asserts F
is a type of bundled bialgebra 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
Equations
- ⋯ = ⋯
Reinterpret an element of a type of bialgebra equivalences as a bialgebra equivalence.
Equations
- ↑f = { toCoalgEquiv := ↑f, map_mul' := ⋯ }
Instances For
Reinterpret an element of a type of bialgebra equivalences as a bialgebra equivalence.
Equations
- BialgEquivClass.instCoeToBialgEquiv = { coe := fun (f : F) => ↑f }
Equations
- ⋯ = ⋯
The bialgebra morphism underlying a bialgebra equivalence.
Equations
- f.toBialgHom = { toCoalgHom := f.toCoalgHom, map_one' := ⋯, map_mul' := ⋯ }
Instances For
The algebra equivalence underlying a bialgebra equivalence.
Equations
- f.toAlgEquiv = { toFun := f.toFun, invFun := f.invFun, left_inv := ⋯, right_inv := ⋯, map_mul' := ⋯, map_add' := ⋯, commutes' := ⋯ }
Instances For
The equivalence of types underlying a bialgebra equivalence.
Equations
- f.toEquiv = f.toEquiv
Instances For
Equations
- BialgEquiv.instFunLike = { coe := DFunLike.coe, coe_injective' := ⋯ }
Equations
- ⋯ = ⋯
See Note [custom simps projection]
Equations
- BialgEquiv.Simps.apply f = ⇑f
Instances For
The identity map is a bialgebra equivalence.
Equations
- BialgEquiv.refl R A = { toCoalgEquiv := CoalgEquiv.refl R A, map_mul' := ⋯ }
Instances For
Bialgebra equivalences are symmetric.
Equations
- e.symm = { toCoalgEquiv := (↑e).symm, map_mul' := ⋯ }
Instances For
See Note [custom simps projection]
Equations
- BialgEquiv.Simps.symm_apply e = ⇑e.symm
Instances For
Bialgebra equivalences are transitive.
Equations
- e₁₂.trans e₂₃ = { toCoalgEquiv := (↑e₁₂).trans ↑e₂₃, map_mul' := ⋯ }