refactor: Lint

This commit is contained in:
jstoobysmith 2025-02-06 13:31:59 +00:00
parent ee2134e448
commit e4c6da1cd6
12 changed files with 30 additions and 38 deletions

View file

@ -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