Home | Metamath
Proof Explorer Theorem List (p. 170 of 466) | < 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: | Metamath Proof Explorer
(1-29289) |
Hilbert Space Explorer
(29290-30812) |
Users' Mathboxes
(30813-46532) |
Type | Label | Description |
---|---|---|
Statement | ||
Theorem | fveqprc 16901 | Lemma for showing the equality of values for functions like slot extractors 𝐸 at a proper class. Extracted from several former proofs of lemmas like zlmlem 20727. (Contributed by AV, 31-Oct-2024.) |
⊢ (𝐸‘∅) = ∅ & ⊢ 𝑌 = (𝐹‘𝑋) ⇒ ⊢ (¬ 𝑋 ∈ V → (𝐸‘𝑋) = (𝐸‘𝑌)) | ||
Theorem | oveqprc 16902 | Lemma for showing the equality of values for functions like slot extractors 𝐸 at a proper class. Extracted from several former proofs of lemmas like resvlem 31539. (Contributed by AV, 31-Oct-2024.) |
⊢ (𝐸‘∅) = ∅ & ⊢ 𝑍 = (𝑋𝑂𝑌) & ⊢ Rel dom 𝑂 ⇒ ⊢ (¬ 𝑋 ∈ V → (𝐸‘𝑋) = (𝐸‘𝑍)) | ||
The structure component index extractor ndx, defined in this subsection, is used to get the numeric argument from a defined structure component extractor such as df-base 16922 (see ndxarg 16906). For each defined structure component extractor, there should be a corresponding specific theorem providing its index, like basendx 16930. The usage of these theorems, however, is discouraged since the particular value for the index is an implementation detail. It is generally sufficient to work with (Base‘ndx) instead of the hard-coded index value, and use theorems such as baseid 16924 and basendxnplusgndx 17001. The main circumstance in which it is necessary to look at indices directly is when showing that a set of indices are disjoint (for example in proofs such as cznabel 45523, based on setsnid 16919) or even ordered (in proofs such as lmodstr 17044). The requirement that the indices are distinct is necessary for sets of ordered pairs to be extensible structures, whereas the ordering allows for proofs avoiding the usage of quadradically many inequalities (compare cnfldfun 20618 with cnfldfunALT 20619). As for the inequalities, it is recommended to provide them explicitly as theorems like basendxnplusgndx 17001, whenever they are required. Since these theorems use discouraged slot theorems, they should be placed near the definition of a slot (within the same subsection), so that the range of usages of discouraged theorems is tightly limited. Although there could be quadradically many of them in the total number of indices, much less are actually available (and not much more are expected). As for the ordering, there are some theorems like basendxltplusgndx 17000 providing the less-than relationship between two indices. These theorems are also proved by discouraged theorems, so they should be placed near the definition of a slot (within the same subsection), too. However, since such theorems are rarely used (in structure building theorems *str like rngstr 17017), it is not recommended to provide explicit theorems for all of them, but to use the (discouraged) *ndx theorems as in lmodstr 17044. Therefore, *str theorems generally depend on the hard-coded values of the indices. | ||
Syntax | cnx 16903 | Extend class notation with the structure component index extractor. |
class ndx | ||
Definition | df-ndx 16904 | Define the structure component index extractor. See Theorem ndxarg 16906 to understand its purpose. The restriction to ℕ ensures that ndx is a set. The restriction to some set is necessary since I is a proper class. In principle, we could have chosen ℂ or (if we revise all structure component definitions such as df-base 16922) another set such as the set of finite ordinals ω (df-om 7722). (Contributed by NM, 4-Sep-2011.) |
⊢ ndx = ( I ↾ ℕ) | ||
Theorem | wunndx 16905 | Closure of the index extractor in an infinite weak universe. (Contributed by Mario Carneiro, 12-Jan-2017.) |
⊢ (𝜑 → 𝑈 ∈ WUni) & ⊢ (𝜑 → ω ∈ 𝑈) ⇒ ⊢ (𝜑 → ndx ∈ 𝑈) | ||
Theorem | ndxarg 16906 | Get the numeric argument from a defined structure component extractor such as df-base 16922. (Contributed by Mario Carneiro, 6-Oct-2013.) |
⊢ 𝐸 = Slot 𝑁 & ⊢ 𝑁 ∈ ℕ ⇒ ⊢ (𝐸‘ndx) = 𝑁 | ||
Theorem | ndxid 16907 |
A structure component extractor is defined by its own index. This
theorem, together with strfv 16914 below, is useful for avoiding direct
reference to the hard-coded numeric index in component extractor
definitions, such as the 1 in df-base 16922 and the ;10 in
df-ple 16991, making it easier to change should the need
arise.
For example, we can refer to a specific poset with base set 𝐵 and order relation 𝐿 using {〈(Base‘ndx), 𝐵〉, 〈(le‘ndx), 𝐿〉} rather than {〈1, 𝐵〉, 〈;10, 𝐿〉}. The latter, while shorter to state, requires revision if we later change ;10 to some other number, and it may also be harder to remember. (Contributed by NM, 19-Oct-2012.) (Revised by Mario Carneiro, 6-Oct-2013.) (Proof shortened by BJ, 27-Dec-2021.) |
⊢ 𝐸 = Slot 𝑁 & ⊢ 𝑁 ∈ ℕ ⇒ ⊢ 𝐸 = Slot (𝐸‘ndx) | ||
Theorem | strndxid 16908 | The value of a structure component extractor is the value of the corresponding slot of the structure. (Contributed by AV, 13-Mar-2020.) (New usage is discouraged.) Use strfvnd 16895 directly with 𝑁 set to (𝐸‘ndx) if possible. |
⊢ (𝜑 → 𝑆 ∈ 𝑉) & ⊢ 𝐸 = Slot 𝑁 & ⊢ 𝑁 ∈ ℕ ⇒ ⊢ (𝜑 → (𝑆‘(𝐸‘ndx)) = (𝐸‘𝑆)) | ||
Theorem | setsidvald 16909 |
Value of the structure replacement function, deduction version.
Hint: Do not substitute 𝑁 by a specific (positive) integer to be independent of a hard-coded index value. Often, (𝐸‘ndx) can be used instead of 𝑁. (Contributed by AV, 14-Mar-2020.) (Revised by AV, 17-Oct-2024.) |
⊢ 𝐸 = Slot 𝑁 & ⊢ (𝜑 → 𝑆 ∈ 𝑉) & ⊢ (𝜑 → Fun 𝑆) & ⊢ (𝜑 → 𝑁 ∈ dom 𝑆) ⇒ ⊢ (𝜑 → 𝑆 = (𝑆 sSet 〈𝑁, (𝐸‘𝑆)〉)) | ||
Theorem | setsidvaldOLD 16910 | Obsolete version of setsidvald 16909 as of 17-Oct-2024. (Contributed by AV, 14-Mar-2020.) (New usage is discouraged.) (Proof modification is discouraged.) |
⊢ 𝐸 = Slot 𝑁 & ⊢ 𝑁 ∈ ℕ & ⊢ (𝜑 → 𝑆 ∈ 𝑉) & ⊢ (𝜑 → Fun 𝑆) & ⊢ (𝜑 → (𝐸‘ndx) ∈ dom 𝑆) ⇒ ⊢ (𝜑 → 𝑆 = (𝑆 sSet 〈(𝐸‘ndx), (𝐸‘𝑆)〉)) | ||
Theorem | strfvd 16911 | Deduction version of strfv 16914. (Contributed by Mario Carneiro, 15-Nov-2014.) |
⊢ 𝐸 = Slot (𝐸‘ndx) & ⊢ (𝜑 → 𝑆 ∈ 𝑉) & ⊢ (𝜑 → Fun 𝑆) & ⊢ (𝜑 → 〈(𝐸‘ndx), 𝐶〉 ∈ 𝑆) ⇒ ⊢ (𝜑 → 𝐶 = (𝐸‘𝑆)) | ||
Theorem | strfv2d 16912 | Deduction version of strfv2 16913. (Contributed by Mario Carneiro, 30-Apr-2015.) |
⊢ 𝐸 = Slot (𝐸‘ndx) & ⊢ (𝜑 → 𝑆 ∈ 𝑉) & ⊢ (𝜑 → Fun ◡◡𝑆) & ⊢ (𝜑 → 〈(𝐸‘ndx), 𝐶〉 ∈ 𝑆) & ⊢ (𝜑 → 𝐶 ∈ 𝑊) ⇒ ⊢ (𝜑 → 𝐶 = (𝐸‘𝑆)) | ||
Theorem | strfv2 16913 | A variation on strfv 16914 to avoid asserting that 𝑆 itself is a function, which involves sethood of all the ordered pair components of 𝑆. (Contributed by Mario Carneiro, 30-Apr-2015.) |
⊢ 𝑆 ∈ V & ⊢ Fun ◡◡𝑆 & ⊢ 𝐸 = Slot (𝐸‘ndx) & ⊢ 〈(𝐸‘ndx), 𝐶〉 ∈ 𝑆 ⇒ ⊢ (𝐶 ∈ 𝑉 → 𝐶 = (𝐸‘𝑆)) | ||
Theorem | strfv 16914 | Extract a structure component 𝐶 (such as the base set) from a structure 𝑆 (such as a member of Poset, df-poset 18040) with a component extractor 𝐸 (such as the base set extractor df-base 16922). By virtue of ndxid 16907, this can be done without having to refer to the hard-coded numeric index of 𝐸. (Contributed by Mario Carneiro, 6-Oct-2013.) (Revised by Mario Carneiro, 29-Aug-2015.) |
⊢ 𝑆 Struct 𝑋 & ⊢ 𝐸 = Slot (𝐸‘ndx) & ⊢ {〈(𝐸‘ndx), 𝐶〉} ⊆ 𝑆 ⇒ ⊢ (𝐶 ∈ 𝑉 → 𝐶 = (𝐸‘𝑆)) | ||
Theorem | strfv3 16915 | Variant on strfv 16914 for large structures. (Contributed by Mario Carneiro, 10-Jan-2017.) |
⊢ (𝜑 → 𝑈 = 𝑆) & ⊢ 𝑆 Struct 𝑋 & ⊢ 𝐸 = Slot (𝐸‘ndx) & ⊢ {〈(𝐸‘ndx), 𝐶〉} ⊆ 𝑆 & ⊢ (𝜑 → 𝐶 ∈ 𝑉) & ⊢ 𝐴 = (𝐸‘𝑈) ⇒ ⊢ (𝜑 → 𝐴 = 𝐶) | ||
Theorem | strssd 16916 | Deduction version of strss 16917. (Contributed by Mario Carneiro, 15-Nov-2014.) (Revised by Mario Carneiro, 30-Apr-2015.) |
⊢ 𝐸 = Slot (𝐸‘ndx) & ⊢ (𝜑 → 𝑇 ∈ 𝑉) & ⊢ (𝜑 → Fun 𝑇) & ⊢ (𝜑 → 𝑆 ⊆ 𝑇) & ⊢ (𝜑 → 〈(𝐸‘ndx), 𝐶〉 ∈ 𝑆) ⇒ ⊢ (𝜑 → (𝐸‘𝑇) = (𝐸‘𝑆)) | ||
Theorem | strss 16917 | Propagate component extraction to a structure 𝑇 from a subset structure 𝑆. (Contributed by Mario Carneiro, 11-Oct-2013.) (Revised by Mario Carneiro, 15-Jan-2014.) |
⊢ 𝑇 ∈ V & ⊢ Fun 𝑇 & ⊢ 𝑆 ⊆ 𝑇 & ⊢ 𝐸 = Slot (𝐸‘ndx) & ⊢ 〈(𝐸‘ndx), 𝐶〉 ∈ 𝑆 ⇒ ⊢ (𝐸‘𝑇) = (𝐸‘𝑆) | ||
Theorem | setsid 16918 | Value of the structure replacement function at a replaced index. (Contributed by Mario Carneiro, 1-Dec-2014.) (Revised by Mario Carneiro, 30-Apr-2015.) |
⊢ 𝐸 = Slot (𝐸‘ndx) ⇒ ⊢ ((𝑊 ∈ 𝐴 ∧ 𝐶 ∈ 𝑉) → 𝐶 = (𝐸‘(𝑊 sSet 〈(𝐸‘ndx), 𝐶〉))) | ||
Theorem | setsnid 16919 | Value of the structure replacement function at an untouched index. (Contributed by Mario Carneiro, 1-Dec-2014.) (Revised by Mario Carneiro, 30-Apr-2015.) (Proof shortened by AV, 7-Nov-2024.) |
⊢ 𝐸 = Slot (𝐸‘ndx) & ⊢ (𝐸‘ndx) ≠ 𝐷 ⇒ ⊢ (𝐸‘𝑊) = (𝐸‘(𝑊 sSet 〈𝐷, 𝐶〉)) | ||
Theorem | setsnidOLD 16920 | Obsolete proof of setsnid 16919 as of 7-Nov-2024. Value of the structure replacement function at an untouched index. (Contributed by Mario Carneiro, 1-Dec-2014.) (Revised by Mario Carneiro, 30-Apr-2015.) (New usage is discouraged.) (Proof modification is discouraged.) |
⊢ 𝐸 = Slot (𝐸‘ndx) & ⊢ (𝐸‘ndx) ≠ 𝐷 ⇒ ⊢ (𝐸‘𝑊) = (𝐸‘(𝑊 sSet 〈𝐷, 𝐶〉)) | ||
Syntax | cbs 16921 | Extend class notation with the class of all base set extractors. |
class Base | ||
Definition | df-base 16922 | Define the base set (also called underlying set, ground set, carrier set, or carrier) extractor for extensible structures. (Contributed by NM, 4-Sep-2011.) (Revised by Mario Carneiro, 14-Aug-2015.) Use its index-independent form baseid 16924 instead. (New usage is discouraged.) |
⊢ Base = Slot 1 | ||
Theorem | baseval 16923 | Value of the base set extractor. (Normally it is preferred to work with (Base‘ndx) rather than the hard-coded 1 in order to make structure theorems portable. This is an example of how to obtain it when needed.) (New usage is discouraged.) (Contributed by NM, 4-Sep-2011.) |
⊢ 𝐾 ∈ V ⇒ ⊢ (Base‘𝐾) = (𝐾‘1) | ||
Theorem | baseid 16924 | Utility theorem: index-independent form of df-base 16922. (Contributed by NM, 20-Oct-2012.) |
⊢ Base = Slot (Base‘ndx) | ||
Theorem | basfn 16925 | The base set extractor is a function on V. (Contributed by Stefan O'Rear, 8-Jul-2015.) |
⊢ Base Fn V | ||
Theorem | base0 16926 | The base set of the empty structure. (Contributed by David A. Wheeler, 7-Jul-2016.) |
⊢ ∅ = (Base‘∅) | ||
Theorem | elbasfv 16927 | Utility theorem: reverse closure for any structure defined as a function. (Contributed by Stefan O'Rear, 24-Aug-2015.) |
⊢ 𝑆 = (𝐹‘𝑍) & ⊢ 𝐵 = (Base‘𝑆) ⇒ ⊢ (𝑋 ∈ 𝐵 → 𝑍 ∈ V) | ||
Theorem | elbasov 16928 | Utility theorem: reverse closure for any structure defined as a two-argument function. (Contributed by Mario Carneiro, 3-Oct-2015.) |
⊢ Rel dom 𝑂 & ⊢ 𝑆 = (𝑋𝑂𝑌) & ⊢ 𝐵 = (Base‘𝑆) ⇒ ⊢ (𝐴 ∈ 𝐵 → (𝑋 ∈ V ∧ 𝑌 ∈ V)) | ||
Theorem | strov2rcl 16929 | Partial reverse closure for any structure defined as a two-argument function. (Contributed by Stefan O'Rear, 27-Mar-2015.) (Proof shortened by AV, 2-Dec-2019.) |
⊢ 𝑆 = (𝐼𝐹𝑅) & ⊢ 𝐵 = (Base‘𝑆) & ⊢ Rel dom 𝐹 ⇒ ⊢ (𝑋 ∈ 𝐵 → 𝐼 ∈ V) | ||
Theorem | basendx 16930 | Index value of the base set extractor. (Contributed by Mario Carneiro, 2-Aug-2013.) Use of this theorem is discouraged since the particular value 1 for the index is an implementation detail, see section header comment mmtheorems.html#cnx for more information. (New usage is discouraged.) |
⊢ (Base‘ndx) = 1 | ||
Theorem | basendxnn 16931 | The index value of the base set extractor is a positive integer. This property should be ensured for every concrete coding because otherwise it could not be used in an extensible structure (slots must be positive integers). (Contributed by AV, 23-Sep-2020.) (Proof shortened by AV, 13-Oct-2024.) |
⊢ (Base‘ndx) ∈ ℕ | ||
Theorem | basendxnnOLD 16932 | Obsolete proof of basendxnn 16931 as of 13-Oct-2024. (Contributed by AV, 23-Sep-2020.) (Proof modification is discouraged.) (New usage is discouraged.) |
⊢ (Base‘ndx) ∈ ℕ | ||
Theorem | basndxelwund 16933 | The index of the base set is an element in a weak universe containing the natural numbers. Formerly part of proof for 1strwun 16941. (Contributed by AV, 27-Mar-2020.) (Revised by AV, 17-Oct-2024.) |
⊢ (𝜑 → 𝑈 ∈ WUni) & ⊢ (𝜑 → ω ∈ 𝑈) ⇒ ⊢ (𝜑 → (Base‘ndx) ∈ 𝑈) | ||
Theorem | basprssdmsets 16934 | The pair of the base index and another index is a subset of the domain of the structure obtained by replacing/adding a slot at the other index in a structure having a base slot. (Contributed by AV, 7-Jun-2021.) (Revised by AV, 16-Nov-2021.) |
⊢ (𝜑 → 𝑆 Struct 𝑋) & ⊢ (𝜑 → 𝐼 ∈ 𝑈) & ⊢ (𝜑 → 𝐸 ∈ 𝑊) & ⊢ (𝜑 → (Base‘ndx) ∈ dom 𝑆) ⇒ ⊢ (𝜑 → {(Base‘ndx), 𝐼} ⊆ dom (𝑆 sSet 〈𝐼, 𝐸〉)) | ||
Theorem | opelstrbas 16935 | The base set of a structure with a base set. (Contributed by AV, 10-Nov-2021.) |
⊢ (𝜑 → 𝑆 Struct 𝑋) & ⊢ (𝜑 → 𝑉 ∈ 𝑌) & ⊢ (𝜑 → 〈(Base‘ndx), 𝑉〉 ∈ 𝑆) ⇒ ⊢ (𝜑 → 𝑉 = (Base‘𝑆)) | ||
Theorem | 1strstr 16936 | A constructed one-slot structure. Depending on hard-coded index. Use 1strstr1 16937 instead. (Contributed by AV, 27-Mar-2020.) (New usage is discouraged.) |
⊢ 𝐺 = {〈(Base‘ndx), 𝐵〉} ⇒ ⊢ 𝐺 Struct 〈1, 1〉 | ||
Theorem | 1strstr1 16937 | A constructed one-slot structure. (Contributed by AV, 15-Nov-2024.) |
⊢ 𝐺 = {〈(Base‘ndx), 𝐵〉} ⇒ ⊢ 𝐺 Struct 〈(Base‘ndx), (Base‘ndx)〉 | ||
Theorem | 1strbas 16938 | The base set of a constructed one-slot structure. (Contributed by AV, 27-Mar-2020.) (Proof shortened by AV, 15-Nov-2024.) |
⊢ 𝐺 = {〈(Base‘ndx), 𝐵〉} ⇒ ⊢ (𝐵 ∈ 𝑉 → 𝐵 = (Base‘𝐺)) | ||
Theorem | 1strbasOLD 16939 | Obsolete proof of 1strbas 16938 as of 15-Nov-2024. The base set of a constructed one-slot structure. (Contributed by AV, 27-Mar-2020.) (Proof modification is discouraged.) (New usage is discouraged.) |
⊢ 𝐺 = {〈(Base‘ndx), 𝐵〉} ⇒ ⊢ (𝐵 ∈ 𝑉 → 𝐵 = (Base‘𝐺)) | ||
Theorem | 1strwunbndx 16940 | A constructed one-slot structure in a weak universe containing the index of the base set extractor. (Contributed by AV, 27-Mar-2020.) |
⊢ 𝐺 = {〈(Base‘ndx), 𝐵〉} & ⊢ (𝜑 → 𝑈 ∈ WUni) & ⊢ (𝜑 → (Base‘ndx) ∈ 𝑈) ⇒ ⊢ ((𝜑 ∧ 𝐵 ∈ 𝑈) → 𝐺 ∈ 𝑈) | ||
Theorem | 1strwun 16941 | A constructed one-slot structure in a weak universe. (Contributed by AV, 27-Mar-2020.) (Proof shortened by AV, 17-Oct-2024.) |
⊢ 𝐺 = {〈(Base‘ndx), 𝐵〉} & ⊢ (𝜑 → 𝑈 ∈ WUni) & ⊢ (𝜑 → ω ∈ 𝑈) ⇒ ⊢ ((𝜑 ∧ 𝐵 ∈ 𝑈) → 𝐺 ∈ 𝑈) | ||
Theorem | 1strwunOLD 16942 | Obsolete version of 1strwun 16941 as of 17-Oct-2024. A constructed one-slot structure in a weak universe. (Contributed by AV, 27-Mar-2020.) (Proof modification is discouraged.) (New usage is discouraged.) |
⊢ 𝐺 = {〈(Base‘ndx), 𝐵〉} & ⊢ (𝜑 → 𝑈 ∈ WUni) & ⊢ (𝜑 → ω ∈ 𝑈) ⇒ ⊢ ((𝜑 ∧ 𝐵 ∈ 𝑈) → 𝐺 ∈ 𝑈) | ||
Theorem | 2strstr 16943 | A constructed two-slot structure. Depending on hard-coded indices. Use 2strstr1 16946 instead. (Contributed by Mario Carneiro, 29-Aug-2015.) (New usage is discouraged.) |
⊢ 𝐺 = {〈(Base‘ndx), 𝐵〉, 〈(𝐸‘ndx), + 〉} & ⊢ 𝐸 = Slot 𝑁 & ⊢ 1 < 𝑁 & ⊢ 𝑁 ∈ ℕ ⇒ ⊢ 𝐺 Struct 〈1, 𝑁〉 | ||
Theorem | 2strbas 16944 | The base set of a constructed two-slot structure. (Contributed by Mario Carneiro, 29-Aug-2015.) Use the index-independent version 2strbas1 16948 instead. (New usage is discouraged.) |
⊢ 𝐺 = {〈(Base‘ndx), 𝐵〉, 〈(𝐸‘ndx), + 〉} & ⊢ 𝐸 = Slot 𝑁 & ⊢ 1 < 𝑁 & ⊢ 𝑁 ∈ ℕ ⇒ ⊢ (𝐵 ∈ 𝑉 → 𝐵 = (Base‘𝐺)) | ||
Theorem | 2strop 16945 | The other slot of a constructed two-slot structure. (Contributed by Mario Carneiro, 29-Aug-2015.) Use the index-independent version 2strop1 16949 instead. (New usage is discouraged.) |
⊢ 𝐺 = {〈(Base‘ndx), 𝐵〉, 〈(𝐸‘ndx), + 〉} & ⊢ 𝐸 = Slot 𝑁 & ⊢ 1 < 𝑁 & ⊢ 𝑁 ∈ ℕ ⇒ ⊢ ( + ∈ 𝑉 → + = (𝐸‘𝐺)) | ||
Theorem | 2strstr1 16946 | A constructed two-slot structure. Version of 2strstr 16943 not depending on the hard-coded index value of the base set. (Contributed by AV, 22-Sep-2020.) (Proof shortened by AV, 17-Oct-2024.) |
⊢ 𝐺 = {〈(Base‘ndx), 𝐵〉, 〈𝑁, + 〉} & ⊢ (Base‘ndx) < 𝑁 & ⊢ 𝑁 ∈ ℕ ⇒ ⊢ 𝐺 Struct 〈(Base‘ndx), 𝑁〉 | ||
Theorem | 2strstr1OLD 16947 | Obsolete version of 2strstr1 16946 as of 27-Oct-2024. A constructed two-slot structure. Version of 2strstr 16943 not depending on the hard-coded index value of the base set. (Contributed by AV, 22-Sep-2020.) (Proof modification is discouraged.) (New usage is discouraged.) |
⊢ 𝐺 = {〈(Base‘ndx), 𝐵〉, 〈𝑁, + 〉} & ⊢ (Base‘ndx) < 𝑁 & ⊢ 𝑁 ∈ ℕ ⇒ ⊢ 𝐺 Struct 〈(Base‘ndx), 𝑁〉 | ||
Theorem | 2strbas1 16948 | The base set of a constructed two-slot structure. Version of 2strbas 16944 not depending on the hard-coded index value of the base set. (Contributed by AV, 22-Sep-2020.) |
⊢ 𝐺 = {〈(Base‘ndx), 𝐵〉, 〈𝑁, + 〉} & ⊢ (Base‘ndx) < 𝑁 & ⊢ 𝑁 ∈ ℕ ⇒ ⊢ (𝐵 ∈ 𝑉 → 𝐵 = (Base‘𝐺)) | ||
Theorem | 2strop1 16949 | The other slot of a constructed two-slot structure. Version of 2strop 16945 not depending on the hard-coded index value of the base set. (Contributed by AV, 22-Sep-2020.) |
⊢ 𝐺 = {〈(Base‘ndx), 𝐵〉, 〈𝑁, + 〉} & ⊢ (Base‘ndx) < 𝑁 & ⊢ 𝑁 ∈ ℕ & ⊢ 𝐸 = Slot 𝑁 ⇒ ⊢ ( + ∈ 𝑉 → + = (𝐸‘𝐺)) | ||
Syntax | cress 16950 | Extend class notation with the extensible structure builder restriction operator. |
class ↾s | ||
Definition | df-ress 16951* |
Define a multifunction restriction operator for extensible structures,
which can be used to turn statements about rings into statements about
subrings, modules into submodules, etc. This definition knows nothing
about individual structures and merely truncates the Base set while
leaving operators alone; individual kinds of structures will need to
handle this behavior, by ignoring operators' values outside the range
(like Ring), defining a function using the base
set and applying
that (like TopGrp), or explicitly truncating the
slot before use
(like MetSp).
(Credit for this operator goes to Mario Carneiro.) See ressbas 16956 for the altered base set, and resseqnbas 16960 (subrg0 20040, ressplusg 17009, subrg1 20043, ressmulr 17026) for the (un)altered other operations. (Contributed by Stefan O'Rear, 29-Nov-2014.) |
⊢ ↾s = (𝑤 ∈ V, 𝑥 ∈ V ↦ if((Base‘𝑤) ⊆ 𝑥, 𝑤, (𝑤 sSet 〈(Base‘ndx), (𝑥 ∩ (Base‘𝑤))〉))) | ||
Theorem | reldmress 16952 | The structure restriction is a proper operator, so it can be used with ovprc1 7323. (Contributed by Stefan O'Rear, 29-Nov-2014.) |
⊢ Rel dom ↾s | ||
Theorem | ressval 16953 | Value of structure restriction. (Contributed by Stefan O'Rear, 29-Nov-2014.) |
⊢ 𝑅 = (𝑊 ↾s 𝐴) & ⊢ 𝐵 = (Base‘𝑊) ⇒ ⊢ ((𝑊 ∈ 𝑋 ∧ 𝐴 ∈ 𝑌) → 𝑅 = if(𝐵 ⊆ 𝐴, 𝑊, (𝑊 sSet 〈(Base‘ndx), (𝐴 ∩ 𝐵)〉))) | ||
Theorem | ressid2 16954 | General behavior of trivial restriction. (Contributed by Stefan O'Rear, 29-Nov-2014.) |
⊢ 𝑅 = (𝑊 ↾s 𝐴) & ⊢ 𝐵 = (Base‘𝑊) ⇒ ⊢ ((𝐵 ⊆ 𝐴 ∧ 𝑊 ∈ 𝑋 ∧ 𝐴 ∈ 𝑌) → 𝑅 = 𝑊) | ||
Theorem | ressval2 16955 | Value of nontrivial structure restriction. (Contributed by Stefan O'Rear, 29-Nov-2014.) |
⊢ 𝑅 = (𝑊 ↾s 𝐴) & ⊢ 𝐵 = (Base‘𝑊) ⇒ ⊢ ((¬ 𝐵 ⊆ 𝐴 ∧ 𝑊 ∈ 𝑋 ∧ 𝐴 ∈ 𝑌) → 𝑅 = (𝑊 sSet 〈(Base‘ndx), (𝐴 ∩ 𝐵)〉)) | ||
Theorem | ressbas 16956 | Base set of a structure restriction. (Contributed by Stefan O'Rear, 26-Nov-2014.) (Proof shortened by AV, 7-Nov-2024.) |
⊢ 𝑅 = (𝑊 ↾s 𝐴) & ⊢ 𝐵 = (Base‘𝑊) ⇒ ⊢ (𝐴 ∈ 𝑉 → (𝐴 ∩ 𝐵) = (Base‘𝑅)) | ||
Theorem | ressbasOLD 16957 | Obsolete proof of ressbas 16956 as of 7-Nov-2024. Base set of a structure restriction. (Contributed by Stefan O'Rear, 26-Nov-2014.) (New usage is discouraged.) (Proof modification is discouraged.) |
⊢ 𝑅 = (𝑊 ↾s 𝐴) & ⊢ 𝐵 = (Base‘𝑊) ⇒ ⊢ (𝐴 ∈ 𝑉 → (𝐴 ∩ 𝐵) = (Base‘𝑅)) | ||
Theorem | ressbas2 16958 | Base set of a structure restriction. (Contributed by Mario Carneiro, 2-Dec-2014.) |
⊢ 𝑅 = (𝑊 ↾s 𝐴) & ⊢ 𝐵 = (Base‘𝑊) ⇒ ⊢ (𝐴 ⊆ 𝐵 → 𝐴 = (Base‘𝑅)) | ||
Theorem | ressbasss 16959 | The base set of a restriction is a subset of the base set of the original structure. (Contributed by Stefan O'Rear, 27-Nov-2014.) (Revised by Mario Carneiro, 30-Apr-2015.) |
⊢ 𝑅 = (𝑊 ↾s 𝐴) & ⊢ 𝐵 = (Base‘𝑊) ⇒ ⊢ (Base‘𝑅) ⊆ 𝐵 | ||
Theorem | resseqnbas 16960 | The components of an extensible structure except the base set remain unchanged on a structure restriction. (Contributed by Mario Carneiro, 26-Nov-2014.) (Revised by Mario Carneiro, 2-Dec-2014.) (Revised by AV, 19-Oct-2024.) |
⊢ 𝑅 = (𝑊 ↾s 𝐴) & ⊢ 𝐶 = (𝐸‘𝑊) & ⊢ 𝐸 = Slot (𝐸‘ndx) & ⊢ (𝐸‘ndx) ≠ (Base‘ndx) ⇒ ⊢ (𝐴 ∈ 𝑉 → 𝐶 = (𝐸‘𝑅)) | ||
Theorem | resslemOLD 16961 | Obsolete version of resseqnbas 16960 as of 21-Oct-2024. (Contributed by Mario Carneiro, 26-Nov-2014.) (Revised by Mario Carneiro, 2-Dec-2014.) (Proof modification is discouraged.) (New usage is discouraged.) |
⊢ 𝑅 = (𝑊 ↾s 𝐴) & ⊢ 𝐶 = (𝐸‘𝑊) & ⊢ 𝐸 = Slot 𝑁 & ⊢ 𝑁 ∈ ℕ & ⊢ 1 < 𝑁 ⇒ ⊢ (𝐴 ∈ 𝑉 → 𝐶 = (𝐸‘𝑅)) | ||
Theorem | ress0 16962 | All restrictions of the null set are trivial. (Contributed by Stefan O'Rear, 29-Nov-2014.) (Revised by Mario Carneiro, 30-Apr-2015.) |
⊢ (∅ ↾s 𝐴) = ∅ | ||
Theorem | ressid 16963 | Behavior of trivial restriction. (Contributed by Stefan O'Rear, 29-Nov-2014.) |
⊢ 𝐵 = (Base‘𝑊) ⇒ ⊢ (𝑊 ∈ 𝑋 → (𝑊 ↾s 𝐵) = 𝑊) | ||
Theorem | ressinbas 16964 | Restriction only cares about the part of the second set which intersects the base of the first. (Contributed by Stefan O'Rear, 29-Nov-2014.) |
⊢ 𝐵 = (Base‘𝑊) ⇒ ⊢ (𝐴 ∈ 𝑋 → (𝑊 ↾s 𝐴) = (𝑊 ↾s (𝐴 ∩ 𝐵))) | ||
Theorem | ressval3d 16965 | Value of structure restriction, deduction version. (Contributed by AV, 14-Mar-2020.) (Revised by AV, 3-Jul-2022.) (Proof shortened by AV, 17-Oct-2024.) |
⊢ 𝑅 = (𝑆 ↾s 𝐴) & ⊢ 𝐵 = (Base‘𝑆) & ⊢ 𝐸 = (Base‘ndx) & ⊢ (𝜑 → 𝑆 ∈ 𝑉) & ⊢ (𝜑 → Fun 𝑆) & ⊢ (𝜑 → 𝐸 ∈ dom 𝑆) & ⊢ (𝜑 → 𝐴 ⊆ 𝐵) ⇒ ⊢ (𝜑 → 𝑅 = (𝑆 sSet 〈𝐸, 𝐴〉)) | ||
Theorem | ressval3dOLD 16966 | Obsolete version of ressval3d 16965 as of 17-Oct-2024. Value of structure restriction, deduction version. (Contributed by AV, 14-Mar-2020.) (Revised by AV, 3-Jul-2022.) (New usage is discouraged.) (Proof modification is discouraged.) |
⊢ 𝑅 = (𝑆 ↾s 𝐴) & ⊢ 𝐵 = (Base‘𝑆) & ⊢ 𝐸 = (Base‘ndx) & ⊢ (𝜑 → 𝑆 ∈ 𝑉) & ⊢ (𝜑 → Fun 𝑆) & ⊢ (𝜑 → 𝐸 ∈ dom 𝑆) & ⊢ (𝜑 → 𝐴 ⊆ 𝐵) ⇒ ⊢ (𝜑 → 𝑅 = (𝑆 sSet 〈𝐸, 𝐴〉)) | ||
Theorem | ressress 16967 | Restriction composition law. (Contributed by Stefan O'Rear, 29-Nov-2014.) (Proof shortened by Mario Carneiro, 2-Dec-2014.) |
⊢ ((𝐴 ∈ 𝑋 ∧ 𝐵 ∈ 𝑌) → ((𝑊 ↾s 𝐴) ↾s 𝐵) = (𝑊 ↾s (𝐴 ∩ 𝐵))) | ||
Theorem | ressabs 16968 | Restriction absorption law. (Contributed by Mario Carneiro, 12-Jun-2015.) |
⊢ ((𝐴 ∈ 𝑋 ∧ 𝐵 ⊆ 𝐴) → ((𝑊 ↾s 𝐴) ↾s 𝐵) = (𝑊 ↾s 𝐵)) | ||
Theorem | wunress 16969 | Closure of structure restriction in a weak universe. (Contributed by Mario Carneiro, 12-Jan-2017.) (Proof shortened by AV, 28-Oct-2024.) |
⊢ (𝜑 → 𝑈 ∈ WUni) & ⊢ (𝜑 → ω ∈ 𝑈) & ⊢ (𝜑 → 𝑊 ∈ 𝑈) ⇒ ⊢ (𝜑 → (𝑊 ↾s 𝐴) ∈ 𝑈) | ||
Theorem | wunressOLD 16970 | Obsolete proof of wunress 16969 as of 28-Oct-2024. Closure of structure restriction in a weak universe. (Contributed by Mario Carneiro, 12-Jan-2017.) (Proof modification is discouraged.) (New usage is discouraged.) |
⊢ (𝜑 → 𝑈 ∈ WUni) & ⊢ (𝜑 → ω ∈ 𝑈) & ⊢ (𝜑 → 𝑊 ∈ 𝑈) ⇒ ⊢ (𝜑 → (𝑊 ↾s 𝐴) ∈ 𝑈) | ||
Syntax | cplusg 16971 | Extend class notation with group (addition) operation. |
class +g | ||
Syntax | cmulr 16972 | Extend class notation with ring multiplication. |
class .r | ||
Syntax | cstv 16973 | Extend class notation with involution. |
class *𝑟 | ||
Syntax | csca 16974 | Extend class notation with scalar field. |
class Scalar | ||
Syntax | cvsca 16975 | Extend class notation with scalar product. |
class ·𝑠 | ||
Syntax | cip 16976 | Extend class notation with Hermitian form (inner product). |
class ·𝑖 | ||
Syntax | cts 16977 | Extend class notation with the topology component of a topological space. |
class TopSet | ||
Syntax | cple 16978 | Extend class notation with "less than or equal to" for posets. |
class le | ||
Syntax | coc 16979 | Extend class notation with the class of orthocomplementation extractors. |
class oc | ||
Syntax | cds 16980 | Extend class notation with the metric space distance function. |
class dist | ||
Syntax | cunif 16981 | Extend class notation with the uniform structure. |
class UnifSet | ||
Syntax | chom 16982 | Extend class notation with the hom-set structure. |
class Hom | ||
Syntax | cco 16983 | Extend class notation with the composition operation. |
class comp | ||
Definition | df-plusg 16984 | Define group operation. (Contributed by NM, 4-Sep-2011.) (Revised by Mario Carneiro, 14-Aug-2015.) Use its index-independent form plusgid 16998 instead. (New usage is discouraged.) |
⊢ +g = Slot 2 | ||
Definition | df-mulr 16985 | Define ring multiplication. (Contributed by NM, 4-Sep-2011.) (Revised by Mario Carneiro, 14-Aug-2015.) Use its index-independent form mulrid 17013 instead. (New usage is discouraged.) |
⊢ .r = Slot 3 | ||
Definition | df-starv 16986 | Define the involution function of a *-ring. (Contributed by NM, 4-Sep-2011.) (Revised by Mario Carneiro, 14-Aug-2015.) Use its index-independent form starvid 17022 instead. (New usage is discouraged.) |
⊢ *𝑟 = Slot 4 | ||
Definition | df-sca 16987 | Define scalar field component of a vector space 𝑣. (Contributed by NM, 4-Sep-2011.) (Revised by Mario Carneiro, 14-Aug-2015.) Use its index-independent form scaid 17034 instead. (New usage is discouraged.) |
⊢ Scalar = Slot 5 | ||
Definition | df-vsca 16988 | Define scalar product. (Contributed by NM, 4-Sep-2011.) (Revised by Mario Carneiro, 14-Aug-2015.) Use its index-independent form vscaid 17039 instead. (New usage is discouraged.) |
⊢ ·𝑠 = Slot 6 | ||
Definition | df-ip 16989 | Define Hermitian form (inner product). (Contributed by NM, 4-Sep-2011.) (Revised by Mario Carneiro, 14-Aug-2015.) Use its index-independent form ipid 17050 instead. (New usage is discouraged.) |
⊢ ·𝑖 = Slot 8 | ||
Definition | df-tset 16990 | Define the topology component of a topological space (structure). (Contributed by NM, 4-Sep-2011.) (Revised by Mario Carneiro, 14-Aug-2015.) Use its index-independent form tsetid 17072 instead. (New usage is discouraged.) |
⊢ TopSet = Slot 9 | ||
Definition | df-ple 16991 | Define "less than or equal to" ordering extractor for posets and related structures. (Contributed by NM, 4-Sep-2011.) (Revised by Mario Carneiro, 14-Aug-2015.) (Revised by AV, 9-Sep-2021.) Use its index-independent form pleid 17086 instead. (New usage is discouraged.) |
⊢ le = Slot ;10 | ||
Definition | df-ocomp 16992 | Define the orthocomplementation extractor for posets and related structures. (Contributed by NM, 4-Sep-2011.) (Revised by Mario Carneiro, 14-Aug-2015.) Use its index-independent form ocid 17101 instead. (New usage is discouraged.) |
⊢ oc = Slot ;11 | ||
Definition | df-ds 16993 | Define the distance function component of a metric space (structure). (Contributed by NM, 4-Sep-2011.) (Revised by Mario Carneiro, 14-Aug-2015.) Use its index-independent form dsid 17105 instead. (New usage is discouraged.) |
⊢ dist = Slot ;12 | ||
Definition | df-unif 16994 | Define the uniform structure component of a uniform space. (Contributed by Mario Carneiro, 14-Aug-2015.) Use its index-independent form unifid 17115 instead. (New usage is discouraged.) |
⊢ UnifSet = Slot ;13 | ||
Definition | df-hom 16995 | Define the hom-set component of a category. (Contributed by Mario Carneiro, 2-Jan-2017.) Use its index-independent form homid 17131 instead. (New usage is discouraged.) |
⊢ Hom = Slot ;14 | ||
Definition | df-cco 16996 | Define the composition operation of a category. (Contributed by Mario Carneiro, 2-Jan-2017.) Use its index-independent form ccoid 17133 instead. (New usage is discouraged.) |
⊢ comp = Slot ;15 | ||
Theorem | plusgndx 16997 | Index value of the df-plusg 16984 slot. (Contributed by Mario Carneiro, 14-Aug-2015.) (New usage is discouraged.) |
⊢ (+g‘ndx) = 2 | ||
Theorem | plusgid 16998 | Utility theorem: index-independent form of df-plusg 16984. (Contributed by NM, 20-Oct-2012.) |
⊢ +g = Slot (+g‘ndx) | ||
Theorem | plusgndxnn 16999 | The index of the slot for the group operation in an extensible structure is a positive integer. (Contributed by AV, 17-Oct-2024.) |
⊢ (+g‘ndx) ∈ ℕ | ||
Theorem | basendxltplusgndx 17000 | The index of the slot for the base set is less then the index of the slot for the group operation in an extensible structure. (Contributed by AV, 17-Oct-2024.) |
⊢ (Base‘ndx) < (+g‘ndx) |
< Previous Next > |
Copyright terms: Public domain | < Previous Next > |