mathlib3
f15389d9 - feat(linear_algebra/basis): add basis.ext_elem_iff (#18155)

Commit
2 years ago
feat(linear_algebra/basis): add basis.ext_elem_iff (#18155) Replace the lemma ```lean theorem basis.ext_elem (b : basis ι R M) {x y : M} (h : ∀ i, b.repr x i = b.repr y i) : x = y := ``` by an `iff` version: ```lean theorem basis.ext_elem_iff (b : basis ι R M) {x y : M} : x = y ↔ ∀ i, b.repr x i = b.repr y i := ```
Author
Parents
Loading