Transfer algebraic structures across Equiv
s #
This continues the pattern set in Mathlib/Algebra/Group/TransferInstance.lean
.
@[reducible, inline]
abbrev
Equiv.algebra
(R : Type u_1)
{α : Type u_2}
{β : Type u_3}
[CommSemiring R]
(e : α ≃ β)
[Semiring β]
:
Transfer Algebra
across an Equiv
Equations
- @Equiv.algebra R α β inst✝¹ e inst✝ = fun [Algebra R β] => Algebra.ofModule ⋯ ⋯
Instances For
theorem
Equiv.algebraMap_def
{R : Type u_1}
{α : Type u_2}
{β : Type u_3}
[CommSemiring R]
(e : α ≃ β)
[Semiring β]
[Algebra R β]
(r : R)
:
def
Equiv.algEquiv
(R : Type u_1)
{α : Type u_2}
{β : Type u_3}
[CommSemiring R]
(e : α ≃ β)
[Semiring β]
[Algebra R β]
:
let semiring := e.semiring;
have algebra := Equiv.algebra R e;
α ≃ₐ[R] β
An equivalence e : α ≃ β
gives an algebra equivalence α ≃ₐ[R] β
where the R
-algebra structure on α
is
the one obtained by transporting an R
-algebra structure on β
back along e
.
Equations
Instances For
theorem
Equiv.algEquiv_symm_apply
{R : Type u_1}
{α : Type u_2}
{β : Type u_3}
[CommSemiring R]
(e : α ≃ β)
[Semiring β]
[Algebra R β]
(b : β)
: