Skip to content

Commit

Permalink
merge master, including dimension lemmas of #3054
Browse files Browse the repository at this point in the history
  • Loading branch information
hrmacbeth committed Jun 13, 2020
1 parent 8871e94 commit d5d35a7
Showing 1 changed file with 0 additions and 8 deletions.
8 changes: 0 additions & 8 deletions src/linear_algebra/dimension.lean
Original file line number Diff line number Diff line change
Expand Up @@ -360,14 +360,6 @@ lemma exists_mem_ne_zero_of_dim_pos {s : submodule K V} (h : vector_space.dim K
∃ b : V, b ∈ s ∧ b ≠ 0 :=
exists_mem_ne_zero_of_ne_bot $ assume eq, by rw [(>), eq, dim_bot] at h; exact lt_irrefl _ h

lemma exists_mem_ne_zero_of_dim_pos' (h : vector_space.dim K V > 0) :
∃ b : V, b ≠ 0 :=
begin
have h' : vector_space.dim K (⊤ : subspace K V) > 0 := by {convert h using 1, simp},
cases exists_mem_ne_zero_of_dim_pos h' with b hb,
use b, exact hb.2,
end

lemma exists_is_basis_fintype (h : dim K V < cardinal.omega) :
∃ s : (set V), (is_basis K (subtype.val : s → V)) ∧ nonempty (fintype s) :=
begin
Expand Down

0 comments on commit d5d35a7

Please sign in to comment.