refactor: Lint
This commit is contained in:
parent
cd63ec0716
commit
c739a5eeb8
3 changed files with 5 additions and 4 deletions
|
@ -99,13 +99,13 @@ def ofListLift {I : Type} (f : I → Type) [∀ i, Fintype (f i)] (l : List I) (
|
|||
sumFiber f (ofList l x)
|
||||
|
||||
lemma ofListLift_empty {I : Type} (f : I → Type) [∀ i, Fintype (f i)] :
|
||||
ofListLift f [] 1 = 1 := by
|
||||
ofListLift f [] 1 = 1 := by
|
||||
simp only [ofListLift, EmbeddingLike.map_eq_one_iff]
|
||||
rw [ofList_empty]
|
||||
exact map_one (sumFiber f)
|
||||
|
||||
lemma ofListLift_empty_smul {I : Type} (f : I → Type) [∀ i, Fintype (f i)] (x : ℂ) :
|
||||
ofListLift f [] x = x • 1 := by
|
||||
ofListLift f [] x = x • 1 := by
|
||||
simp only [ofListLift, EmbeddingLike.map_eq_one_iff]
|
||||
rw [ofList_eq_smul_one]
|
||||
rw [ofList_empty]
|
||||
|
|
Loading…
Add table
Add a link
Reference in a new issue