Unitary elements of a star monoid #
This file defines unitary R, where R is a star monoid, as the submonoid made of the elements
that satisfy star U * U = 1 and U * star U = 1, and these form a group.
This includes, for instance, unitary operators on Hilbert spaces.
See also Matrix.UnitaryGroup for specializations to unitary (Matrix n n R).
Tags #
unitary
In a *-monoid, unitary R is the submonoid consisting of all the elements U of
R such that star U * U = 1 and U * star U = 1.
Equations
Instances For
Equations
- Unitary.instInvolutiveStarSubtypeMemSubmonoidUnitary = { toStar := Unitary.instStarSubtypeMemSubmonoidUnitary, star_involutive := ⋯ }
Equations
- Unitary.instStarMulSubtypeMemSubmonoidUnitary = { toInvolutiveStar := Unitary.instInvolutiveStarSubtypeMemSubmonoidUnitary, star_mul := ⋯ }
unitary as a Subgroup of a group.
Note the group structure on this type is not defeq to the one on unitary.
This situation naturally arises when considering the unitary elements as a
subgroup of the group of units of a star monoid.
Equations
- unitarySubgroup G = { toSubmonoid := unitary G, inv_mem' := ⋯ }
Instances For
Equations
- Unitary.instMulActionSubtypeMemSubmonoidUnitary = { toSMul := Unitary.instSMulSubtypeMemSubmonoidUnitary, one_smul := ⋯, mul_smul := ⋯ }
The star monoid homomorphism between unitary subgroups induced by a star monoid homomorphism of the underlying star monoids.
Equations
- Unitary.map f = { toFun := Subtype.map ⇑f ⋯, map_one' := ⋯, map_mul' := ⋯, map_star' := ⋯ }
Instances For
The star monoid isomorphism between unitary subgroups induced by a star monoid isomorphism of the underlying star monoids.
Equations
- Unitary.mapEquiv f = { toFun := ⇑(Unitary.map f.toStarMonoidHom), invFun := ⇑(Unitary.map f.symm.toStarMonoidHom), left_inv := ⋯, right_inv := ⋯, map_mul' := ⋯, map_star' := ⋯ }
Instances For
The unitary subgroup of the units is equivalent to the unitary elements of the monoid.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Unitary.instCommGroupSubtypeMemSubmonoidUnitary = { toGroup := inferInstanceAs (Group ↥(unitary R)), mul_comm := ⋯ }
Equations
- Unitary.instHasDistribNegSubtypeMemSubmonoidUnitary = Function.Injective.hasDistribNeg (fun (a : ↥(unitary R)) => ↑a) ⋯ ⋯ ⋯
Deprecated results #
Alias of Unitary.coe_star.
Alias of Unitary.coe_star_mul_self.
Alias of Unitary.coe_mul_star_self.
Alias of Unitary.star_mul_self.
Alias of Unitary.mul_star_self.
Alias of Unitary.star_eq_inv.
Alias of Unitary.star_eq_inv'.
Alias of Unitary.toUnits.
The unitary elements embed into the units.
Equations
Instances For
Alias of Unitary.val_toUnits_apply.
Alias of Unitary.toUnits_injective.
Alias of Unitary.mul_left_inj.
For unitary U in a star-monoid R, x * U = y * U if and only if x = y
for all x and y in R.
Alias of Unitary.mul_right_inj.
For unitary U in a star-monoid R, U * x = U * y if and only if x = y
for all x and y in R.
Alias of Unitary.smul_mem_of_mem.
Alias of Unitary.smul_mem.
Alias of Unitary.coe_smul.
Alias of Unitary.map_mem.
Alias of Unitary.map.
The star monoid homomorphism between unitary subgroups induced by a star monoid homomorphism of the underlying star monoids.
Equations
Instances For
Alias of Unitary.coe_map.
Alias of Unitary.coe_map_star.
Alias of Unitary.map_id.
Alias of Unitary.map_injective.
Alias of Unitary.toUnits_comp_map.
Alias of Unitary.mapEquiv.
The star monoid isomorphism between unitary subgroups induced by a star monoid isomorphism of the underlying star monoids.
Equations
Instances For
Alias of Unitary.mapEquiv_refl.
Alias of Unitary.mapEquiv_symm.
Alias of Unitary.toMonoidHom_mapEquiv.
Alias of Unitary.mem_iff_star_mul_self.
Alias of Unitary.mem_iff_self_mul_star.
Alias of Unitary.coe_inv.
Alias of Unitary.coe_div.
Alias of Unitary.coe_zpow.
Alias of Unitary.coe_neg.
Alias of Unitary.spectrum_star_right_conjugate.
Unitary conjugation preserves the spectrum, star on right.
Alias of Unitary.spectrum_star_left_conjugate.
Unitary conjugation preserves the spectrum, star on left.