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

@ -167,7 +167,7 @@ lemma ofListLift_expand (f : 𝓕 → Type) [∀ i, Fintype (f i)] (x : ) :
lemma koszulOrder_ofListLift {f : 𝓕 → Type} [∀ i, Fintype (f i)]
(l : List 𝓕) (x : ) :
koszulOrder (fun i => q i.fst) (fun i j => le i.1 j.1) (ofListLift f l x) =
koszulOrder (fun i => q i.fst) (fun i j => le i.1 j.1) (ofListLift f l x) =
sumFiber f (koszulOrder q le (ofList l x)) := by
rw [koszulOrder_ofList]
rw [map_smul]