refactor: Lint

This commit is contained in:
jstoobysmith 2024-12-20 13:34:49 +00:00
parent a5e0f3ceac
commit e4dafbd291
5 changed files with 9 additions and 9 deletions

View file

@ -24,7 +24,8 @@ open FieldStatistic
is zero.
This can be thought as as a condtion on the operator algebra `A` as much as it can
on `F`. -/
class OperatorMap {A : Type} [Semiring A] [Algebra A] (q : I → FieldStatistic) (le1 : I → I → Prop)
class OperatorMap {A : Type} [Semiring A] [Algebra A]
(q : I → FieldStatistic) (le1 : I → I → Prop)
[DecidableRel le1] (F : FreeAlgebra I →ₐ[] A) : Prop where
superCommute_mem_center : ∀ i j, F (superCommute q (FreeAlgebra.ι i) (FreeAlgebra.ι j)) ∈
Subalgebra.center A
@ -255,7 +256,8 @@ lemma le_all_mul_koszulOrder_ofList_expand {I : Type}
exact fun j => hi j
lemma le_all_mul_koszulOrder_ofListLift_expand {I : Type} {f : I → Type} [∀ i, Fintype (f i)]
(q : I → FieldStatistic) (r : List I) (x : ) (le1 : (Σ i, f i) → (Σ i, f i) → Prop) [DecidableRel le1]
(q : I → FieldStatistic) (r : List I) (x : )
(le1 : (Σ i, f i) → (Σ i, f i) → Prop) [DecidableRel le1]
[IsTotal (Σ i, f i) le1] [IsTrans (Σ i, f i) le1]
(i : (Σ i, f i)) (hi : ∀ (j : (Σ i, f i)), le1 j i)
{A : Type} [Semiring A] [Algebra A]