| Metamath
Proof Explorer Theorem List (p. 217 of 497) | < Previous Next > | |
| Bad symbols? Try the
GIF version. |
||
|
Mirrors > Metamath Home Page > MPE Home Page > Theorem List Contents > Recent Proofs This page: Page List |
||
| Color key: | (1-30845) |
(30846-32368) |
(32369-49617) |
| Type | Label | Description |
|---|---|---|
| Statement | ||
| Theorem | ipsubdi 21601 | Distributive law for inner product subtraction. (Contributed by NM, 20-Nov-2007.) (Revised by Mario Carneiro, 7-Oct-2015.) |
| ⊢ 𝐹 = (Scalar‘𝑊) & ⊢ , = (·𝑖‘𝑊) & ⊢ 𝑉 = (Base‘𝑊) & ⊢ − = (-g‘𝑊) & ⊢ 𝑆 = (-g‘𝐹) ⇒ ⊢ ((𝑊 ∈ PreHil ∧ (𝐴 ∈ 𝑉 ∧ 𝐵 ∈ 𝑉 ∧ 𝐶 ∈ 𝑉)) → (𝐴 , (𝐵 − 𝐶)) = ((𝐴 , 𝐵)𝑆(𝐴 , 𝐶))) | ||
| Theorem | ip2subdi 21602 | Distributive law for inner product subtraction. (Contributed by Mario Carneiro, 8-Oct-2015.) |
| ⊢ 𝐹 = (Scalar‘𝑊) & ⊢ , = (·𝑖‘𝑊) & ⊢ 𝑉 = (Base‘𝑊) & ⊢ − = (-g‘𝑊) & ⊢ 𝑆 = (-g‘𝐹) & ⊢ + = (+g‘𝐹) & ⊢ (𝜑 → 𝑊 ∈ PreHil) & ⊢ (𝜑 → 𝐴 ∈ 𝑉) & ⊢ (𝜑 → 𝐵 ∈ 𝑉) & ⊢ (𝜑 → 𝐶 ∈ 𝑉) & ⊢ (𝜑 → 𝐷 ∈ 𝑉) ⇒ ⊢ (𝜑 → ((𝐴 − 𝐵) , (𝐶 − 𝐷)) = (((𝐴 , 𝐶) + (𝐵 , 𝐷))𝑆((𝐴 , 𝐷) + (𝐵 , 𝐶)))) | ||
| Theorem | ipass 21603 | Associative law for inner product. Equation I2 of [Ponnusamy] p. 363. (Contributed by NM, 25-Aug-2007.) (Revised by Mario Carneiro, 7-Oct-2015.) |
| ⊢ 𝐹 = (Scalar‘𝑊) & ⊢ , = (·𝑖‘𝑊) & ⊢ 𝑉 = (Base‘𝑊) & ⊢ 𝐾 = (Base‘𝐹) & ⊢ · = ( ·𝑠 ‘𝑊) & ⊢ × = (.r‘𝐹) ⇒ ⊢ ((𝑊 ∈ PreHil ∧ (𝐴 ∈ 𝐾 ∧ 𝐵 ∈ 𝑉 ∧ 𝐶 ∈ 𝑉)) → ((𝐴 · 𝐵) , 𝐶) = (𝐴 × (𝐵 , 𝐶))) | ||
| Theorem | ipassr 21604 | "Associative" law for second argument of inner product (compare ipass 21603). (Contributed by NM, 25-Aug-2007.) (Revised by Mario Carneiro, 7-Oct-2015.) |
| ⊢ 𝐹 = (Scalar‘𝑊) & ⊢ , = (·𝑖‘𝑊) & ⊢ 𝑉 = (Base‘𝑊) & ⊢ 𝐾 = (Base‘𝐹) & ⊢ · = ( ·𝑠 ‘𝑊) & ⊢ × = (.r‘𝐹) & ⊢ ∗ = (*𝑟‘𝐹) ⇒ ⊢ ((𝑊 ∈ PreHil ∧ (𝐴 ∈ 𝑉 ∧ 𝐵 ∈ 𝑉 ∧ 𝐶 ∈ 𝐾)) → (𝐴 , (𝐶 · 𝐵)) = ((𝐴 , 𝐵) × ( ∗ ‘𝐶))) | ||
| Theorem | ipassr2 21605 | "Associative" law for inner product. Conjugate version of ipassr 21604. (Contributed by NM, 25-Aug-2007.) (Revised by Mario Carneiro, 7-Oct-2015.) |
| ⊢ 𝐹 = (Scalar‘𝑊) & ⊢ , = (·𝑖‘𝑊) & ⊢ 𝑉 = (Base‘𝑊) & ⊢ 𝐾 = (Base‘𝐹) & ⊢ · = ( ·𝑠 ‘𝑊) & ⊢ × = (.r‘𝐹) & ⊢ ∗ = (*𝑟‘𝐹) ⇒ ⊢ ((𝑊 ∈ PreHil ∧ (𝐴 ∈ 𝑉 ∧ 𝐵 ∈ 𝑉 ∧ 𝐶 ∈ 𝐾)) → ((𝐴 , 𝐵) × 𝐶) = (𝐴 , (( ∗ ‘𝐶) · 𝐵))) | ||
| Theorem | ipffval 21606* | The inner product operation as a function. (Contributed by Mario Carneiro, 12-Oct-2015.) (Proof shortened by AV, 2-Mar-2024.) |
| ⊢ 𝑉 = (Base‘𝑊) & ⊢ , = (·𝑖‘𝑊) & ⊢ · = (·if‘𝑊) ⇒ ⊢ · = (𝑥 ∈ 𝑉, 𝑦 ∈ 𝑉 ↦ (𝑥 , 𝑦)) | ||
| Theorem | ipfval 21607 | The inner product operation as a function. (Contributed by Mario Carneiro, 14-Aug-2015.) |
| ⊢ 𝑉 = (Base‘𝑊) & ⊢ , = (·𝑖‘𝑊) & ⊢ · = (·if‘𝑊) ⇒ ⊢ ((𝑋 ∈ 𝑉 ∧ 𝑌 ∈ 𝑉) → (𝑋 · 𝑌) = (𝑋 , 𝑌)) | ||
| Theorem | ipfeq 21608 | If the inner product operation is already a function, the functionalization of it is equal to the original operation. (Contributed by Mario Carneiro, 14-Aug-2015.) |
| ⊢ 𝑉 = (Base‘𝑊) & ⊢ , = (·𝑖‘𝑊) & ⊢ · = (·if‘𝑊) ⇒ ⊢ ( , Fn (𝑉 × 𝑉) → · = , ) | ||
| Theorem | ipffn 21609 | The inner product operation is a function. (Contributed by Mario Carneiro, 20-Sep-2015.) |
| ⊢ 𝑉 = (Base‘𝑊) & ⊢ , = (·if‘𝑊) ⇒ ⊢ , Fn (𝑉 × 𝑉) | ||
| Theorem | phlipf 21610 | The inner product operation is a function. (Contributed by Mario Carneiro, 14-Aug-2015.) |
| ⊢ 𝑉 = (Base‘𝑊) & ⊢ , = (·if‘𝑊) & ⊢ 𝑆 = (Scalar‘𝑊) & ⊢ 𝐾 = (Base‘𝑆) ⇒ ⊢ (𝑊 ∈ PreHil → , :(𝑉 × 𝑉)⟶𝐾) | ||
| Theorem | ip2eq 21611* | Two vectors are equal iff their inner products with all other vectors are equal. (Contributed by NM, 24-Jan-2008.) (Revised by Mario Carneiro, 7-Oct-2015.) |
| ⊢ , = (·𝑖‘𝑊) & ⊢ 𝑉 = (Base‘𝑊) ⇒ ⊢ ((𝑊 ∈ PreHil ∧ 𝐴 ∈ 𝑉 ∧ 𝐵 ∈ 𝑉) → (𝐴 = 𝐵 ↔ ∀𝑥 ∈ 𝑉 (𝑥 , 𝐴) = (𝑥 , 𝐵))) | ||
| Theorem | isphld 21612* | Properties that determine a pre-Hilbert (inner product) space. (Contributed by Mario Carneiro, 18-Nov-2013.) (Revised by Mario Carneiro, 7-Oct-2015.) |
| ⊢ (𝜑 → 𝑉 = (Base‘𝑊)) & ⊢ (𝜑 → + = (+g‘𝑊)) & ⊢ (𝜑 → · = ( ·𝑠 ‘𝑊)) & ⊢ (𝜑 → 𝐼 = (·𝑖‘𝑊)) & ⊢ (𝜑 → 0 = (0g‘𝑊)) & ⊢ (𝜑 → 𝐹 = (Scalar‘𝑊)) & ⊢ (𝜑 → 𝐾 = (Base‘𝐹)) & ⊢ (𝜑 → ⨣ = (+g‘𝐹)) & ⊢ (𝜑 → × = (.r‘𝐹)) & ⊢ (𝜑 → ∗ = (*𝑟‘𝐹)) & ⊢ (𝜑 → 𝑂 = (0g‘𝐹)) & ⊢ (𝜑 → 𝑊 ∈ LVec) & ⊢ (𝜑 → 𝐹 ∈ *-Ring) & ⊢ ((𝜑 ∧ 𝑥 ∈ 𝑉 ∧ 𝑦 ∈ 𝑉) → (𝑥𝐼𝑦) ∈ 𝐾) & ⊢ ((𝜑 ∧ 𝑞 ∈ 𝐾 ∧ (𝑥 ∈ 𝑉 ∧ 𝑦 ∈ 𝑉 ∧ 𝑧 ∈ 𝑉)) → (((𝑞 · 𝑥) + 𝑦)𝐼𝑧) = ((𝑞 × (𝑥𝐼𝑧)) ⨣ (𝑦𝐼𝑧))) & ⊢ ((𝜑 ∧ 𝑥 ∈ 𝑉 ∧ (𝑥𝐼𝑥) = 𝑂) → 𝑥 = 0 ) & ⊢ ((𝜑 ∧ 𝑥 ∈ 𝑉 ∧ 𝑦 ∈ 𝑉) → ( ∗ ‘(𝑥𝐼𝑦)) = (𝑦𝐼𝑥)) ⇒ ⊢ (𝜑 → 𝑊 ∈ PreHil) | ||
| Theorem | phlpropd 21613* | If two structures have the same components (properties), one is a pre-Hilbert space iff the other one is. (Contributed by Mario Carneiro, 8-Oct-2015.) |
| ⊢ (𝜑 → 𝐵 = (Base‘𝐾)) & ⊢ (𝜑 → 𝐵 = (Base‘𝐿)) & ⊢ ((𝜑 ∧ (𝑥 ∈ 𝐵 ∧ 𝑦 ∈ 𝐵)) → (𝑥(+g‘𝐾)𝑦) = (𝑥(+g‘𝐿)𝑦)) & ⊢ (𝜑 → 𝐹 = (Scalar‘𝐾)) & ⊢ (𝜑 → 𝐹 = (Scalar‘𝐿)) & ⊢ 𝑃 = (Base‘𝐹) & ⊢ ((𝜑 ∧ (𝑥 ∈ 𝑃 ∧ 𝑦 ∈ 𝐵)) → (𝑥( ·𝑠 ‘𝐾)𝑦) = (𝑥( ·𝑠 ‘𝐿)𝑦)) & ⊢ ((𝜑 ∧ (𝑥 ∈ 𝐵 ∧ 𝑦 ∈ 𝐵)) → (𝑥(·𝑖‘𝐾)𝑦) = (𝑥(·𝑖‘𝐿)𝑦)) ⇒ ⊢ (𝜑 → (𝐾 ∈ PreHil ↔ 𝐿 ∈ PreHil)) | ||
| Theorem | ssipeq 21614 | The inner product on a subspace equals the inner product on the parent space. (Contributed by AV, 19-Oct-2021.) |
| ⊢ 𝑋 = (𝑊 ↾s 𝑈) & ⊢ , = (·𝑖‘𝑊) & ⊢ 𝑃 = (·𝑖‘𝑋) ⇒ ⊢ (𝑈 ∈ 𝑆 → 𝑃 = , ) | ||
| Theorem | phssipval 21615 | The inner product on a subspace in terms of the inner product on the parent space. (Contributed by NM, 28-Jan-2008.) (Revised by AV, 19-Oct-2021.) |
| ⊢ 𝑋 = (𝑊 ↾s 𝑈) & ⊢ , = (·𝑖‘𝑊) & ⊢ 𝑃 = (·𝑖‘𝑋) & ⊢ 𝑆 = (LSubSp‘𝑊) ⇒ ⊢ (((𝑊 ∈ PreHil ∧ 𝑈 ∈ 𝑆) ∧ (𝐴 ∈ 𝑈 ∧ 𝐵 ∈ 𝑈)) → (𝐴𝑃𝐵) = (𝐴 , 𝐵)) | ||
| Theorem | phssip 21616 | The inner product (as a function) on a subspace is a restriction of the inner product (as a function) on the parent space. (Contributed by NM, 28-Jan-2008.) (Revised by AV, 19-Oct-2021.) |
| ⊢ 𝑋 = (𝑊 ↾s 𝑈) & ⊢ 𝑆 = (LSubSp‘𝑊) & ⊢ · = (·if‘𝑊) & ⊢ 𝑃 = (·if‘𝑋) ⇒ ⊢ ((𝑊 ∈ PreHil ∧ 𝑈 ∈ 𝑆) → 𝑃 = ( · ↾ (𝑈 × 𝑈))) | ||
| Theorem | phlssphl 21617 | A subspace of an inner product space (pre-Hilbert space) is an inner product space. (Contributed by AV, 25-Sep-2022.) |
| ⊢ 𝑋 = (𝑊 ↾s 𝑈) & ⊢ 𝑆 = (LSubSp‘𝑊) ⇒ ⊢ ((𝑊 ∈ PreHil ∧ 𝑈 ∈ 𝑆) → 𝑋 ∈ PreHil) | ||
| Syntax | cocv 21618 | Extend class notation with orthocomplement of a subset. |
| class ocv | ||
| Syntax | ccss 21619 | Extend class notation with set of closed subspaces. |
| class ClSubSp | ||
| Syntax | cthl 21620 | Extend class notation with the Hilbert lattice. |
| class toHL | ||
| Definition | df-ocv 21621* | Define the orthocomplement function in a given set (which usually is a pre-Hilbert space): it associates with a subset its orthogonal subset (which in the case of a closed linear subspace is its orthocomplement). (Contributed by NM, 7-Oct-2011.) |
| ⊢ ocv = (ℎ ∈ V ↦ (𝑠 ∈ 𝒫 (Base‘ℎ) ↦ {𝑥 ∈ (Base‘ℎ) ∣ ∀𝑦 ∈ 𝑠 (𝑥(·𝑖‘ℎ)𝑦) = (0g‘(Scalar‘ℎ))})) | ||
| Definition | df-css 21622* | Define the set of closed (linear) subspaces of a given pre-Hilbert space. (Contributed by NM, 7-Oct-2011.) |
| ⊢ ClSubSp = (ℎ ∈ V ↦ {𝑠 ∣ 𝑠 = ((ocv‘ℎ)‘((ocv‘ℎ)‘𝑠))}) | ||
| Definition | df-thl 21623 | Define the Hilbert lattice of closed subspaces of a given pre-Hilbert space. (Contributed by Mario Carneiro, 25-Oct-2015.) |
| ⊢ toHL = (ℎ ∈ V ↦ ((toInc‘(ClSubSp‘ℎ)) sSet 〈(oc‘ndx), (ocv‘ℎ)〉)) | ||
| Theorem | ocvfval 21624* | The orthocomplement operation. (Contributed by NM, 7-Oct-2011.) (Revised by Mario Carneiro, 13-Oct-2015.) |
| ⊢ 𝑉 = (Base‘𝑊) & ⊢ , = (·𝑖‘𝑊) & ⊢ 𝐹 = (Scalar‘𝑊) & ⊢ 0 = (0g‘𝐹) & ⊢ ⊥ = (ocv‘𝑊) ⇒ ⊢ (𝑊 ∈ 𝑋 → ⊥ = (𝑠 ∈ 𝒫 𝑉 ↦ {𝑥 ∈ 𝑉 ∣ ∀𝑦 ∈ 𝑠 (𝑥 , 𝑦) = 0 })) | ||
| Theorem | ocvval 21625* | Value of the orthocomplement of a subset (normally a subspace) of a pre-Hilbert space. (Contributed by NM, 7-Oct-2011.) (Revised by Mario Carneiro, 13-Oct-2015.) |
| ⊢ 𝑉 = (Base‘𝑊) & ⊢ , = (·𝑖‘𝑊) & ⊢ 𝐹 = (Scalar‘𝑊) & ⊢ 0 = (0g‘𝐹) & ⊢ ⊥ = (ocv‘𝑊) ⇒ ⊢ (𝑆 ⊆ 𝑉 → ( ⊥ ‘𝑆) = {𝑥 ∈ 𝑉 ∣ ∀𝑦 ∈ 𝑆 (𝑥 , 𝑦) = 0 }) | ||
| Theorem | elocv 21626* | Elementhood in the orthocomplement of a subset (normally a subspace) of a pre-Hilbert space. (Contributed by Mario Carneiro, 13-Oct-2015.) |
| ⊢ 𝑉 = (Base‘𝑊) & ⊢ , = (·𝑖‘𝑊) & ⊢ 𝐹 = (Scalar‘𝑊) & ⊢ 0 = (0g‘𝐹) & ⊢ ⊥ = (ocv‘𝑊) ⇒ ⊢ (𝐴 ∈ ( ⊥ ‘𝑆) ↔ (𝑆 ⊆ 𝑉 ∧ 𝐴 ∈ 𝑉 ∧ ∀𝑥 ∈ 𝑆 (𝐴 , 𝑥) = 0 )) | ||
| Theorem | ocvi 21627 | Property of a member of the orthocomplement of a subset. (Contributed by Mario Carneiro, 13-Oct-2015.) |
| ⊢ 𝑉 = (Base‘𝑊) & ⊢ , = (·𝑖‘𝑊) & ⊢ 𝐹 = (Scalar‘𝑊) & ⊢ 0 = (0g‘𝐹) & ⊢ ⊥ = (ocv‘𝑊) ⇒ ⊢ ((𝐴 ∈ ( ⊥ ‘𝑆) ∧ 𝐵 ∈ 𝑆) → (𝐴 , 𝐵) = 0 ) | ||
| Theorem | ocvss 21628 | The orthocomplement of a subset is a subset of the base. (Contributed by Mario Carneiro, 13-Oct-2015.) |
| ⊢ 𝑉 = (Base‘𝑊) & ⊢ ⊥ = (ocv‘𝑊) ⇒ ⊢ ( ⊥ ‘𝑆) ⊆ 𝑉 | ||
| Theorem | ocvocv 21629 | A set is contained in its double orthocomplement. (Contributed by Mario Carneiro, 13-Oct-2015.) |
| ⊢ 𝑉 = (Base‘𝑊) & ⊢ ⊥ = (ocv‘𝑊) ⇒ ⊢ ((𝑊 ∈ PreHil ∧ 𝑆 ⊆ 𝑉) → 𝑆 ⊆ ( ⊥ ‘( ⊥ ‘𝑆))) | ||
| Theorem | ocvlss 21630 | The orthocomplement of a subset is a linear subspace of the pre-Hilbert space. (Contributed by Mario Carneiro, 13-Oct-2015.) |
| ⊢ 𝑉 = (Base‘𝑊) & ⊢ ⊥ = (ocv‘𝑊) & ⊢ 𝐿 = (LSubSp‘𝑊) ⇒ ⊢ ((𝑊 ∈ PreHil ∧ 𝑆 ⊆ 𝑉) → ( ⊥ ‘𝑆) ∈ 𝐿) | ||
| Theorem | ocv2ss 21631 | Orthocomplements reverse subset inclusion. (Contributed by Mario Carneiro, 13-Oct-2015.) |
| ⊢ ⊥ = (ocv‘𝑊) ⇒ ⊢ (𝑇 ⊆ 𝑆 → ( ⊥ ‘𝑆) ⊆ ( ⊥ ‘𝑇)) | ||
| Theorem | ocvin 21632 | An orthocomplement has trivial intersection with the original subspace. (Contributed by Mario Carneiro, 16-Oct-2015.) |
| ⊢ ⊥ = (ocv‘𝑊) & ⊢ 𝐿 = (LSubSp‘𝑊) & ⊢ 0 = (0g‘𝑊) ⇒ ⊢ ((𝑊 ∈ PreHil ∧ 𝑆 ∈ 𝐿) → (𝑆 ∩ ( ⊥ ‘𝑆)) = { 0 }) | ||
| Theorem | ocvsscon 21633 | Two ways to say that 𝑆 and 𝑇 are orthogonal subspaces. (Contributed by Mario Carneiro, 23-Oct-2015.) |
| ⊢ 𝑉 = (Base‘𝑊) & ⊢ ⊥ = (ocv‘𝑊) ⇒ ⊢ ((𝑊 ∈ PreHil ∧ 𝑆 ⊆ 𝑉 ∧ 𝑇 ⊆ 𝑉) → (𝑆 ⊆ ( ⊥ ‘𝑇) ↔ 𝑇 ⊆ ( ⊥ ‘𝑆))) | ||
| Theorem | ocvlsp 21634 | The orthocomplement of a linear span. (Contributed by Mario Carneiro, 23-Oct-2015.) |
| ⊢ 𝑉 = (Base‘𝑊) & ⊢ ⊥ = (ocv‘𝑊) & ⊢ 𝑁 = (LSpan‘𝑊) ⇒ ⊢ ((𝑊 ∈ PreHil ∧ 𝑆 ⊆ 𝑉) → ( ⊥ ‘(𝑁‘𝑆)) = ( ⊥ ‘𝑆)) | ||
| Theorem | ocv0 21635 | The orthocomplement of the empty set. (Contributed by Mario Carneiro, 23-Oct-2015.) |
| ⊢ 𝑉 = (Base‘𝑊) & ⊢ ⊥ = (ocv‘𝑊) ⇒ ⊢ ( ⊥ ‘∅) = 𝑉 | ||
| Theorem | ocvz 21636 | The orthocomplement of the zero subspace. (Contributed by Mario Carneiro, 23-Oct-2015.) |
| ⊢ 𝑉 = (Base‘𝑊) & ⊢ ⊥ = (ocv‘𝑊) & ⊢ 0 = (0g‘𝑊) ⇒ ⊢ (𝑊 ∈ PreHil → ( ⊥ ‘{ 0 }) = 𝑉) | ||
| Theorem | ocv1 21637 | The orthocomplement of the base set. (Contributed by Mario Carneiro, 23-Oct-2015.) |
| ⊢ 𝑉 = (Base‘𝑊) & ⊢ ⊥ = (ocv‘𝑊) & ⊢ 0 = (0g‘𝑊) ⇒ ⊢ (𝑊 ∈ PreHil → ( ⊥ ‘𝑉) = { 0 }) | ||
| Theorem | unocv 21638 | The orthocomplement of a union. (Contributed by Mario Carneiro, 23-Oct-2015.) |
| ⊢ ⊥ = (ocv‘𝑊) ⇒ ⊢ ( ⊥ ‘(𝐴 ∪ 𝐵)) = (( ⊥ ‘𝐴) ∩ ( ⊥ ‘𝐵)) | ||
| Theorem | iunocv 21639* | The orthocomplement of an indexed union. (Contributed by Mario Carneiro, 23-Oct-2015.) |
| ⊢ ⊥ = (ocv‘𝑊) & ⊢ 𝑉 = (Base‘𝑊) ⇒ ⊢ ( ⊥ ‘∪ 𝑥 ∈ 𝐴 𝐵) = (𝑉 ∩ ∩ 𝑥 ∈ 𝐴 ( ⊥ ‘𝐵)) | ||
| Theorem | cssval 21640* | The set of closed subspaces of a pre-Hilbert space. (Contributed by NM, 7-Oct-2011.) (Revised by Mario Carneiro, 13-Oct-2015.) |
| ⊢ ⊥ = (ocv‘𝑊) & ⊢ 𝐶 = (ClSubSp‘𝑊) ⇒ ⊢ (𝑊 ∈ 𝑋 → 𝐶 = {𝑠 ∣ 𝑠 = ( ⊥ ‘( ⊥ ‘𝑠))}) | ||
| Theorem | iscss 21641 | The predicate "is a closed subspace" (of a pre-Hilbert space). (Contributed by NM, 7-Oct-2011.) (Revised by Mario Carneiro, 13-Oct-2015.) |
| ⊢ ⊥ = (ocv‘𝑊) & ⊢ 𝐶 = (ClSubSp‘𝑊) ⇒ ⊢ (𝑊 ∈ 𝑋 → (𝑆 ∈ 𝐶 ↔ 𝑆 = ( ⊥ ‘( ⊥ ‘𝑆)))) | ||
| Theorem | cssi 21642 | Property of a closed subspace (of a pre-Hilbert space). (Contributed by Mario Carneiro, 13-Oct-2015.) |
| ⊢ ⊥ = (ocv‘𝑊) & ⊢ 𝐶 = (ClSubSp‘𝑊) ⇒ ⊢ (𝑆 ∈ 𝐶 → 𝑆 = ( ⊥ ‘( ⊥ ‘𝑆))) | ||
| Theorem | cssss 21643 | A closed subspace is a subset of the base. (Contributed by Mario Carneiro, 13-Oct-2015.) |
| ⊢ 𝑉 = (Base‘𝑊) & ⊢ 𝐶 = (ClSubSp‘𝑊) ⇒ ⊢ (𝑆 ∈ 𝐶 → 𝑆 ⊆ 𝑉) | ||
| Theorem | iscss2 21644 | It is sufficient to prove that the double orthocomplement is a subset of the target set to show that the set is a closed subspace. (Contributed by Mario Carneiro, 13-Oct-2015.) |
| ⊢ 𝑉 = (Base‘𝑊) & ⊢ 𝐶 = (ClSubSp‘𝑊) & ⊢ ⊥ = (ocv‘𝑊) ⇒ ⊢ ((𝑊 ∈ PreHil ∧ 𝑆 ⊆ 𝑉) → (𝑆 ∈ 𝐶 ↔ ( ⊥ ‘( ⊥ ‘𝑆)) ⊆ 𝑆)) | ||
| Theorem | ocvcss 21645 | The orthocomplement of any set is a closed subspace. (Contributed by Mario Carneiro, 13-Oct-2015.) |
| ⊢ 𝑉 = (Base‘𝑊) & ⊢ 𝐶 = (ClSubSp‘𝑊) & ⊢ ⊥ = (ocv‘𝑊) ⇒ ⊢ ((𝑊 ∈ PreHil ∧ 𝑆 ⊆ 𝑉) → ( ⊥ ‘𝑆) ∈ 𝐶) | ||
| Theorem | cssincl 21646 | The zero subspace is a closed subspace. (Contributed by Mario Carneiro, 13-Oct-2015.) |
| ⊢ 𝐶 = (ClSubSp‘𝑊) ⇒ ⊢ ((𝑊 ∈ PreHil ∧ 𝐴 ∈ 𝐶 ∧ 𝐵 ∈ 𝐶) → (𝐴 ∩ 𝐵) ∈ 𝐶) | ||
| Theorem | css0 21647 | The zero subspace is a closed subspace. (Contributed by Mario Carneiro, 13-Oct-2015.) |
| ⊢ 𝐶 = (ClSubSp‘𝑊) & ⊢ 0 = (0g‘𝑊) ⇒ ⊢ (𝑊 ∈ PreHil → { 0 } ∈ 𝐶) | ||
| Theorem | css1 21648 | The whole space is a closed subspace. (Contributed by Mario Carneiro, 13-Oct-2015.) |
| ⊢ 𝑉 = (Base‘𝑊) & ⊢ 𝐶 = (ClSubSp‘𝑊) ⇒ ⊢ (𝑊 ∈ PreHil → 𝑉 ∈ 𝐶) | ||
| Theorem | csslss 21649 | A closed subspace of a pre-Hilbert space is a linear subspace. (Contributed by Mario Carneiro, 13-Oct-2015.) |
| ⊢ 𝐶 = (ClSubSp‘𝑊) & ⊢ 𝐿 = (LSubSp‘𝑊) ⇒ ⊢ ((𝑊 ∈ PreHil ∧ 𝑆 ∈ 𝐶) → 𝑆 ∈ 𝐿) | ||
| Theorem | lsmcss 21650 | A subset of a pre-Hilbert space whose double orthocomplement has a projection decomposition is a closed subspace. This is the core of the proof that a topologically closed subspace is algebraically closed in a Hilbert space. (Contributed by Mario Carneiro, 13-Oct-2015.) |
| ⊢ 𝐶 = (ClSubSp‘𝑊) & ⊢ 𝑉 = (Base‘𝑊) & ⊢ ⊥ = (ocv‘𝑊) & ⊢ ⊕ = (LSSum‘𝑊) & ⊢ (𝜑 → 𝑊 ∈ PreHil) & ⊢ (𝜑 → 𝑆 ⊆ 𝑉) & ⊢ (𝜑 → ( ⊥ ‘( ⊥ ‘𝑆)) ⊆ (𝑆 ⊕ ( ⊥ ‘𝑆))) ⇒ ⊢ (𝜑 → 𝑆 ∈ 𝐶) | ||
| Theorem | cssmre 21651 | The closed subspaces of a pre-Hilbert space are a Moore system. Unlike many of our other examples of closure systems, this one is not usually an algebraic closure system df-acs 17599: consider the Hilbert space of sequences ℕ⟶ℝ with convergent sum; the subspace of all sequences with finite support is the classic example of a non-closed subspace, but for every finite set of sequences of finite support, there is a finite-dimensional (and hence closed) subspace containing all of the sequences, so if closed subspaces were an algebraic closure system this would violate acsfiel 17664. (Contributed by Mario Carneiro, 13-Oct-2015.) |
| ⊢ 𝑉 = (Base‘𝑊) & ⊢ 𝐶 = (ClSubSp‘𝑊) ⇒ ⊢ (𝑊 ∈ PreHil → 𝐶 ∈ (Moore‘𝑉)) | ||
| Theorem | mrccss 21652 | The Moore closure corresponding to the system of closed subspaces is the double orthocomplement operation. (Contributed by Mario Carneiro, 13-Oct-2015.) |
| ⊢ 𝑉 = (Base‘𝑊) & ⊢ ⊥ = (ocv‘𝑊) & ⊢ 𝐶 = (ClSubSp‘𝑊) & ⊢ 𝐹 = (mrCls‘𝐶) ⇒ ⊢ ((𝑊 ∈ PreHil ∧ 𝑆 ⊆ 𝑉) → (𝐹‘𝑆) = ( ⊥ ‘( ⊥ ‘𝑆))) | ||
| Theorem | thlval 21653 | Value of the Hilbert lattice. (Contributed by Mario Carneiro, 25-Oct-2015.) |
| ⊢ 𝐾 = (toHL‘𝑊) & ⊢ 𝐶 = (ClSubSp‘𝑊) & ⊢ 𝐼 = (toInc‘𝐶) & ⊢ ⊥ = (ocv‘𝑊) ⇒ ⊢ (𝑊 ∈ 𝑉 → 𝐾 = (𝐼 sSet 〈(oc‘ndx), ⊥ 〉)) | ||
| Theorem | thlbas 21654 | Base set of the Hilbert lattice of closed subspaces. (Contributed by Mario Carneiro, 25-Oct-2015.) (Proof shortened by AV, 11-Nov-2024.) |
| ⊢ 𝐾 = (toHL‘𝑊) & ⊢ 𝐶 = (ClSubSp‘𝑊) ⇒ ⊢ 𝐶 = (Base‘𝐾) | ||
| Theorem | thlle 21655 | Ordering on the Hilbert lattice of closed subspaces. (Contributed by Mario Carneiro, 25-Oct-2015.) (Proof shortened by AV, 11-Nov-2024.) |
| ⊢ 𝐾 = (toHL‘𝑊) & ⊢ 𝐶 = (ClSubSp‘𝑊) & ⊢ 𝐼 = (toInc‘𝐶) & ⊢ ≤ = (le‘𝐼) ⇒ ⊢ ≤ = (le‘𝐾) | ||
| Theorem | thlleval 21656 | Ordering on the Hilbert lattice of closed subspaces. (Contributed by Mario Carneiro, 25-Oct-2015.) |
| ⊢ 𝐾 = (toHL‘𝑊) & ⊢ 𝐶 = (ClSubSp‘𝑊) & ⊢ ≤ = (le‘𝐾) ⇒ ⊢ ((𝑆 ∈ 𝐶 ∧ 𝑇 ∈ 𝐶) → (𝑆 ≤ 𝑇 ↔ 𝑆 ⊆ 𝑇)) | ||
| Theorem | thloc 21657 | Orthocomplement on the Hilbert lattice of closed subspaces. (Contributed by Mario Carneiro, 25-Oct-2015.) |
| ⊢ 𝐾 = (toHL‘𝑊) & ⊢ ⊥ = (ocv‘𝑊) ⇒ ⊢ ⊥ = (oc‘𝐾) | ||
| Syntax | cpj 21658 | Extend class notation with orthogonal projection function. |
| class proj | ||
| Syntax | chil 21659 | Extend class notation with class of all Hilbert spaces. |
| class Hil | ||
| Syntax | cobs 21660 | Extend class notation with the set of orthonormal bases. |
| class OBasis | ||
| Definition | df-pj 21661* | Define orthogonal projection onto a subspace. This is just a wrapping of df-pj1 19616, but we restrict the domain of this function to only total projection functions. (Contributed by Mario Carneiro, 16-Oct-2015.) |
| ⊢ proj = (ℎ ∈ V ↦ ((𝑥 ∈ (LSubSp‘ℎ) ↦ (𝑥(proj1‘ℎ)((ocv‘ℎ)‘𝑥))) ∩ (V × ((Base‘ℎ) ↑m (Base‘ℎ))))) | ||
| Definition | df-hil 21662 | Define class of all Hilbert spaces. Based on Proposition 4.5, p. 176, Gudrun Kalmbach, Quantum Measures and Spaces, Kluwer, Dordrecht, 1998. (Contributed by NM, 7-Oct-2011.) (Revised by Mario Carneiro, 16-Oct-2015.) |
| ⊢ Hil = {ℎ ∈ PreHil ∣ dom (proj‘ℎ) = (ClSubSp‘ℎ)} | ||
| Definition | df-obs 21663* | Define the set of all orthonormal bases for a pre-Hilbert space. An orthonormal basis is a set of mutually orthogonal vectors with norm 1 and such that the linear span is dense in the whole space. (As this is an "algebraic" definition, before we have topology available, we express this denseness by saying that the double orthocomplement is the whole space, or equivalently, the single orthocomplement is trivial.) (Contributed by Mario Carneiro, 23-Oct-2015.) |
| ⊢ OBasis = (ℎ ∈ PreHil ↦ {𝑏 ∈ 𝒫 (Base‘ℎ) ∣ (∀𝑥 ∈ 𝑏 ∀𝑦 ∈ 𝑏 (𝑥(·𝑖‘ℎ)𝑦) = if(𝑥 = 𝑦, (1r‘(Scalar‘ℎ)), (0g‘(Scalar‘ℎ))) ∧ ((ocv‘ℎ)‘𝑏) = {(0g‘ℎ)})}) | ||
| Theorem | pjfval 21664* | The value of the projection function. (Contributed by Mario Carneiro, 16-Oct-2015.) |
| ⊢ 𝑉 = (Base‘𝑊) & ⊢ 𝐿 = (LSubSp‘𝑊) & ⊢ ⊥ = (ocv‘𝑊) & ⊢ 𝑃 = (proj1‘𝑊) & ⊢ 𝐾 = (proj‘𝑊) ⇒ ⊢ 𝐾 = ((𝑥 ∈ 𝐿 ↦ (𝑥𝑃( ⊥ ‘𝑥))) ∩ (V × (𝑉 ↑m 𝑉))) | ||
| Theorem | pjdm 21665 | A subspace is in the domain of the projection function iff the subspace admits a projection decomposition of the whole space. (Contributed by Mario Carneiro, 16-Oct-2015.) |
| ⊢ 𝑉 = (Base‘𝑊) & ⊢ 𝐿 = (LSubSp‘𝑊) & ⊢ ⊥ = (ocv‘𝑊) & ⊢ 𝑃 = (proj1‘𝑊) & ⊢ 𝐾 = (proj‘𝑊) ⇒ ⊢ (𝑇 ∈ dom 𝐾 ↔ (𝑇 ∈ 𝐿 ∧ (𝑇𝑃( ⊥ ‘𝑇)):𝑉⟶𝑉)) | ||
| Theorem | pjpm 21666 | The projection map is a partial function from subspaces of the pre-Hilbert space to total operators. (Contributed by Mario Carneiro, 16-Oct-2015.) |
| ⊢ 𝑉 = (Base‘𝑊) & ⊢ 𝐿 = (LSubSp‘𝑊) & ⊢ 𝐾 = (proj‘𝑊) ⇒ ⊢ 𝐾 ∈ ((𝑉 ↑m 𝑉) ↑pm 𝐿) | ||
| Theorem | pjfval2 21667* | Value of the projection map with implicit domain. (Contributed by Mario Carneiro, 16-Oct-2015.) |
| ⊢ ⊥ = (ocv‘𝑊) & ⊢ 𝑃 = (proj1‘𝑊) & ⊢ 𝐾 = (proj‘𝑊) ⇒ ⊢ 𝐾 = (𝑥 ∈ dom 𝐾 ↦ (𝑥𝑃( ⊥ ‘𝑥))) | ||
| Theorem | pjval 21668 | Value of the projection map. (Contributed by Mario Carneiro, 16-Oct-2015.) |
| ⊢ ⊥ = (ocv‘𝑊) & ⊢ 𝑃 = (proj1‘𝑊) & ⊢ 𝐾 = (proj‘𝑊) ⇒ ⊢ (𝑇 ∈ dom 𝐾 → (𝐾‘𝑇) = (𝑇𝑃( ⊥ ‘𝑇))) | ||
| Theorem | pjdm2 21669 | A subspace is in the domain of the projection function iff the subspace admits a projection decomposition of the whole space. (Contributed by Mario Carneiro, 16-Oct-2015.) |
| ⊢ 𝑉 = (Base‘𝑊) & ⊢ 𝐿 = (LSubSp‘𝑊) & ⊢ ⊥ = (ocv‘𝑊) & ⊢ ⊕ = (LSSum‘𝑊) & ⊢ 𝐾 = (proj‘𝑊) ⇒ ⊢ (𝑊 ∈ PreHil → (𝑇 ∈ dom 𝐾 ↔ (𝑇 ∈ 𝐿 ∧ (𝑇 ⊕ ( ⊥ ‘𝑇)) = 𝑉))) | ||
| Theorem | pjff 21670 | A projection is a linear operator. (Contributed by Mario Carneiro, 16-Oct-2015.) |
| ⊢ 𝐾 = (proj‘𝑊) ⇒ ⊢ (𝑊 ∈ PreHil → 𝐾:dom 𝐾⟶(𝑊 LMHom 𝑊)) | ||
| Theorem | pjf 21671 | A projection is a function on the base set. (Contributed by Mario Carneiro, 16-Oct-2015.) |
| ⊢ 𝐾 = (proj‘𝑊) & ⊢ 𝑉 = (Base‘𝑊) ⇒ ⊢ (𝑇 ∈ dom 𝐾 → (𝐾‘𝑇):𝑉⟶𝑉) | ||
| Theorem | pjf2 21672 | A projection is a function from the base set to the subspace. (Contributed by Mario Carneiro, 16-Oct-2015.) |
| ⊢ 𝐾 = (proj‘𝑊) & ⊢ 𝑉 = (Base‘𝑊) ⇒ ⊢ ((𝑊 ∈ PreHil ∧ 𝑇 ∈ dom 𝐾) → (𝐾‘𝑇):𝑉⟶𝑇) | ||
| Theorem | pjfo 21673 | A projection is a surjection onto the subspace. (Contributed by Mario Carneiro, 16-Oct-2015.) |
| ⊢ 𝐾 = (proj‘𝑊) & ⊢ 𝑉 = (Base‘𝑊) ⇒ ⊢ ((𝑊 ∈ PreHil ∧ 𝑇 ∈ dom 𝐾) → (𝐾‘𝑇):𝑉–onto→𝑇) | ||
| Theorem | pjcss 21674 | A projection subspace is an (algebraically) closed subspace. (Contributed by Mario Carneiro, 16-Oct-2015.) |
| ⊢ 𝐾 = (proj‘𝑊) & ⊢ 𝐶 = (ClSubSp‘𝑊) ⇒ ⊢ (𝑊 ∈ PreHil → dom 𝐾 ⊆ 𝐶) | ||
| Theorem | ocvpj 21675 | The orthocomplement of a projection subspace is a projection subspace. (Contributed by Mario Carneiro, 16-Oct-2015.) |
| ⊢ 𝐾 = (proj‘𝑊) & ⊢ ⊥ = (ocv‘𝑊) ⇒ ⊢ ((𝑊 ∈ PreHil ∧ 𝑇 ∈ dom 𝐾) → ( ⊥ ‘𝑇) ∈ dom 𝐾) | ||
| Theorem | ishil 21676 | The predicate "is a Hilbert space" (over a *-division ring). A Hilbert space is a pre-Hilbert space such that all closed subspaces have a projection decomposition. (Contributed by NM, 7-Oct-2011.) (Revised by Mario Carneiro, 22-Jun-2014.) |
| ⊢ 𝐾 = (proj‘𝐻) & ⊢ 𝐶 = (ClSubSp‘𝐻) ⇒ ⊢ (𝐻 ∈ Hil ↔ (𝐻 ∈ PreHil ∧ dom 𝐾 = 𝐶)) | ||
| Theorem | ishil2 21677* | The predicate "is a Hilbert space" (over a *-division ring). (Contributed by NM, 7-Oct-2011.) (Revised by Mario Carneiro, 22-Jun-2014.) |
| ⊢ 𝑉 = (Base‘𝐻) & ⊢ ⊕ = (LSSum‘𝐻) & ⊢ ⊥ = (ocv‘𝐻) & ⊢ 𝐶 = (ClSubSp‘𝐻) ⇒ ⊢ (𝐻 ∈ Hil ↔ (𝐻 ∈ PreHil ∧ ∀𝑠 ∈ 𝐶 (𝑠 ⊕ ( ⊥ ‘𝑠)) = 𝑉)) | ||
| Theorem | isobs 21678* | The predicate "is an orthonormal basis" (over a pre-Hilbert space). (Contributed by Mario Carneiro, 23-Oct-2015.) |
| ⊢ 𝑉 = (Base‘𝑊) & ⊢ , = (·𝑖‘𝑊) & ⊢ 𝐹 = (Scalar‘𝑊) & ⊢ 1 = (1r‘𝐹) & ⊢ 0 = (0g‘𝐹) & ⊢ ⊥ = (ocv‘𝑊) & ⊢ 𝑌 = (0g‘𝑊) ⇒ ⊢ (𝐵 ∈ (OBasis‘𝑊) ↔ (𝑊 ∈ PreHil ∧ 𝐵 ⊆ 𝑉 ∧ (∀𝑥 ∈ 𝐵 ∀𝑦 ∈ 𝐵 (𝑥 , 𝑦) = if(𝑥 = 𝑦, 1 , 0 ) ∧ ( ⊥ ‘𝐵) = {𝑌}))) | ||
| Theorem | obsip 21679 | The inner product of two elements of an orthonormal basis. (Contributed by Mario Carneiro, 23-Oct-2015.) |
| ⊢ 𝑉 = (Base‘𝑊) & ⊢ , = (·𝑖‘𝑊) & ⊢ 𝐹 = (Scalar‘𝑊) & ⊢ 1 = (1r‘𝐹) & ⊢ 0 = (0g‘𝐹) ⇒ ⊢ ((𝐵 ∈ (OBasis‘𝑊) ∧ 𝑃 ∈ 𝐵 ∧ 𝑄 ∈ 𝐵) → (𝑃 , 𝑄) = if(𝑃 = 𝑄, 1 , 0 )) | ||
| Theorem | obsipid 21680 | A basis element has length one. (Contributed by Mario Carneiro, 23-Oct-2015.) |
| ⊢ , = (·𝑖‘𝑊) & ⊢ 𝐹 = (Scalar‘𝑊) & ⊢ 1 = (1r‘𝐹) ⇒ ⊢ ((𝐵 ∈ (OBasis‘𝑊) ∧ 𝐴 ∈ 𝐵) → (𝐴 , 𝐴) = 1 ) | ||
| Theorem | obsrcl 21681 | Reverse closure for an orthonormal basis. (Contributed by Mario Carneiro, 23-Oct-2015.) |
| ⊢ (𝐵 ∈ (OBasis‘𝑊) → 𝑊 ∈ PreHil) | ||
| Theorem | obsss 21682 | An orthonormal basis is a subset of the base set. (Contributed by Mario Carneiro, 23-Oct-2015.) |
| ⊢ 𝑉 = (Base‘𝑊) ⇒ ⊢ (𝐵 ∈ (OBasis‘𝑊) → 𝐵 ⊆ 𝑉) | ||
| Theorem | obsne0 21683 | A basis element is nonzero. (Contributed by Mario Carneiro, 23-Oct-2015.) |
| ⊢ 0 = (0g‘𝑊) ⇒ ⊢ ((𝐵 ∈ (OBasis‘𝑊) ∧ 𝐴 ∈ 𝐵) → 𝐴 ≠ 0 ) | ||
| Theorem | obsocv 21684 | An orthonormal basis has trivial orthocomplement. (Contributed by Mario Carneiro, 23-Oct-2015.) |
| ⊢ 0 = (0g‘𝑊) & ⊢ ⊥ = (ocv‘𝑊) ⇒ ⊢ (𝐵 ∈ (OBasis‘𝑊) → ( ⊥ ‘𝐵) = { 0 }) | ||
| Theorem | obs2ocv 21685 | The double orthocomplement (closure) of an orthonormal basis is the whole space. (Contributed by Mario Carneiro, 23-Oct-2015.) |
| ⊢ ⊥ = (ocv‘𝑊) & ⊢ 𝑉 = (Base‘𝑊) ⇒ ⊢ (𝐵 ∈ (OBasis‘𝑊) → ( ⊥ ‘( ⊥ ‘𝐵)) = 𝑉) | ||
| Theorem | obselocv 21686 | A basis element is in the orthocomplement of a subset of the basis iff it is not in the subset. (Contributed by Mario Carneiro, 23-Oct-2015.) |
| ⊢ ⊥ = (ocv‘𝑊) ⇒ ⊢ ((𝐵 ∈ (OBasis‘𝑊) ∧ 𝐶 ⊆ 𝐵 ∧ 𝐴 ∈ 𝐵) → (𝐴 ∈ ( ⊥ ‘𝐶) ↔ ¬ 𝐴 ∈ 𝐶)) | ||
| Theorem | obs2ss 21687 | A basis has no proper subsets that are also bases. (Contributed by Mario Carneiro, 23-Oct-2015.) |
| ⊢ ((𝐵 ∈ (OBasis‘𝑊) ∧ 𝐶 ∈ (OBasis‘𝑊) ∧ 𝐶 ⊆ 𝐵) → 𝐶 = 𝐵) | ||
| Theorem | obslbs 21688 | An orthogonal basis is a linear basis iff the span of the basis elements is closed (which is usually not true). (Contributed by Mario Carneiro, 29-Oct-2015.) |
| ⊢ 𝐽 = (LBasis‘𝑊) & ⊢ 𝑁 = (LSpan‘𝑊) & ⊢ 𝐶 = (ClSubSp‘𝑊) ⇒ ⊢ (𝐵 ∈ (OBasis‘𝑊) → (𝐵 ∈ 𝐽 ↔ (𝑁‘𝐵) ∈ 𝐶)) | ||
According to Wikipedia ("Linear algebra", 03-Mar-2019, https://en.wikipedia.org/wiki/Linear_algebra) "Linear algebra is the branch of mathematics concerning linear equations [...], linear functions [...] and their representations through matrices and vector spaces." Or according to the Merriam-Webster dictionary ("linear algebra", 12-Mar-2019, https://www.merriam-webster.com/dictionary/linear%20algebra) "Definition of linear algebra: a branch of mathematics that is concerned with mathematical structures closed under the operations of addition and scalar multiplication and that includes the theory of systems of linear equations, matrices, determinants, vector spaces, and linear transformations." Dealing with modules (over rings) instead of vector spaces (over fields) allows for a more unified approach. Therefore, linear equations, matrices, determinants, are usually regarded as "over a ring" in this part. Unless otherwise stated, the rings of scalars need not be commutative (see df-cring 20194), but the existence of a unity element is always assumed (our rings are unital, see df-ring 20193). For readers knowing vector spaces but unfamiliar with modules: the elements of a module are still called "vectors" and they still form a group under addition, with a zero vector as neutral element, like in a vector space. Like in a vector space, vectors can be multiplied by scalars, with the usual rules, the only difference being that the scalars are only required to form a ring, and not necessarily a field or a division ring. Note that any vector space is a (special kind of) module, so any theorem proved below for modules applies to any vector space. | ||
According to Wikipedia ("Direct sum of modules", 28-Mar-2019,
https://en.wikipedia.org/wiki/Direct_sum_of_modules) "Let R be a ring, and
{ Mi: i ∈ I } a family of left R-modules indexed by the set I.
The direct sum of {Mi} is then defined to be the set of all
sequences (αi) where αi ∈ Mi
and αi = 0 for cofinitely many indices i. (The direct product
is analogous but the indices do not need to cofinitely vanish.)". In this
definition, "cofinitely many" means "almost all" or "for all but finitely
many". Furthemore, "This set inherits the module structure via componentwise
addition and scalar multiplication. Explicitly, two such sequences α and
β can be added by writing (α + β)i =
αi + βi for all i (note that this is again
zero for all but finitely many indices), and such a sequence can be multiplied
with an element r from R by defining r(α)i =
(rα)i for all i.".
| ||
| Syntax | cdsmm 21689 | Class of module direct sum generator. |
| class ⊕m | ||
| Definition | df-dsmm 21690* | The direct sum of a family of Abelian groups or left modules is the induced group structure on finite linear combinations of elements, here represented as functions with finite support. (Contributed by Stefan O'Rear, 7-Jan-2015.) |
| ⊢ ⊕m = (𝑠 ∈ V, 𝑟 ∈ V ↦ ((𝑠Xs𝑟) ↾s {𝑓 ∈ X𝑥 ∈ dom 𝑟(Base‘(𝑟‘𝑥)) ∣ {𝑥 ∈ dom 𝑟 ∣ (𝑓‘𝑥) ≠ (0g‘(𝑟‘𝑥))} ∈ Fin})) | ||
| Theorem | reldmdsmm 21691 | The direct sum is a well-behaved binary operator. (Contributed by Stefan O'Rear, 7-Jan-2015.) |
| ⊢ Rel dom ⊕m | ||
| Theorem | dsmmval 21692* | Value of the module direct sum. (Contributed by Stefan O'Rear, 7-Jan-2015.) |
| ⊢ 𝐵 = {𝑓 ∈ (Base‘(𝑆Xs𝑅)) ∣ {𝑥 ∈ dom 𝑅 ∣ (𝑓‘𝑥) ≠ (0g‘(𝑅‘𝑥))} ∈ Fin} ⇒ ⊢ (𝑅 ∈ 𝑉 → (𝑆 ⊕m 𝑅) = ((𝑆Xs𝑅) ↾s 𝐵)) | ||
| Theorem | dsmmbase 21693* | Base set of the module direct sum. (Contributed by Stefan O'Rear, 7-Jan-2015.) |
| ⊢ 𝐵 = {𝑓 ∈ (Base‘(𝑆Xs𝑅)) ∣ {𝑥 ∈ dom 𝑅 ∣ (𝑓‘𝑥) ≠ (0g‘(𝑅‘𝑥))} ∈ Fin} ⇒ ⊢ (𝑅 ∈ 𝑉 → 𝐵 = (Base‘(𝑆 ⊕m 𝑅))) | ||
| Theorem | dsmmval2 21694 | Self-referential definition of the module direct sum. (Contributed by Stefan O'Rear, 7-Jan-2015.) (Revised by Stefan O'Rear, 6-May-2015.) |
| ⊢ 𝐵 = (Base‘(𝑆 ⊕m 𝑅)) ⇒ ⊢ (𝑆 ⊕m 𝑅) = ((𝑆Xs𝑅) ↾s 𝐵) | ||
| Theorem | dsmmbas2 21695* | Base set of the direct sum module using the fndmin 7034 abbreviation. (Contributed by Stefan O'Rear, 1-Feb-2015.) |
| ⊢ 𝑃 = (𝑆Xs𝑅) & ⊢ 𝐵 = {𝑓 ∈ (Base‘𝑃) ∣ dom (𝑓 ∖ (0g ∘ 𝑅)) ∈ Fin} ⇒ ⊢ ((𝑅 Fn 𝐼 ∧ 𝐼 ∈ 𝑉) → 𝐵 = (Base‘(𝑆 ⊕m 𝑅))) | ||
| Theorem | dsmmfi 21696 | For finite products, the direct sum is just the module product. See also the observation in [Lang] p. 129. (Contributed by Stefan O'Rear, 1-Feb-2015.) |
| ⊢ ((𝑅 Fn 𝐼 ∧ 𝐼 ∈ Fin) → (𝑆 ⊕m 𝑅) = (𝑆Xs𝑅)) | ||
| Theorem | dsmmelbas 21697* | Membership in the finitely supported hull of a structure product in terms of the index set. (Contributed by Stefan O'Rear, 11-Jan-2015.) |
| ⊢ 𝑃 = (𝑆Xs𝑅) & ⊢ 𝐶 = (𝑆 ⊕m 𝑅) & ⊢ 𝐵 = (Base‘𝑃) & ⊢ 𝐻 = (Base‘𝐶) & ⊢ (𝜑 → 𝐼 ∈ 𝑉) & ⊢ (𝜑 → 𝑅 Fn 𝐼) ⇒ ⊢ (𝜑 → (𝑋 ∈ 𝐻 ↔ (𝑋 ∈ 𝐵 ∧ {𝑎 ∈ 𝐼 ∣ (𝑋‘𝑎) ≠ (0g‘(𝑅‘𝑎))} ∈ Fin))) | ||
| Theorem | dsmm0cl 21698 | The all-zero vector is contained in the finite hull, since its support is empty and therefore finite. This theorem along with the next one effectively proves that the finite hull is a "submonoid", although that does not exist as a defined concept yet. (Contributed by Stefan O'Rear, 11-Jan-2015.) |
| ⊢ 𝑃 = (𝑆Xs𝑅) & ⊢ 𝐻 = (Base‘(𝑆 ⊕m 𝑅)) & ⊢ (𝜑 → 𝐼 ∈ 𝑊) & ⊢ (𝜑 → 𝑆 ∈ 𝑉) & ⊢ (𝜑 → 𝑅:𝐼⟶Mnd) & ⊢ 0 = (0g‘𝑃) ⇒ ⊢ (𝜑 → 0 ∈ 𝐻) | ||
| Theorem | dsmmacl 21699 | The finite hull is closed under addition. (Contributed by Stefan O'Rear, 11-Jan-2015.) |
| ⊢ 𝑃 = (𝑆Xs𝑅) & ⊢ 𝐻 = (Base‘(𝑆 ⊕m 𝑅)) & ⊢ (𝜑 → 𝐼 ∈ 𝑊) & ⊢ (𝜑 → 𝑆 ∈ 𝑉) & ⊢ (𝜑 → 𝑅:𝐼⟶Mnd) & ⊢ (𝜑 → 𝐽 ∈ 𝐻) & ⊢ (𝜑 → 𝐾 ∈ 𝐻) & ⊢ + = (+g‘𝑃) ⇒ ⊢ (𝜑 → (𝐽 + 𝐾) ∈ 𝐻) | ||
| Theorem | prdsinvgd2 21700 | Negation of a single coordinate in a structure product. (Contributed by Stefan O'Rear, 11-Jan-2015.) |
| ⊢ 𝑌 = (𝑆Xs𝑅) & ⊢ (𝜑 → 𝐼 ∈ 𝑊) & ⊢ (𝜑 → 𝑆 ∈ 𝑉) & ⊢ (𝜑 → 𝑅:𝐼⟶Grp) & ⊢ 𝐵 = (Base‘𝑌) & ⊢ 𝑁 = (invg‘𝑌) & ⊢ (𝜑 → 𝑋 ∈ 𝐵) & ⊢ (𝜑 → 𝐽 ∈ 𝐼) ⇒ ⊢ (𝜑 → ((𝑁‘𝑋)‘𝐽) = ((invg‘(𝑅‘𝐽))‘(𝑋‘𝐽))) | ||
| < Previous Next > |
| Copyright terms: Public domain | < Previous Next > |