refactor: Removing unneeded brackets

This commit is contained in:
jstoobysmith 2024-07-15 06:54:32 -04:00
parent e87156ddfd
commit e6c378603d
4 changed files with 10 additions and 5 deletions

View file

@ -601,7 +601,7 @@ lemma Pa'_eq (f f' : (Fin n.succ) ⊕ (Fin n.succ) → ) : Pa' f = Pa' f' ↔
rw [← Finset.sum_add_distrib]
simp
have h2 : ∀ i, (f i + (- f' i)) = 0 := by
exact Fintype.linearIndependent_iff.mp (@basisa_linear_independent (n))
exact Fintype.linearIndependent_iff.mp (@basisa_linear_independent n)
(fun i => f i + -f' i) h1
have h2i := h2 i
linarith