Quadratic algebras : involution and norm. #
Let R be a commutative ring. We define:
QuadraticAlgebra.star: the quadratic involutionQuadraticAlgebra.norm: the norm
We prove :
QuadraticAlgebra.isUnit_iff_norm_isUnit:w : QuadraticAlgebra R a bis a unit iffw.normis a unit inR.QuadraticAlgebra.norm_mem_nonZero_divisors_iff:w : QuadraticAlgebra R a bisn't a zero divisor iffw.normisn't a zero divisor inR.If
Ris a field, and∀ r, r ^ 2 ≠ a + b * r, thenQuadraticAlgebra R a bis a field. `
The representative of the root in the quadratic algebra
Equations
- QuadraticAlgebra.omega = { re := 0, im := 1 }
 
Instances For
the canonical element ⟨0, 1⟩ in a quadratic algebra QuadraticAlgebra R a b.
Equations
- QuadraticAlgebra.termω = Lean.ParserDescr.node `QuadraticAlgebra.termω 1024 (Lean.ParserDescr.symbol "ω")
 
Instances For
The unique AlgHom from QuadraticAlgebra R a b to an R-algebra A,
constructed by replacing ω with the provided root.
Conversely, this associates to every algebra morphism QuadraticAlgebra R a b →ₐ[R] A
a value of ω in A.
Equations
- One or more equations did not get rendered due to their size.
 
Instances For
Conjugation in QuadraticAlgebra R a b.
The conjugate of x + y ω is x + y ω' = (x - a * y) - y ω.
Equations
- QuadraticAlgebra.instStarRing = { toStar := QuadraticAlgebra.instStar, star_involutive := ⋯, star_mul := ⋯, star_add := ⋯ }
 
An element of QuadraticAlgebra R a b has norm equal to 1
if and only if it is contained in the submonoid of unitary elements.
Alias of the forward direction of QuadraticAlgebra.norm_eq_one_iff_mem_unitary.
An element of QuadraticAlgebra R a b has norm equal to 1
if and only if it is contained in the submonoid of unitary elements.
Alias of the reverse direction of QuadraticAlgebra.norm_eq_one_iff_mem_unitary.
An element of QuadraticAlgebra R a b has norm equal to 1
if and only if it is contained in the submonoid of unitary elements.
The kernel of the norm map on QuadraticAlgebra R a b equals
the submonoid of unitary elements.
If R is a field and there is no r : R such that r ^ 2 = a + b * r,
then QuadraticAlgebra R a b is a field.
Equations
- One or more equations did not get rendered due to their size.