Skip to content

Commit

Permalink
feat(linear_algebra/finite_dimensional): add dim_sup_add_dim_inf_eq (#…
Browse files Browse the repository at this point in the history
…3304)

Adding a finite-dimensional version of dim(W+X)+dim(W \cap X)=dim(W)+dim(X)
  • Loading branch information
kbuzzard committed Jul 7, 2020
1 parent ea10944 commit 35940dd
Showing 1 changed file with 10 additions and 0 deletions.
10 changes: 10 additions & 0 deletions src/linear_algebra/finite_dimensional.lean
Expand Up @@ -455,6 +455,16 @@ lemma findim_quotient_le [finite_dimensional K V] (s : submodule K V) :
findim K s.quotient ≤ findim K V :=
by { rw ← s.findim_quotient_add_findim, exact nat.le_add_right _ _ }

/-- The sum of the dimensions of s + t and s ∩ t is the sum of the dimensions of s and t -/
theorem dim_sup_add_dim_inf_eq [finite_dimensional K V] (s t : submodule K V) :
findim K ↥(s ⊔ t) + findim K ↥(s ⊓ t) = findim K ↥s + findim K ↥t :=
begin
have key : dim K ↥(s ⊔ t) + dim K ↥(s ⊓ t) = dim K s + dim K t := dim_sup_add_dim_inf_eq s t,
repeat { rw ←findim_eq_dim at key },
norm_cast at key,
exact key
end

end submodule

namespace linear_equiv
Expand Down

0 comments on commit 35940dd

Please sign in to comment.