Basis
Definition 1. A basis ββ for VV is a linearly independent subset of VV such that <ββ> = VV.
generating set은 해당 벡터 공간의 정보를 알려주는 집합이고, 이때 최대한 그 크기를 줄인 집합이 linearly independent set이었다. 즉 두 조건을 모두 만족시키는 집합이야말로 벡터 공간을 다루기에 가장 좋은 집합이므로, 기저라는 이름으로 정의한다.
Remark
Remark.
(a) A basis can be infinite.
(b) Since <∅∅> = {0}{0} and ∅∅ is linearly independent, ∅∅ is a basis for {0}{0}.
(c) In FnFn, let e1=(1,0,...,0),e2=(0,1,...,0),...,en=(0,0,...,1)e1=(1,0,...,0),e2=(0,1,...,0),...,en=(0,0,...,1). Then the set {e1,e2,...,en}{e1,e2,...,en} is a basis for FnFn and is called the standard basis for FnFn.
Theorem 1
Theorem 1. Let β={u1,u2,...,un}⊆Vβ={u1,u2,...,un}⊆V.
Then ββ is a basis for VV ⟺⟺ ∀v∈V,!∃ai∈F(i=1,...,n)∀v∈V,!∃ai∈F(i=1,...,n) such that v=∑ni=1aiuiv=∑ni=1aiui.
Proof.
(⟹)(⟹) Since <ββ> = VV, it suffices to check the uniqueness. Let v∈Vv∈V. Suppose that vv can be represented as two different ways: v=∑aiuiv=∑aiui and v=∑biuiv=∑biui for ai,bi∈Fai,bi∈F. Then 0=∑(ai−bi)ui0=∑(ai−bi)ui. Since ββ is linearly independent, ai−bi=0⟺ai=biai−bi=0⟺ai=bi. Hence vv is uniquely expressible as a linear combination of the vectors of ββ.
(⟸)(⟸)
Clearly <ββ> = VV.
- Sol 1)
Suppose that ββ is linearly dependent. Then 0=∑aiui0=∑aiui for ai∈Fai∈F, not all zero. Then 0=0+0=∑aiui+∑aiui=∑(2ai)ui0=0+0=∑aiui+∑aiui=∑(2ai)ui. Since 0∈V0∈V, 00 uniquely expressed by vectors of ββ. Thus ai=2ai⟺ai=0⨂ai=2ai⟺ai=0⨂ Hence ββ is linearly independent and so ββ is a basis for VV.
- Sol 2)
Suppose that ββ is linearly dependent and that !∃ai∈F(i=1,...,n)!∃ai∈F(i=1,...,n) such that 0=∑ni=1aiui0=∑ni=1aiui. Then some aiai, says a1a1, is nonzero, so we have u1=∑nj=2(−aja1)uj⟹u1∈u1=∑nj=2(−aja1)uj⟹u1∈ <β∖{u1}β∖{u1}>. Thus <β∖{u1}β∖{u1}> = VV. ⟹!∃bj∈F(j=1,...,n)⟹!∃bj∈F(j=1,...,n) such that 0=∑nj=2bjuj0=∑nj=2bjuj. Then we have two different representations of 00 as a linear combination of the vectors of ββ. ⨂⨂ Hence ββ is linearly independent and so ββ is a basis for VV. ◼■
ββ가 VV의 기저일 때, 각 v∈Vv∈V마다 (a1,...,an)(a1,...,an)이 유일하게 정해지므로 bijection인 T:v⟼(a1,...,an)T:v⟼(a1,...,an)가 존재한다. 즉 V≃FnV≃Fn임을 알 수 있다.
Theorem 2
Theorem 2. If VV is generated by a finite set SS, then some subset of SS is a basis for VV.
Proof. If S=∅S=∅ or S={0}S={0}, then V=V= <SS> = {0}{0} and ∅∅ is a subset of SS that is a basis for VV.
Suppose that SS contains a nonzero vector u1u1. Then {u1}{u1} is a linearly independent set. Continue, if possible, choose vectors u2,...,uk∈Su2,...,uk∈S such that {u1,u2,...,uk}{u1,u2,...,uk} is linearly independent. Since SS is a finite set, we must eventually reach a stage at which β={u1,u2,...,uk}β={u1,u2,...,uk} is a linearly independent subset of SS, but adjoining to ββ any vector in SS, not in ββ, produces a linearly dependent set. (Note that Theorem 2) Since ββ is linearly independent, it suffices to show that <ββ> = VV.
Since <ββ> ⊆⊆ <SS> = VV, we need to show SS ⊆⊆ <ββ>.
Let v∈Sv∈S. If v∈βv∈β, then clearly v∈v∈ <ββ>. Otherwise, if v∉βv∉β, then β∪{v}β∪{v} is linearly dependent on the preceding construction. So v∈v∈ <ββ> by Theorem 2. Thus S⊆S⊆ <ββ> ⟹⟹ <SS> ⊆⊆ <ββ> ⟹⟹ <ββ> = <SS> = VV. Thus ββ is a basis for VV. ◼■
앞서 말했듯 기저는 결국 generating set중 가장 크기가 작은 집합이므로, 뒤집으면 임의의 generating set이 주어지면 그 안에서 적당히 벡터를 골라내어서 기저를 잡아낼 수 있다는 것이다.
Theorem 3 (Replacement Theorem)
Theorem 3. (Replacement Theorem) Let VV be generated by a set GG containing exactly nn vectors, and let LL be a linearly independent subset of VV containing exactly mm vectors. Then m≤nm≤n and ∃H⊆G∃H⊆G containing exactly n−mn−m vectors such that L∪HL∪H generates VV.

기저란 generating set과 linearly independent set 모두를 만족하는 집합이다. 이때 기저에서 크기를 키우면 linearly independent의 조건이 사라지고, 크기를 줄이면 generate의 조건이 사라진다. 즉 두 조건의 경계가 기저가 됨을 알 수 있다. '기저 대체 정리'라고도 불리는 replacement theorem은 이러한 generating set과 linearly independent set 사이의 관계를 보여준다.
Proof. Apply the mathematical induction on mm.
(i) m=0m=0
Clearly 0≤n0≤n, and since L=∅L=∅, we can take H=GH=G.
(ii) m=km=k
Suppose that the theorem is true for some integer k>0k>0. That is, k≤nk≤n and for the linearly independent subset L′={v1,...,vk}L′={v1,...,vk} of VV, ∃H′⊆G∃H′⊆G containing exactly n−kn−k vectors such that L′∪H′L′∪H′ generates VV. Let take H′={u1,...,un−k}H′={u1,...,un−k}.
(iii) m=k+1m=k+1
Let L={v1,...,vk,vk+1}L={v1,...,vk,vk+1} be a linearly independent subset of VV. Since vk+1∈Vvk+1∈V, vk+1=k∑i=1aivi+n−k∑j=1bjujvk+1=k∑i=1aivi+n−k∑j=1bjuj for ai,bj∈F(i=1,...,k,j=1,...,n−k).
Note that
(1) n≠k,
(2) some bj, say b1, is nonzero. ((∵) Otherwise, L is linearly dependent ⨂.)
Thus
(1) k<n⟹k+1≤n,
(2) u1=k∑i=1(−aib1)vi+1b1vk+1+n−k∑j=2(−bjb1)uj.
Let H={u2,...,un−k}. Then u1∈ <L∪H>. Note that L′∪H′⊆ <L∪H> ⟹V=<L′∪H′> ⊆ <L∪H>. Clearly <L∪H> ⊆V. Thus L∪H generates V. ◼
Corollary 3 - 1
Corollary 3 - 1. Let V be a vector space having a finite basis. Then every basis for V contains the same number of vectors.
Proof. Let β be a finite basis for V that contains exactly n vectors, and let γ be any other basis for V. If γ contains more than n vectors, then we can select a subset S of γ containing exactly n+1 vectors. Since S is linearly independent (γ is a basis for V) and β generates V, the replacement theorem implies that n+1≤n.⨂
Therefore γ is finite, and the number m of vectors in γ satisfies m≤n. Reversing the roles of β and γ and arguing as above, we obtain n≤m. Hence m=n. ◼
Dimension
Definition 2. A vector space is called finite-dimensional if it has a basis consisting of a finite number of vectors. This number is called the dimension of V, denoted dim(V).
A vector space that is not finite-dimensional is called infinite-dimensional.
corollary 1에 의해 유한한 크기의 기저를 가지는 각 벡터공간마다 고유한 숫자가 부여되고, 이를 벡터공간의 차원이라 정의한다. 주의할 점은, 벡터 공간에 주어진 field에 따라 차원이 달라질 수 있다. 예컨대 복소수 집합 C는 C 위에서는 차원이 1이지만, R 위에서는 2이다.
Corollary 3 - 2
Corollary 3 - 2. Let dim(V) = n.
(a) Any finite generating set for V contains at least n vectors, and a generating set for V that contains exactly n vectors is a basis for V.
(b) Any linearly independent subset of V contains at most n vectors, and a linearly independent subset of V that contains exactly n vectors is a basis for V.
(c) Every linearly independent subset of V can be extended to a basis for V.
(d) Every generating set for V can be reduced to a basis for V.
Proof.
(a) Let G be a finite generating set for V. By Theorem 2, ∃H∈G such that H is a basis for V. Since |H|=n, G contains at least n vectors. If we take |G|=n, then we must have H=G.
(b) Let L be a finite linearly independent subset of V, and let β be a basis for V. By the replacement theorem, L contains at most n vectors. If we take |L|=n, then, it follows from the replacement theorem that there is a subset H of β containing (n−n)=0 vectors, i.e., H=∅, such that H∪L=L generates V. Hence L is a basis for V.
(c) Let L be a linearly independent subset of V containing m vectors, and let β be a basis for V. The replacement theorem asserts that m≤n and ∃ H∈β such that |H|=n−m and L∪H generates V. Then L∪H contains at most n vectors and also contains at least n vectors by (a). Hence |L∪H|=n so that L∪H is a basis for V by (a).
(d) By theorem 2, it holds. ◼
Theorem 4
Theorem 4. Let W≤V (dim(V) = n). Then W is finite-dimensional and dim(W) ≤ dim(V). Moreover, if dim(W) = dim(V), then V=W.
Proof.
- Sol 1)
Let α and β be bases for W and V, respectively. Then α is a linearly independent subset of V and β is a generating set for V. By the replacement theorem, |α| = dim(W) ≤ dim(V) = |β|. Since V is finite-dimensional, so is W. Moreover, if dim(W) = dim(V), then α is a basis for V by corollary 3 - 2 (b). Thus V = <α> = W.
- Sol 2)
Let β be a basis for V. If W={0}, then clearly the theorem is true. Otherwise, a nonzero vector u1∈W. We can continue the process to choose the vectors in W such that γ={u1,...,uk} is linearly independent until adjoining other vectors in W to γ produces a linearly dependent set. Then by the replacement theorem, k≤n.
Let v∈W but v∉γ. Then γ∪{v} is linearly dependent ⟺ v∈<γ>. Clearly γ⊆<γ> ⊆W. Thus <γ> = W. Hence dim(W) = k. ◼
Corollary 4 - 1
Corollary 4 - 1. If W≤V (V is finite-dimensional), then any basis for W can be extended to a basis for V.
Proof. Since a basis for W is a linearly independent subset of V, it follows from Corollary 3 - 2 (c) that a basis for W can be extended to a basis for V. ◼
Reference is here: https://product.kyobobook.co.kr/detail/S000003155051
Linear Algebra | Stephen Friedberg - 교보문고
Linear Algebra | For courses in Advanced Linear Algebra. This top-selling, theorem-proof text presents a careful treatment of the principle topics of linear algebra, and illustrates the power of the subject through a variety of applications. It emphasizes
product.kyobobook.co.kr