![]() |
Metamath
Proof Explorer Theorem List (p. 469 of 486) | < 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-30851) |
![]() (30852-32374) |
![]() (32375-48553) |
Type | Label | Description |
---|---|---|
Statement | ||
Theorem | aovprc 46801 | The value of an operation when the one of the arguments is a proper class, analogous to ovprc 7462. (Contributed by Alexander van der Vekens, 26-May-2017.) |
⊢ Rel dom 𝐹 ⇒ ⊢ (¬ (𝐴 ∈ V ∧ 𝐵 ∈ V) → ((𝐴𝐹𝐵)) = V) | ||
Theorem | aovrcl 46802 | Reverse closure for an operation value, analogous to afvvv 46758. In contrast to ovrcl 7465, elementhood of the operation's value in a set is required, not containing an element. (Contributed by Alexander van der Vekens, 26-May-2017.) |
⊢ Rel dom 𝐹 ⇒ ⊢ ( ((𝐴𝐹𝐵)) ∈ 𝐶 → (𝐴 ∈ V ∧ 𝐵 ∈ V)) | ||
Theorem | aovpcov0 46803 | If the alternative value of the operation on an ordered pair is the universal class, the operation's value at this ordered pair is the empty set. (Contributed by Alexander van der Vekens, 26-May-2017.) |
⊢ ( ((𝐴𝐹𝐵)) = V → (𝐴𝐹𝐵) = ∅) | ||
Theorem | aovnuoveq 46804 | The alternative value of the operation on an ordered pair equals the operation's value at this ordered pair. (Contributed by Alexander van der Vekens, 26-May-2017.) |
⊢ ( ((𝐴𝐹𝐵)) ≠ V → ((𝐴𝐹𝐵)) = (𝐴𝐹𝐵)) | ||
Theorem | aovvoveq 46805 | The alternative value of the operation on an ordered pair equals the operation's value on this ordered pair. (Contributed by Alexander van der Vekens, 26-May-2017.) |
⊢ ( ((𝐴𝐹𝐵)) ∈ 𝐶 → ((𝐴𝐹𝐵)) = (𝐴𝐹𝐵)) | ||
Theorem | aov0ov0 46806 | If the alternative value of the operation on an ordered pair is the empty set, the operation's value at this ordered pair is the empty set. (Contributed by Alexander van der Vekens, 26-May-2017.) |
⊢ ( ((𝐴𝐹𝐵)) = ∅ → (𝐴𝐹𝐵) = ∅) | ||
Theorem | aovovn0oveq 46807 | If the operation's value at an argument is not the empty set, it equals the value of the alternative operation at this argument. (Contributed by Alexander van der Vekens, 26-May-2017.) |
⊢ ((𝐴𝐹𝐵) ≠ ∅ → ((𝐴𝐹𝐵)) = (𝐴𝐹𝐵)) | ||
Theorem | aov0nbovbi 46808 | The operation's value on an ordered pair is an element of a set if and only if the alternative value of the operation on this ordered pair is an element of that set, if the set does not contain the empty set. (Contributed by Alexander van der Vekens, 26-May-2017.) |
⊢ (∅ ∉ 𝐶 → ( ((𝐴𝐹𝐵)) ∈ 𝐶 ↔ (𝐴𝐹𝐵) ∈ 𝐶)) | ||
Theorem | aovov0bi 46809 | The operation's value on an ordered pair is the empty set if and only if the alternative value of the operation on this ordered pair is either the empty set or the universal class. (Contributed by Alexander van der Vekens, 26-May-2017.) |
⊢ ((𝐴𝐹𝐵) = ∅ ↔ ( ((𝐴𝐹𝐵)) = ∅ ∨ ((𝐴𝐹𝐵)) = V)) | ||
Theorem | rspceaov 46810* | A frequently used special case of rspc2ev 3621 for operation values, analogous to rspceov 7472. (Contributed by Alexander van der Vekens, 26-May-2017.) |
⊢ ((𝐶 ∈ 𝐴 ∧ 𝐷 ∈ 𝐵 ∧ 𝑆 = ((𝐶𝐹𝐷)) ) → ∃𝑥 ∈ 𝐴 ∃𝑦 ∈ 𝐵 𝑆 = ((𝑥𝐹𝑦)) ) | ||
Theorem | fnotaovb 46811 | Equivalence of operation value and ordered triple membership, analogous to fnopfvb 6955. (Contributed by Alexander van der Vekens, 26-May-2017.) |
⊢ ((𝐹 Fn (𝐴 × 𝐵) ∧ 𝐶 ∈ 𝐴 ∧ 𝐷 ∈ 𝐵) → ( ((𝐶𝐹𝐷)) = 𝑅 ↔ 〈𝐶, 𝐷, 𝑅〉 ∈ 𝐹)) | ||
Theorem | ffnaov 46812* | An operation maps to a class to which all values belong, analogous to ffnov 7552. (Contributed by Alexander van der Vekens, 26-May-2017.) |
⊢ (𝐹:(𝐴 × 𝐵)⟶𝐶 ↔ (𝐹 Fn (𝐴 × 𝐵) ∧ ∀𝑥 ∈ 𝐴 ∀𝑦 ∈ 𝐵 ((𝑥𝐹𝑦)) ∈ 𝐶)) | ||
Theorem | faovcl 46813 | Closure law for an operation, analogous to fovcl 7554. (Contributed by Alexander van der Vekens, 26-May-2017.) |
⊢ 𝐹:(𝑅 × 𝑆)⟶𝐶 ⇒ ⊢ ((𝐴 ∈ 𝑅 ∧ 𝐵 ∈ 𝑆) → ((𝐴𝐹𝐵)) ∈ 𝐶) | ||
Theorem | aovmpt4g 46814* | Value of a function given by the maps-to notation, analogous to ovmpt4g 7573. (Contributed by Alexander van der Vekens, 26-May-2017.) |
⊢ 𝐹 = (𝑥 ∈ 𝐴, 𝑦 ∈ 𝐵 ↦ 𝐶) ⇒ ⊢ ((𝑥 ∈ 𝐴 ∧ 𝑦 ∈ 𝐵 ∧ 𝐶 ∈ 𝑉) → ((𝑥𝐹𝑦)) = 𝐶) | ||
Theorem | aoprssdm 46815* | Domain of closure of an operation. In contrast to oprssdm 7607, no additional property for S (¬ ∅ ∈ 𝑆) is required! (Contributed by Alexander van der Vekens, 26-May-2017.) |
⊢ ((𝑥 ∈ 𝑆 ∧ 𝑦 ∈ 𝑆) → ((𝑥𝐹𝑦)) ∈ 𝑆) ⇒ ⊢ (𝑆 × 𝑆) ⊆ dom 𝐹 | ||
Theorem | ndmaovcl 46816 | The "closure" of an operation outside its domain, when the operation's value is a set in contrast to ndmovcl 7611 where it is required that the domain contains the empty set (∅ ∈ 𝑆). (Contributed by Alexander van der Vekens, 26-May-2017.) |
⊢ dom 𝐹 = (𝑆 × 𝑆) & ⊢ ((𝐴 ∈ 𝑆 ∧ 𝐵 ∈ 𝑆) → ((𝐴𝐹𝐵)) ∈ 𝑆) & ⊢ ((𝐴𝐹𝐵)) ∈ V ⇒ ⊢ ((𝐴𝐹𝐵)) ∈ 𝑆 | ||
Theorem | ndmaovrcl 46817 | Reverse closure law, in contrast to ndmovrcl 7612 where it is required that the operation's domain doesn't contain the empty set (¬ ∅ ∈ 𝑆), no additional asumption is required. (Contributed by Alexander van der Vekens, 26-May-2017.) |
⊢ dom 𝐹 = (𝑆 × 𝑆) ⇒ ⊢ ( ((𝐴𝐹𝐵)) ∈ 𝑆 → (𝐴 ∈ 𝑆 ∧ 𝐵 ∈ 𝑆)) | ||
Theorem | ndmaovcom 46818 | Any operation is commutative outside its domain, analogous to ndmovcom 7613. (Contributed by Alexander van der Vekens, 26-May-2017.) |
⊢ dom 𝐹 = (𝑆 × 𝑆) ⇒ ⊢ (¬ (𝐴 ∈ 𝑆 ∧ 𝐵 ∈ 𝑆) → ((𝐴𝐹𝐵)) = ((𝐵𝐹𝐴)) ) | ||
Theorem | ndmaovass 46819 | Any operation is associative outside its domain. In contrast to ndmovass 7614 where it is required that the operation's domain doesn't contain the empty set (¬ ∅ ∈ 𝑆), no additional assumption is required. (Contributed by Alexander van der Vekens, 26-May-2017.) |
⊢ dom 𝐹 = (𝑆 × 𝑆) ⇒ ⊢ (¬ (𝐴 ∈ 𝑆 ∧ 𝐵 ∈ 𝑆 ∧ 𝐶 ∈ 𝑆) → (( ((𝐴𝐹𝐵)) 𝐹𝐶)) = ((𝐴𝐹 ((𝐵𝐹𝐶)) )) ) | ||
Theorem | ndmaovdistr 46820 | Any operation is distributive outside its domain. In contrast to ndmovdistr 7615 where it is required that the operation's domain doesn't contain the empty set (¬ ∅ ∈ 𝑆), no additional assumption is required. (Contributed by Alexander van der Vekens, 26-May-2017.) |
⊢ dom 𝐹 = (𝑆 × 𝑆) & ⊢ dom 𝐺 = (𝑆 × 𝑆) ⇒ ⊢ (¬ (𝐴 ∈ 𝑆 ∧ 𝐵 ∈ 𝑆 ∧ 𝐶 ∈ 𝑆) → ((𝐴𝐺 ((𝐵𝐹𝐶)) )) = (( ((𝐴𝐺𝐵)) 𝐹 ((𝐴𝐺𝐶)) )) ) | ||
In the following, a second approach is followed to define function values alternately to df-afv 46733. The current definition of the value (𝐹‘𝐴) of a function 𝐹 at an argument 𝐴 (see df-fv 6562) assures that this value is always a set, see fex 7243. This is because this definition can be applied to any classes 𝐹 and 𝐴, and evaluates to the empty set when it is not meaningful (as shown by ndmfv 6936 and fvprc 6893). "(𝐹‘𝐴) is meaningful" means "the class 𝐹 regarded as function is defined at the argument 𝐴" in this context. This is also expressed by 𝐹 defAt 𝐴, see df-dfat 46732. In the theory of partial functions, it is a common case that 𝐹 is not defined at 𝐴. Although it is very convenient for many theorems on functions and their proofs, there are some cases in which from (𝐹‘𝐴) = ∅ alone it cannot be decided/derived whether (𝐹‘𝐴) is meaningful (𝐹 is actually a function which is defined for 𝐴 and really has the function value ∅ at 𝐴) or not. Therefore, additional assumptions are required, such as ∅ ∉ ran 𝐹, ∅ ∈ ran 𝐹, 𝐹 defAt 𝐴, or Fun 𝐹 ∧ 𝐴 ∈ dom 𝐹 (see, for example, ndmfvrcl 6937). To avoid such an ambiguity, an alternative definition (𝐹''''𝐴) (see df-afv2 46822) would be possible which evaluates to a set not belonging to the range of 𝐹 ((𝐹''''𝐴) = 𝒫 ∪ ran 𝐹) if it is not meaningful (see ndfatafv2 46824). We say "(𝐹''''𝐴) is not defined (or undefined)" if (𝐹''''𝐴) is not in the range of 𝐹 ((𝐹''''𝐴) ∉ ran 𝐹). Because of afv2ndefb 46837, this is equivalent to ((𝐹''''𝐴) = 𝒫 ∪ ran 𝐹. If (𝐹''''𝐴) is in the range of 𝐹 ((𝐹''''𝐴) ∈ ran 𝐹), we say that "(𝐹''''𝐴) is defined". If ran 𝐹 is a set, we can use the symbol Undef to express that (𝐹''''𝐴) is not defined: (𝐹''''𝐴) = (Undef‘ran 𝐹) (see ndfatafv2undef 46825). We could have used this symbol directly to define the alternate value of a function, which would have the advantage that (𝐹''''𝐴) would always be a set. But first this symbol is defined using the original function value, which would not make it possible to replace the original definition by the alternate definition, and second we would have to assume that ran 𝐹 ∈ V in most of the theorems. To summarize, that means (𝐹''''𝐴) ∉ ran 𝐹 → (𝐹‘𝐴) = ∅ (see afv2ndeffv0 46873), but (𝐹‘𝐴) = ∅ → (𝐹''''𝐴) ∉ ran 𝐹 is not generally valid, see afv2fv0 46878. The alternate definition, however, corresponds to the current definition ((𝐹‘𝐴) = (𝐹''''𝐴)) if the function 𝐹 is defined at 𝐴 (see dfatafv2eqfv 46874). With this definition the following intuitive equivalence holds: (𝐹 defAt 𝐴 ↔ (𝐹''''𝐴) ∈ ran 𝐹), see dfatafv2rnb 46840. An interesting question would be if (𝐹‘𝐴) could be replaced by (𝐹'''𝐴) in most of the theorems based on function values. If we look at the (currently 24) proofs using the definition df-fv 6562 of (𝐹‘𝐴), we see that analogues for the following 7 theorems can be proven using the alternative definition: fveq1 6900-> afv2eq1 46829, fveq2 6901-> afv2eq2 46830, nffv 6911-> nfafv2 46831, csbfv12 6949-> csbafv212g , rlimdm 15553-> rlimdmafv2 46871, tz6.12-1 6924-> tz6.12-1-afv2 46854, fveu 6890-> afv2eu 46851. Six theorems proved by directly using df-fv 6562 are within a mathbox (fvsb 44126, uncov 37302) or not used (rlimdmafv 46790, avril1 30396) or experimental (dfafv2 46745, dfafv22 46872). However, the remaining 11 theorems proved by directly using df-fv 6562 are used more or less often: * fvex 6914: used in about 1600 proofs: Only if the function is defined at the argument, or the range of the function/class is a set, analog theorems can be proven (dfatafv2ex 46826 resp. afv2ex 46827). All of these 1600 proofs have to be checked if one of these two theorems can be used instead of fvex 6914. * fvres 6920: used in about 400 proofs : Only if the function is defined at the argument, an analog theorem can be proven (afv2res 46852). In the undefined case such a theorem cannot exist (without additional assumptions), because the range of (𝐹 ↾ 𝐵) is mostly different from the range of 𝐹, and therefore also the "undefined" values are different. All of these 400 proofs have to be checked if afv2res 46852 can be used instead of fvres 6920. * tz6.12-2 6889 (-> tz6.12-2-afv2 46850): root theorem of many theorems which have not a strict analogue, and which are used many times: ** fvprc 6893 (-> afv2prc 46839), used in 193 proofs, ** tz6.12i 6929 (-> tz6.12i-afv2 46856), used - indirectly via fvbr0 6930 and fvrn0 6931 - in 19 proofs, and in fvclss 7256 used in fvclex 7972 used in fvresex 7973 (which is not used!) and in dcomex 10490 (used in 4 proofs), ** ndmfv 6936 (-> ndmafv2nrn ), used in 124 proofs ** nfunsn 6943 (-> nfunsnafv2 ), used by fvfundmfvn0 6944 (used in 3 proofs), and dffv2 6997 (not used) ** funpartfv 35769, setrec2lem1 48439 (mathboxes) * fv2 6896: only used by elfv 6899, which is only used by fv3 6919, which is not used. * dffv3 6897 (-> dfafv23 ): used by dffv4 6898 (the previous "df-fv"), which now is only used in mathboxes (csbfv12gALTVD 44575), by shftval 15079 (itself used in 11 proofs), by dffv5 35748 (mathbox) and by fvco2 6999 (-> afv2co2 46870). * fvopab5 7042: used only by ajval 30794 (not used) and by adjval 31823, which is used in adjval2 31824 (not used) and in adjbdln 32016 (used in 7 proofs). * zsum 15722: used (via isum 15723, sum0 15725, sumss 15728 and fsumsers 15732) in 76 proofs. * isumshft 15843: used in pserdv2 26460 (used in logtayl 26687, binomcxplemdvsum 44029) , eftlub 16111 (used in 4 proofs), binomcxplemnotnn0 44030 (used in binomcxp 44031 only) and logtayl 26687 (used in 4 proofs). * ovtpos 8256: used in 16 proofs. * zprod 15939: used in 3 proofs: iprod 15940, zprodn0 15941 and prodss 15949 * iprodclim3 16002: not used! As a result of this analysis we can say that the current definition of a function value is crucial for Metamath and cannot be exchanged easily with an alternative definition. While fv2 6896, dffv3 6897, fvopab5 7042, zsum 15722, isumshft 15843, ovtpos 8256 and zprod 15939 are not critical or are, hopefully, also valid for the alternative definition, fvex 6914, fvres 6920 and tz6.12-2 6889 (and the theorems based on them) are essential for the current definition of function values. | ||
Syntax | cafv2 46821 | Extend the definition of a class to include the alternate function value. Read: "the value of 𝐹 at 𝐴 " or "𝐹 of 𝐴". For using several apostrophes as a symbol see comment for cafv 46730. |
class (𝐹''''𝐴) | ||
Definition | df-afv2 46822* | Alternate definition of the value of a function, (𝐹''''𝐴), also known as function application (and called "alternate function value" in the following). In contrast to (𝐹‘𝐴) = ∅ (see comment of df-fv 6562, and especially ndmfv 6936), (𝐹''''𝐴) is guaranteed not to be in the range of 𝐹 if 𝐹 is not defined at 𝐴 (whereas ∅ can be a member of ran 𝐹). (Contributed by AV, 2-Sep-2022.) |
⊢ (𝐹''''𝐴) = if(𝐹 defAt 𝐴, (℩𝑥𝐴𝐹𝑥), 𝒫 ∪ ran 𝐹) | ||
Theorem | dfatafv2iota 46823* | If a function is defined at a class 𝐴 the alternate function value at 𝐴 is the unique value assigned to 𝐴 by the function (analogously to (𝐹‘𝐴)). (Contributed by AV, 2-Sep-2022.) |
⊢ (𝐹 defAt 𝐴 → (𝐹''''𝐴) = (℩𝑥𝐴𝐹𝑥)) | ||
Theorem | ndfatafv2 46824 | The alternate function value at a class 𝐴 if the function is not defined at this set 𝐴. (Contributed by AV, 2-Sep-2022.) |
⊢ (¬ 𝐹 defAt 𝐴 → (𝐹''''𝐴) = 𝒫 ∪ ran 𝐹) | ||
Theorem | ndfatafv2undef 46825 | The alternate function value at a class 𝐴 is undefined if the function, whose range is a set, is not defined at 𝐴. (Contributed by AV, 2-Sep-2022.) |
⊢ ((ran 𝐹 ∈ 𝑉 ∧ ¬ 𝐹 defAt 𝐴) → (𝐹''''𝐴) = (Undef‘ran 𝐹)) | ||
Theorem | dfatafv2ex 46826 | The alternate function value at a class 𝐴 is always a set if the function/class 𝐹 is defined at 𝐴. (Contributed by AV, 6-Sep-2022.) |
⊢ (𝐹 defAt 𝐴 → (𝐹''''𝐴) ∈ V) | ||
Theorem | afv2ex 46827 | The alternate function value is always a set if the range of the function is a set. (Contributed by AV, 2-Sep-2022.) |
⊢ (ran 𝐹 ∈ 𝑉 → (𝐹''''𝐴) ∈ V) | ||
Theorem | afv2eq12d 46828 | Equality deduction for function value, analogous to fveq12d 6908. (Contributed by AV, 4-Sep-2022.) |
⊢ (𝜑 → 𝐹 = 𝐺) & ⊢ (𝜑 → 𝐴 = 𝐵) ⇒ ⊢ (𝜑 → (𝐹''''𝐴) = (𝐺''''𝐵)) | ||
Theorem | afv2eq1 46829 | Equality theorem for function value, analogous to fveq1 6900. (Contributed by AV, 4-Sep-2022.) |
⊢ (𝐹 = 𝐺 → (𝐹''''𝐴) = (𝐺''''𝐴)) | ||
Theorem | afv2eq2 46830 | Equality theorem for function value, analogous to fveq2 6901. (Contributed by AV, 4-Sep-2022.) |
⊢ (𝐴 = 𝐵 → (𝐹''''𝐴) = (𝐹''''𝐵)) | ||
Theorem | nfafv2 46831 | Bound-variable hypothesis builder for function value, analogous to nffv 6911. To prove a deduction version of this analogous to nffvd 6913 is not easily possible because a deduction version of nfdfat 46740 cannot be shown easily. (Contributed by AV, 4-Sep-2022.) |
⊢ Ⅎ𝑥𝐹 & ⊢ Ⅎ𝑥𝐴 ⇒ ⊢ Ⅎ𝑥(𝐹''''𝐴) | ||
Theorem | csbafv212g 46832 | Move class substitution in and out of a function value, analogous to csbfv12 6949, with a direct proof proposed by Mario Carneiro, analogous to csbov123 7467. (Contributed by AV, 4-Sep-2022.) |
⊢ (𝐴 ∈ 𝑉 → ⦋𝐴 / 𝑥⦌(𝐹''''𝐵) = (⦋𝐴 / 𝑥⦌𝐹''''⦋𝐴 / 𝑥⦌𝐵)) | ||
Theorem | fexafv2ex 46833 | The alternate function value is always a set if the function (resp. the domain of the function) is a set. (Contributed by AV, 3-Sep-2022.) |
⊢ (𝐹 ∈ 𝑉 → (𝐹''''𝐴) ∈ V) | ||
Theorem | ndfatafv2nrn 46834 | The alternate function value at a class 𝐴 at which the function is not defined is undefined, i.e., not in the range of the function. (Contributed by AV, 2-Sep-2022.) |
⊢ (¬ 𝐹 defAt 𝐴 → (𝐹''''𝐴) ∉ ran 𝐹) | ||
Theorem | ndmafv2nrn 46835 | The value of a class outside its domain is not in the range, compare with ndmfv 6936. (Contributed by AV, 2-Sep-2022.) |
⊢ (¬ 𝐴 ∈ dom 𝐹 → (𝐹''''𝐴) ∉ ran 𝐹) | ||
Theorem | funressndmafv2rn 46836 | The alternate function value at a class 𝐴 is defined, i.e., in the range of the function if the function is defined at 𝐴. (Contributed by AV, 2-Sep-2022.) |
⊢ (𝐹 defAt 𝐴 → (𝐹''''𝐴) ∈ ran 𝐹) | ||
Theorem | afv2ndefb 46837 | Two ways to say that an alternate function value is not defined. (Contributed by AV, 5-Sep-2022.) |
⊢ ((𝐹''''𝐴) = 𝒫 ∪ ran 𝐹 ↔ (𝐹''''𝐴) ∉ ran 𝐹) | ||
Theorem | nfunsnafv2 46838 | If the restriction of a class to a singleton is not a function, its value at the singleton element is undefined, compare with nfunsn 6943. (Contributed by AV, 2-Sep-2022.) |
⊢ (¬ Fun (𝐹 ↾ {𝐴}) → (𝐹''''𝐴) ∉ ran 𝐹) | ||
Theorem | afv2prc 46839 | A function's value at a proper class is not defined, compare with fvprc 6893. (Contributed by AV, 5-Sep-2022.) |
⊢ (¬ 𝐴 ∈ V → (𝐹''''𝐴) ∉ ran 𝐹) | ||
Theorem | dfatafv2rnb 46840 | The alternate function value at a class 𝐴 is defined, i.e. in the range of the function, iff the function is defined at 𝐴. (Contributed by AV, 2-Sep-2022.) |
⊢ (𝐹 defAt 𝐴 ↔ (𝐹''''𝐴) ∈ ran 𝐹) | ||
Theorem | afv2orxorb 46841 | If a set is in the range of a function, the alternate function value at a class 𝐴 equals this set or is not in the range of the function iff the alternate function value at the class 𝐴 either equals this set or is not in the range of the function. If 𝐵 ∉ ran 𝐹, both disjuncts of the exclusive or can be true: (𝐹''''𝐴) = 𝐵 → (𝐹''''𝐴) ∉ ran 𝐹. (Contributed by AV, 11-Sep-2022.) |
⊢ (𝐵 ∈ ran 𝐹 → (((𝐹''''𝐴) = 𝐵 ∨ (𝐹''''𝐴) ∉ ran 𝐹) ↔ ((𝐹''''𝐴) = 𝐵 ⊻ (𝐹''''𝐴) ∉ ran 𝐹))) | ||
Theorem | dmafv2rnb 46842 | The alternate function value at a class 𝐴 is defined, i.e., in the range of the function, iff 𝐴 is in the domain of the function. (Contributed by AV, 3-Sep-2022.) |
⊢ (Fun (𝐹 ↾ {𝐴}) → (𝐴 ∈ dom 𝐹 ↔ (𝐹''''𝐴) ∈ ran 𝐹)) | ||
Theorem | fundmafv2rnb 46843 | The alternate function value at a class 𝐴 is defined, i.e., in the range of the function iff 𝐴 is in the domain of the function. (Contributed by AV, 3-Sep-2022.) |
⊢ (Fun 𝐹 → (𝐴 ∈ dom 𝐹 ↔ (𝐹''''𝐴) ∈ ran 𝐹)) | ||
Theorem | afv2elrn 46844 | An alternate function value belongs to the range of the function, analogous to fvelrn 7090. (Contributed by AV, 3-Sep-2022.) |
⊢ ((Fun 𝐹 ∧ 𝐴 ∈ dom 𝐹) → (𝐹''''𝐴) ∈ ran 𝐹) | ||
Theorem | afv20defat 46845 | If the alternate function value at an argument is the empty set, the function is defined at this argument. (Contributed by AV, 3-Sep-2022.) |
⊢ ((𝐹''''𝐴) = ∅ → 𝐹 defAt 𝐴) | ||
Theorem | fnafv2elrn 46846 | An alternate function value belongs to the range of the function, analogous to fnfvelrn 7094. (Contributed by AV, 2-Sep-2022.) |
⊢ ((𝐹 Fn 𝐴 ∧ 𝐵 ∈ 𝐴) → (𝐹''''𝐵) ∈ ran 𝐹) | ||
Theorem | fafv2elcdm 46847 | An alternate function value belongs to the codomain of the function, analogous to ffvelcdm 7095. (Contributed by AV, 2-Sep-2022.) |
⊢ ((𝐹:𝐴⟶𝐵 ∧ 𝐶 ∈ 𝐴) → (𝐹''''𝐶) ∈ 𝐵) | ||
Theorem | fafv2elrnb 46848 | An alternate function value is defined, i.e., belongs to the range of the function, iff its argument is in the domain of the function. (Contributed by AV, 3-Sep-2022.) |
⊢ (𝐹:𝐴⟶𝐵 → (𝐶 ∈ 𝐴 ↔ (𝐹''''𝐶) ∈ ran 𝐹)) | ||
Theorem | fcdmvafv2v 46849 | If the codomain of a function is a set, the alternate function value is always also a set. (Contributed by AV, 4-Sep-2022.) |
⊢ ((𝐹:𝐴⟶𝐵 ∧ 𝐵 ∈ 𝑉) → (𝐹''''𝐶) ∈ V) | ||
Theorem | tz6.12-2-afv2 46850* | Function value when 𝐹 is (locally) not a function. Theorem 6.12(2) of [TakeutiZaring] p. 27, analogous to tz6.12-2 6889. (Contributed by AV, 5-Sep-2022.) |
⊢ (¬ ∃!𝑥 𝐴𝐹𝑥 → (𝐹''''𝐴) ∉ ran 𝐹) | ||
Theorem | afv2eu 46851* | The value of a function at a unique point, analogous to fveu 6890. (Contributed by AV, 5-Sep-2022.) |
⊢ (∃!𝑥 𝐴𝐹𝑥 → (𝐹''''𝐴) = ∪ {𝑥 ∣ 𝐴𝐹𝑥}) | ||
Theorem | afv2res 46852 | The value of a restricted function for an argument at which the function is defined. Analog to fvres 6920. (Contributed by AV, 5-Sep-2022.) |
⊢ ((𝐹 defAt 𝐴 ∧ 𝐴 ∈ 𝐵) → ((𝐹 ↾ 𝐵)''''𝐴) = (𝐹''''𝐴)) | ||
Theorem | tz6.12-afv2 46853* | Function value (Theorem 6.12(1) of [TakeutiZaring] p. 27), analogous to tz6.12 6926. (Contributed by AV, 5-Sep-2022.) |
⊢ ((〈𝐴, 𝑦〉 ∈ 𝐹 ∧ ∃!𝑦〈𝐴, 𝑦〉 ∈ 𝐹) → (𝐹''''𝐴) = 𝑦) | ||
Theorem | tz6.12-1-afv2 46854* | Function value (Theorem 6.12(1) of [TakeutiZaring] p. 27), analogous to tz6.12-1 6924. (Contributed by AV, 5-Sep-2022.) |
⊢ ((𝐴𝐹𝑦 ∧ ∃!𝑦 𝐴𝐹𝑦) → (𝐹''''𝐴) = 𝑦) | ||
Theorem | tz6.12c-afv2 46855* | Corollary of Theorem 6.12(1) of [TakeutiZaring] p. 27, analogous to tz6.12c 6923. (Contributed by AV, 5-Sep-2022.) |
⊢ (∃!𝑦 𝐴𝐹𝑦 → ((𝐹''''𝐴) = 𝑦 ↔ 𝐴𝐹𝑦)) | ||
Theorem | tz6.12i-afv2 46856 | Corollary of Theorem 6.12(2) of [TakeutiZaring] p. 27. analogous to tz6.12i 6929. (Contributed by AV, 5-Sep-2022.) |
⊢ (𝐵 ∈ ran 𝐹 → ((𝐹''''𝐴) = 𝐵 → 𝐴𝐹𝐵)) | ||
Theorem | funressnbrafv2 46857 | The second argument of a binary relation on a function is the function's value, analogous to funbrfv 6952. (Contributed by AV, 7-Sep-2022.) |
⊢ (((𝐴 ∈ 𝑉 ∧ 𝐵 ∈ 𝑊) ∧ Fun (𝐹 ↾ {𝐴})) → (𝐴𝐹𝐵 → (𝐹''''𝐴) = 𝐵)) | ||
Theorem | dfatbrafv2b 46858 | Equivalence of function value and binary relation, analogous to fnbrfvb 6954 or funbrfvb 6956. 𝐵 ∈ V is required, because otherwise 𝐴𝐹𝐵 ↔ ∅ ∈ 𝐹 can be true, but (𝐹''''𝐴) = 𝐵 is always false (because of dfatafv2ex 46826). (Contributed by AV, 6-Sep-2022.) |
⊢ ((𝐹 defAt 𝐴 ∧ 𝐵 ∈ 𝑊) → ((𝐹''''𝐴) = 𝐵 ↔ 𝐴𝐹𝐵)) | ||
Theorem | dfatopafv2b 46859 | Equivalence of function value and ordered pair membership, analogous to fnopfvb 6955 or funopfvb 6957. (Contributed by AV, 6-Sep-2022.) |
⊢ ((𝐹 defAt 𝐴 ∧ 𝐵 ∈ 𝑊) → ((𝐹''''𝐴) = 𝐵 ↔ 〈𝐴, 𝐵〉 ∈ 𝐹)) | ||
Theorem | funbrafv2 46860 | The second argument of a binary relation on a function is the function's value, analogous to funbrfv 6952. (Contributed by AV, 6-Sep-2022.) |
⊢ (Fun 𝐹 → (𝐴𝐹𝐵 → (𝐹''''𝐴) = 𝐵)) | ||
Theorem | fnbrafv2b 46861 | Equivalence of function value and binary relation, analogous to fnbrfvb 6954. (Contributed by AV, 6-Sep-2022.) |
⊢ ((𝐹 Fn 𝐴 ∧ 𝐵 ∈ 𝐴) → ((𝐹''''𝐵) = 𝐶 ↔ 𝐵𝐹𝐶)) | ||
Theorem | fnopafv2b 46862 | Equivalence of function value and ordered pair membership, analogous to fnopfvb 6955. (Contributed by AV, 6-Sep-2022.) |
⊢ ((𝐹 Fn 𝐴 ∧ 𝐵 ∈ 𝐴) → ((𝐹''''𝐵) = 𝐶 ↔ 〈𝐵, 𝐶〉 ∈ 𝐹)) | ||
Theorem | funbrafv22b 46863 | Equivalence of function value and binary relation, analogous to funbrfvb 6956. (Contributed by AV, 6-Sep-2022.) |
⊢ ((Fun 𝐹 ∧ 𝐴 ∈ dom 𝐹) → ((𝐹''''𝐴) = 𝐵 ↔ 𝐴𝐹𝐵)) | ||
Theorem | funopafv2b 46864 | Equivalence of function value and ordered pair membership, analogous to funopfvb 6957. (Contributed by AV, 6-Sep-2022.) |
⊢ ((Fun 𝐹 ∧ 𝐴 ∈ dom 𝐹) → ((𝐹''''𝐴) = 𝐵 ↔ 〈𝐴, 𝐵〉 ∈ 𝐹)) | ||
Theorem | dfatsnafv2 46865 | Singleton of function value, analogous to fnsnfv 6981. (Contributed by AV, 7-Sep-2022.) |
⊢ (𝐹 defAt 𝐴 → {(𝐹''''𝐴)} = (𝐹 “ {𝐴})) | ||
Theorem | dfafv23 46866* | A definition of function value in terms of iota, analogous to dffv3 6897. (Contributed by AV, 6-Sep-2022.) |
⊢ (𝐹 defAt 𝐴 → (𝐹''''𝐴) = (℩𝑥𝑥 ∈ (𝐹 “ {𝐴}))) | ||
Theorem | dfatdmfcoafv2 46867 | Domain of a function composition, analogous to dmfco 6998. (Contributed by AV, 7-Sep-2022.) |
⊢ (𝐺 defAt 𝐴 → (𝐴 ∈ dom (𝐹 ∘ 𝐺) ↔ (𝐺''''𝐴) ∈ dom 𝐹)) | ||
Theorem | dfatcolem 46868* | Lemma for dfatco 46869. (Contributed by AV, 8-Sep-2022.) |
⊢ ((𝐺 defAt 𝑋 ∧ 𝐹 defAt (𝐺''''𝑋)) → ∃!𝑦 𝑋(𝐹 ∘ 𝐺)𝑦) | ||
Theorem | dfatco 46869 | The predicate "defined at" for a function composition. (Contributed by AV, 8-Sep-2022.) |
⊢ ((𝐺 defAt 𝑋 ∧ 𝐹 defAt (𝐺''''𝑋)) → (𝐹 ∘ 𝐺) defAt 𝑋) | ||
Theorem | afv2co2 46870 | Value of a function composition, analogous to fvco2 6999. (Contributed by AV, 8-Sep-2022.) |
⊢ ((𝐺 defAt 𝑋 ∧ 𝐹 defAt (𝐺''''𝑋)) → ((𝐹 ∘ 𝐺)''''𝑋) = (𝐹''''(𝐺''''𝑋))) | ||
Theorem | rlimdmafv2 46871 | Two ways to express that a function has a limit, analogous to rlimdm 15553. (Contributed by AV, 5-Sep-2022.) |
⊢ (𝜑 → 𝐹:𝐴⟶ℂ) & ⊢ (𝜑 → sup(𝐴, ℝ*, < ) = +∞) ⇒ ⊢ (𝜑 → (𝐹 ∈ dom ⇝𝑟 ↔ 𝐹 ⇝𝑟 ( ⇝𝑟 ''''𝐹))) | ||
Theorem | dfafv22 46872 | Alternate definition of (𝐹''''𝐴) using (𝐹‘𝐴) directly. (Contributed by AV, 3-Sep-2022.) |
⊢ (𝐹''''𝐴) = if(𝐹 defAt 𝐴, (𝐹‘𝐴), 𝒫 ∪ ran 𝐹) | ||
Theorem | afv2ndeffv0 46873 | If the alternate function value at an argument is undefined, i.e., not in the range of the function, the function's value at this argument is the empty set. (Contributed by AV, 3-Sep-2022.) |
⊢ ((𝐹''''𝐴) ∉ ran 𝐹 → (𝐹‘𝐴) = ∅) | ||
Theorem | dfatafv2eqfv 46874 | If a function is defined at a class 𝐴, the alternate function value equals the function's value at 𝐴. (Contributed by AV, 3-Sep-2022.) |
⊢ (𝐹 defAt 𝐴 → (𝐹''''𝐴) = (𝐹‘𝐴)) | ||
Theorem | afv2rnfveq 46875 | If the alternate function value is defined, i.e., in the range of the function, the alternate function value equals the function's value. (Contributed by AV, 3-Sep-2022.) |
⊢ ((𝐹''''𝐴) ∈ ran 𝐹 → (𝐹''''𝐴) = (𝐹‘𝐴)) | ||
Theorem | afv20fv0 46876 | If the alternate function value at an argument is the empty set, the function's value at this argument is the empty set. (Contributed by AV, 3-Sep-2022.) |
⊢ ((𝐹''''𝐴) = ∅ → (𝐹‘𝐴) = ∅) | ||
Theorem | afv2fvn0fveq 46877 | If the function's value at an argument is not the empty set, it equals the alternate function value at this argument. (Contributed by AV, 3-Sep-2022.) |
⊢ ((𝐹‘𝐴) ≠ ∅ → (𝐹''''𝐴) = (𝐹‘𝐴)) | ||
Theorem | afv2fv0 46878 | If the function's value at an argument is the empty set, then the alternate function value at this argument is the empty set or undefined. (Contributed by AV, 3-Sep-2022.) |
⊢ ((𝐹‘𝐴) = ∅ → ((𝐹''''𝐴) = ∅ ∨ (𝐹''''𝐴) ∉ ran 𝐹)) | ||
Theorem | afv2fv0b 46879 | The function's value at an argument is the empty set if and only if the alternate function value at this argument is the empty set or undefined. (Contributed by AV, 3-Sep-2022.) |
⊢ ((𝐹‘𝐴) = ∅ ↔ ((𝐹''''𝐴) = ∅ ∨ (𝐹''''𝐴) ∉ ran 𝐹)) | ||
Theorem | afv2fv0xorb 46880 | If a set is in the range of a function, the function's value at an argument is the empty set if and only if the alternate function value at this argument is either the empty set or undefined. (Contributed by AV, 11-Sep-2022.) |
⊢ (∅ ∈ ran 𝐹 → ((𝐹‘𝐴) = ∅ ↔ ((𝐹''''𝐴) = ∅ ⊻ (𝐹''''𝐴) ∉ ran 𝐹))) | ||
Theorem | an4com24 46881 | Rearrangement of 4 conjuncts: second and forth positions interchanged. (Contributed by AV, 18-Feb-2022.) |
⊢ (((𝜑 ∧ 𝜓) ∧ (𝜒 ∧ 𝜃)) ↔ ((𝜑 ∧ 𝜃) ∧ (𝜒 ∧ 𝜓))) | ||
Theorem | 3an4ancom24 46882 | Commutative law for a conjunction with a triple conjunction: second and forth positions interchanged. (Contributed by AV, 18-Feb-2022.) |
⊢ (((𝜑 ∧ 𝜓 ∧ 𝜒) ∧ 𝜃) ↔ ((𝜑 ∧ 𝜃 ∧ 𝜒) ∧ 𝜓)) | ||
Theorem | 4an21 46883 | Rearrangement of 4 conjuncts with a triple conjunction. (Contributed by AV, 4-Mar-2022.) |
⊢ (((𝜑 ∧ 𝜓) ∧ 𝜒 ∧ 𝜃) ↔ (𝜓 ∧ (𝜑 ∧ 𝜒 ∧ 𝜃))) | ||
Syntax | cnelbr 46884 | Extend wff notation to include the 'not element of' relation. |
class _∉ | ||
Definition | df-nelbr 46885* | Define negated membership as binary relation. Analogous to df-eprel 5586 (the membership relation). (Contributed by AV, 26-Dec-2021.) |
⊢ _∉ = {〈𝑥, 𝑦〉 ∣ ¬ 𝑥 ∈ 𝑦} | ||
Theorem | dfnelbr2 46886 | Alternate definition of the negated membership as binary relation. (Proposed by BJ, 27-Dec-2021.) (Contributed by AV, 27-Dec-2021.) |
⊢ _∉ = ((V × V) ∖ E ) | ||
Theorem | nelbr 46887 | The binary relation of a set not being a member of another set. (Contributed by AV, 26-Dec-2021.) |
⊢ ((𝐴 ∈ 𝑉 ∧ 𝐵 ∈ 𝑊) → (𝐴 _∉ 𝐵 ↔ ¬ 𝐴 ∈ 𝐵)) | ||
Theorem | nelbrim 46888 | If a set is related to another set by the negated membership relation, then it is not a member of the other set. The other direction of the implication is not generally true, because if 𝐴 is a proper class, then ¬ 𝐴 ∈ 𝐵 would be true, but not 𝐴 _∉ 𝐵. (Contributed by AV, 26-Dec-2021.) |
⊢ (𝐴 _∉ 𝐵 → ¬ 𝐴 ∈ 𝐵) | ||
Theorem | nelbrnel 46889 | A set is related to another set by the negated membership relation iff it is not a member of the other set. (Contributed by AV, 26-Dec-2021.) |
⊢ ((𝐴 ∈ 𝑉 ∧ 𝐵 ∈ 𝑊) → (𝐴 _∉ 𝐵 ↔ 𝐴 ∉ 𝐵)) | ||
Theorem | nelbrnelim 46890 | If a set is related to another set by the negated membership relation, then it is not a member of the other set. (Contributed by AV, 26-Dec-2021.) |
⊢ (𝐴 _∉ 𝐵 → 𝐴 ∉ 𝐵) | ||
Theorem | ralralimp 46891* | Selecting one of two alternatives within a restricted generalization if one of the alternatives is false. (Contributed by AV, 6-Sep-2018.) (Proof shortened by AV, 13-Oct-2018.) |
⊢ ((𝜑 ∧ 𝐴 ≠ ∅) → (∀𝑥 ∈ 𝐴 ((𝜑 → (𝜃 ∨ 𝜏)) ∧ ¬ 𝜃) → 𝜏)) | ||
Theorem | otiunsndisjX 46892* | The union of singletons consisting of ordered triples which have distinct first and third components are disjunct. (Contributed by Alexander van der Vekens, 10-Mar-2018.) |
⊢ (𝐵 ∈ 𝑋 → Disj 𝑎 ∈ 𝑉 ∪ 𝑐 ∈ 𝑊 {〈𝑎, 𝐵, 𝑐〉}) | ||
Theorem | fvifeq 46893 | Equality of function values with conditional arguments, see also fvif 6917. (Contributed by Alexander van der Vekens, 21-May-2018.) |
⊢ (𝐴 = if(𝜑, 𝐵, 𝐶) → (𝐹‘𝐴) = if(𝜑, (𝐹‘𝐵), (𝐹‘𝐶))) | ||
Theorem | rnfdmpr 46894 | The range of a one-to-one function 𝐹 of an unordered pair into a set is the unordered pair of the function values. (Contributed by Alexander van der Vekens, 2-Feb-2018.) |
⊢ ((𝑋 ∈ 𝑉 ∧ 𝑌 ∈ 𝑊) → (𝐹 Fn {𝑋, 𝑌} → ran 𝐹 = {(𝐹‘𝑋), (𝐹‘𝑌)})) | ||
Theorem | imarnf1pr 46895 | The image of the range of a function 𝐹 under a function 𝐸 if 𝐹 is a function from a pair into the domain of 𝐸. (Contributed by Alexander van der Vekens, 2-Feb-2018.) |
⊢ ((𝑋 ∈ 𝑉 ∧ 𝑌 ∈ 𝑊) → (((𝐹:{𝑋, 𝑌}⟶dom 𝐸 ∧ 𝐸:dom 𝐸⟶𝑅) ∧ ((𝐸‘(𝐹‘𝑋)) = 𝐴 ∧ (𝐸‘(𝐹‘𝑌)) = 𝐵)) → (𝐸 “ ran 𝐹) = {𝐴, 𝐵})) | ||
Theorem | funop1 46896* | A function is an ordered pair iff it is a singleton of an ordered pair. (Contributed by AV, 20-Sep-2020.) (Avoid depending on this detail.) |
⊢ (∃𝑥∃𝑦 𝐹 = 〈𝑥, 𝑦〉 → (Fun 𝐹 ↔ ∃𝑥∃𝑦 𝐹 = {〈𝑥, 𝑦〉})) | ||
Theorem | fun2dmnopgexmpl 46897 | A function with a domain containing (at least) two different elements is not an ordered pair. (Contributed by AV, 21-Sep-2020.) (Avoid depending on this detail.) |
⊢ (𝐺 = {〈0, 1〉, 〈1, 1〉} → ¬ 𝐺 ∈ (V × V)) | ||
Theorem | opabresex0d 46898* | A collection of ordered pairs, the class of all possible second components being a set, with a restriction of a binary relation is a set. (Contributed by Alexander van der Vekens, 1-Nov-2017.) (Revised by AV, 1-Jan-2021.) |
⊢ ((𝜑 ∧ 𝑥𝑅𝑦) → 𝑥 ∈ 𝐶) & ⊢ ((𝜑 ∧ 𝑥𝑅𝑦) → 𝜃) & ⊢ ((𝜑 ∧ 𝑥 ∈ 𝐶) → {𝑦 ∣ 𝜃} ∈ 𝑉) & ⊢ (𝜑 → 𝐶 ∈ 𝑊) ⇒ ⊢ (𝜑 → {〈𝑥, 𝑦〉 ∣ (𝑥𝑅𝑦 ∧ 𝜓)} ∈ V) | ||
Theorem | opabbrfex0d 46899* | A collection of ordered pairs, the class of all possible second components being a set, is a set. (Contributed by AV, 15-Jan-2021.) |
⊢ ((𝜑 ∧ 𝑥𝑅𝑦) → 𝑥 ∈ 𝐶) & ⊢ ((𝜑 ∧ 𝑥𝑅𝑦) → 𝜃) & ⊢ ((𝜑 ∧ 𝑥 ∈ 𝐶) → {𝑦 ∣ 𝜃} ∈ 𝑉) & ⊢ (𝜑 → 𝐶 ∈ 𝑊) ⇒ ⊢ (𝜑 → {〈𝑥, 𝑦〉 ∣ 𝑥𝑅𝑦} ∈ V) | ||
Theorem | opabresexd 46900* | A collection of ordered pairs, the second component being a function, with a restriction of a binary relation is a set. (Contributed by Alexander van der Vekens, 1-Nov-2017.) (Revised by AV, 15-Jan-2021.) |
⊢ ((𝜑 ∧ 𝑥𝑅𝑦) → 𝑥 ∈ 𝐶) & ⊢ ((𝜑 ∧ 𝑥𝑅𝑦) → 𝑦:𝐴⟶𝐵) & ⊢ ((𝜑 ∧ 𝑥 ∈ 𝐶) → 𝐴 ∈ 𝑈) & ⊢ ((𝜑 ∧ 𝑥 ∈ 𝐶) → 𝐵 ∈ 𝑉) & ⊢ (𝜑 → 𝐶 ∈ 𝑊) ⇒ ⊢ (𝜑 → {〈𝑥, 𝑦〉 ∣ (𝑥𝑅𝑦 ∧ 𝜓)} ∈ V) |
< Previous Next > |
Copyright terms: Public domain | < Previous Next > |