refactor: Lint
This commit is contained in:
parent
ee2134e448
commit
e4c6da1cd6
12 changed files with 30 additions and 38 deletions
|
@ -40,7 +40,6 @@ abbrev FieldOpFreeAlgebra (𝓕 : FieldSpecification) : Type := FreeAlgebra ℂ
|
|||
|
||||
namespace FieldOpFreeAlgebra
|
||||
|
||||
|
||||
remark naming_convention := "
|
||||
For mathematicial objects defined in relation to `FieldOpFreeAlgebra` we will often postfix
|
||||
their names with an `F` to indicate that they are related to the free algebra.
|
||||
|
@ -62,7 +61,7 @@ The algebra `𝓕.FieldOpFreeAlgebra` satisfies the universal property that for
|
|||
The unique `g` is given by `FreeAlgebra.lift ℂ f`.
|
||||
-/
|
||||
lemma universality {A : Type} [Semiring A] [Algebra ℂ A] (f : 𝓕.CrAnFieldOp → A) :
|
||||
∃! g : FieldOpFreeAlgebra 𝓕 →ₐ[ℂ] A, g ∘ ofCrAnOpF = f := by
|
||||
∃! g : FieldOpFreeAlgebra 𝓕 →ₐ[ℂ] A, g ∘ ofCrAnOpF = f := by
|
||||
use FreeAlgebra.lift ℂ f
|
||||
apply And.intro
|
||||
· funext x
|
||||
|
|
Loading…
Add table
Add a link
Reference in a new issue