Theorem List for Intuitionistic Logic Explorer - 5601-5700   *Has distinct variable
 group(s)
| Type | Label | Description | 
| Statement | 
|   | 
| Theorem | fnbrfvb 5601 | 
Equivalence of function value and binary relation.  (Contributed by NM,
       19-Apr-2004.)  (Revised by Mario Carneiro, 28-Apr-2015.)
 | 
| ⊢ ((𝐹 Fn 𝐴 ∧ 𝐵 ∈ 𝐴) → ((𝐹‘𝐵) = 𝐶 ↔ 𝐵𝐹𝐶)) | 
|   | 
| Theorem | fnopfvb 5602 | 
Equivalence of function value and ordered pair membership.  (Contributed
     by NM, 7-Nov-1995.)
 | 
| ⊢ ((𝐹 Fn 𝐴 ∧ 𝐵 ∈ 𝐴) → ((𝐹‘𝐵) = 𝐶 ↔ 〈𝐵, 𝐶〉 ∈ 𝐹)) | 
|   | 
| Theorem | funbrfvb 5603 | 
Equivalence of function value and binary relation.  (Contributed by NM,
     26-Mar-2006.)
 | 
| ⊢ ((Fun 𝐹 ∧ 𝐴 ∈ dom 𝐹) → ((𝐹‘𝐴) = 𝐵 ↔ 𝐴𝐹𝐵)) | 
|   | 
| Theorem | funopfvb 5604 | 
Equivalence of function value and ordered pair membership.  Theorem
     4.3(ii) of [Monk1] p. 42.  (Contributed by
NM, 26-Jan-1997.)
 | 
| ⊢ ((Fun 𝐹 ∧ 𝐴 ∈ dom 𝐹) → ((𝐹‘𝐴) = 𝐵 ↔ 〈𝐴, 𝐵〉 ∈ 𝐹)) | 
|   | 
| Theorem | funbrfv2b 5605 | 
Function value in terms of a binary relation.  (Contributed by Mario
       Carneiro, 19-Mar-2014.)
 | 
| ⊢ (Fun 𝐹 → (𝐴𝐹𝐵 ↔ (𝐴 ∈ dom 𝐹 ∧ (𝐹‘𝐴) = 𝐵))) | 
|   | 
| Theorem | dffn5im 5606* | 
Representation of a function in terms of its values.  The converse holds
       given the law of the excluded middle; as it is we have most of the
       converse via funmpt 5296 and dmmptss 5166.  (Contributed by Jim Kingdon,
       31-Dec-2018.)
 | 
| ⊢ (𝐹 Fn 𝐴 → 𝐹 = (𝑥 ∈ 𝐴 ↦ (𝐹‘𝑥))) | 
|   | 
| Theorem | fnrnfv 5607* | 
The range of a function expressed as a collection of the function's
       values.  (Contributed by NM, 20-Oct-2005.)  (Proof shortened by Mario
       Carneiro, 31-Aug-2015.)
 | 
| ⊢ (𝐹 Fn 𝐴 → ran 𝐹 = {𝑦 ∣ ∃𝑥 ∈ 𝐴 𝑦 = (𝐹‘𝑥)}) | 
|   | 
| Theorem | fvelrnb 5608* | 
A member of a function's range is a value of the function.  (Contributed
       by NM, 31-Oct-1995.)
 | 
| ⊢ (𝐹 Fn 𝐴 → (𝐵 ∈ ran 𝐹 ↔ ∃𝑥 ∈ 𝐴 (𝐹‘𝑥) = 𝐵)) | 
|   | 
| Theorem | dfimafn 5609* | 
Alternate definition of the image of a function.  (Contributed by Raph
       Levien, 20-Nov-2006.)
 | 
| ⊢ ((Fun 𝐹 ∧ 𝐴 ⊆ dom 𝐹) → (𝐹 “ 𝐴) = {𝑦 ∣ ∃𝑥 ∈ 𝐴 (𝐹‘𝑥) = 𝑦}) | 
|   | 
| Theorem | dfimafn2 5610* | 
Alternate definition of the image of a function as an indexed union of
       singletons of function values.  (Contributed by Raph Levien,
       20-Nov-2006.)
 | 
| ⊢ ((Fun 𝐹 ∧ 𝐴 ⊆ dom 𝐹) → (𝐹 “ 𝐴) = ∪
 𝑥 ∈ 𝐴 {(𝐹‘𝑥)}) | 
|   | 
| Theorem | funimass4 5611* | 
Membership relation for the values of a function whose image is a
       subclass.  (Contributed by Raph Levien, 20-Nov-2006.)
 | 
| ⊢ ((Fun 𝐹 ∧ 𝐴 ⊆ dom 𝐹) → ((𝐹 “ 𝐴) ⊆ 𝐵 ↔ ∀𝑥 ∈ 𝐴 (𝐹‘𝑥) ∈ 𝐵)) | 
|   | 
| Theorem | fvelima 5612* | 
Function value in an image.  Part of Theorem 4.4(iii) of [Monk1] p. 42.
       (Contributed by NM, 29-Apr-2004.)  (Proof shortened by Andrew Salmon,
       22-Oct-2011.)
 | 
| ⊢ ((Fun 𝐹 ∧ 𝐴 ∈ (𝐹 “ 𝐵)) → ∃𝑥 ∈ 𝐵 (𝐹‘𝑥) = 𝐴) | 
|   | 
| Theorem | foelcdmi 5613* | 
A member of a surjective function's codomain is a value of the function.
       (Contributed by Thierry Arnoux, 23-Jan-2020.)
 | 
| ⊢ ((𝐹:𝐴–onto→𝐵 ∧ 𝑌 ∈ 𝐵) → ∃𝑥 ∈ 𝐴 (𝐹‘𝑥) = 𝑌) | 
|   | 
| Theorem | feqmptd 5614* | 
Deduction form of dffn5im 5606.  (Contributed by Mario Carneiro,
       8-Jan-2015.)
 | 
| ⊢ (𝜑 → 𝐹:𝐴⟶𝐵)    ⇒   ⊢ (𝜑 → 𝐹 = (𝑥 ∈ 𝐴 ↦ (𝐹‘𝑥))) | 
|   | 
| Theorem | feqresmpt 5615* | 
Express a restricted function as a mapping.  (Contributed by Mario
       Carneiro, 18-May-2016.)
 | 
| ⊢ (𝜑 → 𝐹:𝐴⟶𝐵)   
 &   ⊢ (𝜑 → 𝐶 ⊆ 𝐴)    ⇒   ⊢ (𝜑 → (𝐹 ↾ 𝐶) = (𝑥 ∈ 𝐶 ↦ (𝐹‘𝑥))) | 
|   | 
| Theorem | dffn5imf 5616* | 
Representation of a function in terms of its values.  (Contributed by
       Jim Kingdon, 31-Dec-2018.)
 | 
| ⊢ Ⅎ𝑥𝐹    ⇒   ⊢ (𝐹 Fn 𝐴 → 𝐹 = (𝑥 ∈ 𝐴 ↦ (𝐹‘𝑥))) | 
|   | 
| Theorem | fvelimab 5617* | 
Function value in an image.  (Contributed by NM, 20-Jan-2007.)  (Proof
       shortened by Andrew Salmon, 22-Oct-2011.)  (Revised by David Abernethy,
       17-Dec-2011.)
 | 
| ⊢ ((𝐹 Fn 𝐴 ∧ 𝐵 ⊆ 𝐴) → (𝐶 ∈ (𝐹 “ 𝐵) ↔ ∃𝑥 ∈ 𝐵 (𝐹‘𝑥) = 𝐶)) | 
|   | 
| Theorem | fvi 5618 | 
The value of the identity function.  (Contributed by NM, 1-May-2004.)
     (Revised by Mario Carneiro, 28-Apr-2015.)
 | 
| ⊢ (𝐴 ∈ 𝑉 → ( I ‘𝐴) = 𝐴) | 
|   | 
| Theorem | fniinfv 5619* | 
The indexed intersection of a function's values is the intersection of
       its range.  (Contributed by NM, 20-Oct-2005.)
 | 
| ⊢ (𝐹 Fn 𝐴 → ∩
 𝑥 ∈ 𝐴 (𝐹‘𝑥) = ∩ ran 𝐹) | 
|   | 
| Theorem | fnsnfv 5620 | 
Singleton of function value.  (Contributed by NM, 22-May-1998.)
 | 
| ⊢ ((𝐹 Fn 𝐴 ∧ 𝐵 ∈ 𝐴) → {(𝐹‘𝐵)} = (𝐹 “ {𝐵})) | 
|   | 
| Theorem | fnimapr 5621 | 
The image of a pair under a function.  (Contributed by Jeff Madsen,
     6-Jan-2011.)
 | 
| ⊢ ((𝐹 Fn 𝐴 ∧ 𝐵 ∈ 𝐴 ∧ 𝐶 ∈ 𝐴) → (𝐹 “ {𝐵, 𝐶}) = {(𝐹‘𝐵), (𝐹‘𝐶)}) | 
|   | 
| Theorem | ssimaex 5622* | 
The existence of a subimage.  (Contributed by NM, 8-Apr-2007.)
 | 
| ⊢ 𝐴 ∈ V    ⇒   ⊢ ((Fun 𝐹 ∧ 𝐵 ⊆ (𝐹 “ 𝐴)) → ∃𝑥(𝑥 ⊆ 𝐴 ∧ 𝐵 = (𝐹 “ 𝑥))) | 
|   | 
| Theorem | ssimaexg 5623* | 
The existence of a subimage.  (Contributed by FL, 15-Apr-2007.)
 | 
| ⊢ ((𝐴 ∈ 𝐶 ∧ Fun 𝐹 ∧ 𝐵 ⊆ (𝐹 “ 𝐴)) → ∃𝑥(𝑥 ⊆ 𝐴 ∧ 𝐵 = (𝐹 “ 𝑥))) | 
|   | 
| Theorem | funfvdm 5624 | 
A simplified expression for the value of a function when we know it's a
     function.  (Contributed by Jim Kingdon, 1-Jan-2019.)
 | 
| ⊢ ((Fun 𝐹 ∧ 𝐴 ∈ dom 𝐹) → (𝐹‘𝐴) = ∪ (𝐹 “ {𝐴})) | 
|   | 
| Theorem | funfvdm2 5625* | 
The value of a function.  Definition of function value in [Enderton]
       p. 43.  (Contributed by Jim Kingdon, 1-Jan-2019.)
 | 
| ⊢ ((Fun 𝐹 ∧ 𝐴 ∈ dom 𝐹) → (𝐹‘𝐴) = ∪ {𝑦 ∣ 𝐴𝐹𝑦}) | 
|   | 
| Theorem | funfvdm2f 5626 | 
The value of a function.  Version of funfvdm2 5625 using a bound-variable
       hypotheses instead of distinct variable conditions.  (Contributed by Jim
       Kingdon, 1-Jan-2019.)
 | 
| ⊢ Ⅎ𝑦𝐴   
 &   ⊢ Ⅎ𝑦𝐹    ⇒   ⊢ ((Fun 𝐹 ∧ 𝐴 ∈ dom 𝐹) → (𝐹‘𝐴) = ∪ {𝑦 ∣ 𝐴𝐹𝑦}) | 
|   | 
| Theorem | fvun1 5627 | 
The value of a union when the argument is in the first domain.
     (Contributed by Scott Fenton, 29-Jun-2013.)
 | 
| ⊢ ((𝐹 Fn 𝐴 ∧ 𝐺 Fn 𝐵 ∧ ((𝐴 ∩ 𝐵) = ∅ ∧ 𝑋 ∈ 𝐴)) → ((𝐹 ∪ 𝐺)‘𝑋) = (𝐹‘𝑋)) | 
|   | 
| Theorem | fvun2 5628 | 
The value of a union when the argument is in the second domain.
     (Contributed by Scott Fenton, 29-Jun-2013.)
 | 
| ⊢ ((𝐹 Fn 𝐴 ∧ 𝐺 Fn 𝐵 ∧ ((𝐴 ∩ 𝐵) = ∅ ∧ 𝑋 ∈ 𝐵)) → ((𝐹 ∪ 𝐺)‘𝑋) = (𝐺‘𝑋)) | 
|   | 
| Theorem | dmfco 5629 | 
Domains of a function composition.  (Contributed by NM, 27-Jan-1997.)
 | 
| ⊢ ((Fun 𝐺 ∧ 𝐴 ∈ dom 𝐺) → (𝐴 ∈ dom (𝐹 ∘ 𝐺) ↔ (𝐺‘𝐴) ∈ dom 𝐹)) | 
|   | 
| Theorem | fvco2 5630 | 
Value of a function composition.  Similar to second part of Theorem 3H
       of [Enderton] p. 47.  (Contributed by
NM, 9-Oct-2004.)  (Proof shortened
       by Andrew Salmon, 22-Oct-2011.)  (Revised by Stefan O'Rear,
       16-Oct-2014.)
 | 
| ⊢ ((𝐺 Fn 𝐴 ∧ 𝑋 ∈ 𝐴) → ((𝐹 ∘ 𝐺)‘𝑋) = (𝐹‘(𝐺‘𝑋))) | 
|   | 
| Theorem | fvco 5631 | 
Value of a function composition.  Similar to Exercise 5 of [TakeutiZaring]
     p. 28.  (Contributed by NM, 22-Apr-2006.)  (Proof shortened by Mario
     Carneiro, 26-Dec-2014.)
 | 
| ⊢ ((Fun 𝐺 ∧ 𝐴 ∈ dom 𝐺) → ((𝐹 ∘ 𝐺)‘𝐴) = (𝐹‘(𝐺‘𝐴))) | 
|   | 
| Theorem | fvco3 5632 | 
Value of a function composition.  (Contributed by NM, 3-Jan-2004.)
     (Revised by Mario Carneiro, 26-Dec-2014.)
 | 
| ⊢ ((𝐺:𝐴⟶𝐵 ∧ 𝐶 ∈ 𝐴) → ((𝐹 ∘ 𝐺)‘𝐶) = (𝐹‘(𝐺‘𝐶))) | 
|   | 
| Theorem | fvco4 5633 | 
Value of a composition.  (Contributed by BJ, 7-Jul-2022.)
 | 
| ⊢ (((𝐾:𝐴⟶𝑋 ∧ (𝐻 ∘ 𝐾) = 𝐹) ∧ (𝑢 ∈ 𝐴 ∧ 𝑥 = (𝐾‘𝑢))) → (𝐻‘𝑥) = (𝐹‘𝑢)) | 
|   | 
| Theorem | fvopab3g 5634* | 
Value of a function given by ordered-pair class abstraction.
       (Contributed by NM, 6-Mar-1996.)  (Revised by Mario Carneiro,
       28-Apr-2015.)
 | 
| ⊢ (𝑥 = 𝐴 → (𝜑 ↔ 𝜓))    &   ⊢ (𝑦 = 𝐵 → (𝜓 ↔ 𝜒))    &   ⊢ (𝑥 ∈ 𝐶 → ∃!𝑦𝜑)   
 &   ⊢ 𝐹 = {〈𝑥, 𝑦〉 ∣ (𝑥 ∈ 𝐶 ∧ 𝜑)}    ⇒   ⊢ ((𝐴 ∈ 𝐶 ∧ 𝐵 ∈ 𝐷) → ((𝐹‘𝐴) = 𝐵 ↔ 𝜒)) | 
|   | 
| Theorem | fvopab3ig 5635* | 
Value of a function given by ordered-pair class abstraction.
       (Contributed by NM, 23-Oct-1999.)
 | 
| ⊢ (𝑥 = 𝐴 → (𝜑 ↔ 𝜓))    &   ⊢ (𝑦 = 𝐵 → (𝜓 ↔ 𝜒))    &   ⊢ (𝑥 ∈ 𝐶 → ∃*𝑦𝜑)   
 &   ⊢ 𝐹 = {〈𝑥, 𝑦〉 ∣ (𝑥 ∈ 𝐶 ∧ 𝜑)}    ⇒   ⊢ ((𝐴 ∈ 𝐶 ∧ 𝐵 ∈ 𝐷) → (𝜒 → (𝐹‘𝐴) = 𝐵)) | 
|   | 
| Theorem | fvmptss2 5636* | 
A mapping always evaluates to a subset of the substituted expression in
       the mapping, even if this is a proper class, or we are out of the
       domain.  (Contributed by Mario Carneiro, 13-Feb-2015.)  (Revised by
       Mario Carneiro, 3-Jul-2019.)
 | 
| ⊢ (𝑥 = 𝐷 → 𝐵 = 𝐶)   
 &   ⊢ 𝐹 = (𝑥 ∈ 𝐴 ↦ 𝐵)    ⇒   ⊢ (𝐹‘𝐷) ⊆ 𝐶 | 
|   | 
| Theorem | fvmptg 5637* | 
Value of a function given in maps-to notation.  (Contributed by NM,
       2-Oct-2007.)  (Revised by Mario Carneiro, 31-Aug-2015.)
 | 
| ⊢ (𝑥 = 𝐴 → 𝐵 = 𝐶)   
 &   ⊢ 𝐹 = (𝑥 ∈ 𝐷 ↦ 𝐵)    ⇒   ⊢ ((𝐴 ∈ 𝐷 ∧ 𝐶 ∈ 𝑅) → (𝐹‘𝐴) = 𝐶) | 
|   | 
| Theorem | fvmpt 5638* | 
Value of a function given in maps-to notation.  (Contributed by NM,
         17-Aug-2011.)
 | 
| ⊢ (𝑥 = 𝐴 → 𝐵 = 𝐶)   
 &   ⊢ 𝐹 = (𝑥 ∈ 𝐷 ↦ 𝐵)   
 &   ⊢ 𝐶 ∈ V    ⇒   ⊢ (𝐴 ∈ 𝐷 → (𝐹‘𝐴) = 𝐶) | 
|   | 
| Theorem | fvmpts 5639* | 
Value of a function given in maps-to notation, using explicit class
       substitution.  (Contributed by Scott Fenton, 17-Jul-2013.)  (Revised by
       Mario Carneiro, 31-Aug-2015.)
 | 
| ⊢ 𝐹 = (𝑥 ∈ 𝐶 ↦ 𝐵)    ⇒   ⊢ ((𝐴 ∈ 𝐶 ∧ ⦋𝐴 / 𝑥⦌𝐵 ∈ 𝑉) → (𝐹‘𝐴) = ⦋𝐴 / 𝑥⦌𝐵) | 
|   | 
| Theorem | fvmpt3 5640* | 
Value of a function given in maps-to notation, with a slightly
         different sethood condition.  (Contributed by Stefan O'Rear,
         30-Jan-2015.)
 | 
| ⊢ (𝑥 = 𝐴 → 𝐵 = 𝐶)   
 &   ⊢ 𝐹 = (𝑥 ∈ 𝐷 ↦ 𝐵)   
 &   ⊢ (𝑥 ∈ 𝐷 → 𝐵 ∈ 𝑉)    ⇒   ⊢ (𝐴 ∈ 𝐷 → (𝐹‘𝐴) = 𝐶) | 
|   | 
| Theorem | fvmpt3i 5641* | 
Value of a function given in maps-to notation, with a slightly different
       sethood condition.  (Contributed by Mario Carneiro, 11-Sep-2015.)
 | 
| ⊢ (𝑥 = 𝐴 → 𝐵 = 𝐶)   
 &   ⊢ 𝐹 = (𝑥 ∈ 𝐷 ↦ 𝐵)   
 &   ⊢ 𝐵 ∈ V    ⇒   ⊢ (𝐴 ∈ 𝐷 → (𝐹‘𝐴) = 𝐶) | 
|   | 
| Theorem | fvmptd 5642* | 
Deduction version of fvmpt 5638.  (Contributed by Scott Fenton,
       18-Feb-2013.)  (Revised by Mario Carneiro, 31-Aug-2015.)
 | 
| ⊢ (𝜑 → 𝐹 = (𝑥 ∈ 𝐷 ↦ 𝐵))    &   ⊢ ((𝜑 ∧ 𝑥 = 𝐴) → 𝐵 = 𝐶)   
 &   ⊢ (𝜑 → 𝐴 ∈ 𝐷)   
 &   ⊢ (𝜑 → 𝐶 ∈ 𝑉)    ⇒   ⊢ (𝜑 → (𝐹‘𝐴) = 𝐶) | 
|   | 
| Theorem | fvmptd2 5643* | 
Deduction version of fvmpt 5638 (where the definition of the mapping does
       not depend on the common antecedent 𝜑).  (Contributed by Glauco
       Siliprandi, 23-Oct-2021.)
 | 
| ⊢ 𝐹 = (𝑥 ∈ 𝐷 ↦ 𝐵)   
 &   ⊢ ((𝜑 ∧ 𝑥 = 𝐴) → 𝐵 = 𝐶)   
 &   ⊢ (𝜑 → 𝐴 ∈ 𝐷)   
 &   ⊢ (𝜑 → 𝐶 ∈ 𝑉)    ⇒   ⊢ (𝜑 → (𝐹‘𝐴) = 𝐶) | 
|   | 
| Theorem | mptrcl 5644* | 
Reverse closure for a mapping:  If the function value of a mapping has a
       member, the argument belongs to the base class of the mapping.
       (Contributed by AV, 4-Apr-2020.)  (Revised by Jim Kingdon,
       27-Mar-2023.)
 | 
| ⊢ 𝐹 = (𝑥 ∈ 𝐴 ↦ 𝐵)    ⇒   ⊢ (𝐼 ∈ (𝐹‘𝑋) → 𝑋 ∈ 𝐴) | 
|   | 
| Theorem | fvmpt2 5645* | 
Value of a function given by the maps-to notation.  (Contributed by FL,
       21-Jun-2010.)
 | 
| ⊢ 𝐹 = (𝑥 ∈ 𝐴 ↦ 𝐵)    ⇒   ⊢ ((𝑥 ∈ 𝐴 ∧ 𝐵 ∈ 𝐶) → (𝐹‘𝑥) = 𝐵) | 
|   | 
| Theorem | fvmptssdm 5646* | 
If all the values of the mapping are subsets of a class 𝐶, then so
       is any evaluation of the mapping at a value in the domain of the
       mapping.  (Contributed by Jim Kingdon, 3-Jan-2018.)
 | 
| ⊢ 𝐹 = (𝑥 ∈ 𝐴 ↦ 𝐵)    ⇒   ⊢ ((𝐷 ∈ dom 𝐹 ∧ ∀𝑥 ∈ 𝐴 𝐵 ⊆ 𝐶) → (𝐹‘𝐷) ⊆ 𝐶) | 
|   | 
| Theorem | mptfvex 5647* | 
Sufficient condition for a maps-to notation to be set-like.
       (Contributed by Mario Carneiro, 3-Jul-2019.)
 | 
| ⊢ 𝐹 = (𝑥 ∈ 𝐴 ↦ 𝐵)    ⇒   ⊢ ((∀𝑥 𝐵 ∈ 𝑉 ∧ 𝐶 ∈ 𝑊) → (𝐹‘𝐶) ∈ V) | 
|   | 
| Theorem | fvmpt2d 5648* | 
Deduction version of fvmpt2 5645.  (Contributed by Thierry Arnoux,
       8-Dec-2016.)
 | 
| ⊢ (𝜑 → 𝐹 = (𝑥 ∈ 𝐴 ↦ 𝐵))    &   ⊢ ((𝜑 ∧ 𝑥 ∈ 𝐴) → 𝐵 ∈ 𝑉)    ⇒   ⊢ ((𝜑 ∧ 𝑥 ∈ 𝐴) → (𝐹‘𝑥) = 𝐵) | 
|   | 
| Theorem | fvmptdf 5649* | 
Alternate deduction version of fvmpt 5638, suitable for iteration.
         (Contributed by Mario Carneiro, 7-Jan-2017.)
 | 
| ⊢ (𝜑 → 𝐴 ∈ 𝐷)   
 &   ⊢ ((𝜑 ∧ 𝑥 = 𝐴) → 𝐵 ∈ 𝑉)   
 &   ⊢ ((𝜑 ∧ 𝑥 = 𝐴) → ((𝐹‘𝐴) = 𝐵 → 𝜓))    &   ⊢
 Ⅎ𝑥𝐹   
 &   ⊢ Ⅎ𝑥𝜓    ⇒   ⊢ (𝜑 → (𝐹 = (𝑥 ∈ 𝐷 ↦ 𝐵) → 𝜓)) | 
|   | 
| Theorem | fvmptdv 5650* | 
Alternate deduction version of fvmpt 5638, suitable for iteration.
       (Contributed by Mario Carneiro, 7-Jan-2017.)
 | 
| ⊢ (𝜑 → 𝐴 ∈ 𝐷)   
 &   ⊢ ((𝜑 ∧ 𝑥 = 𝐴) → 𝐵 ∈ 𝑉)   
 &   ⊢ ((𝜑 ∧ 𝑥 = 𝐴) → ((𝐹‘𝐴) = 𝐵 → 𝜓))    ⇒   ⊢ (𝜑 → (𝐹 = (𝑥 ∈ 𝐷 ↦ 𝐵) → 𝜓)) | 
|   | 
| Theorem | fvmptdv2 5651* | 
Alternate deduction version of fvmpt 5638, suitable for iteration.
       (Contributed by Mario Carneiro, 7-Jan-2017.)
 | 
| ⊢ (𝜑 → 𝐴 ∈ 𝐷)   
 &   ⊢ ((𝜑 ∧ 𝑥 = 𝐴) → 𝐵 ∈ 𝑉)   
 &   ⊢ ((𝜑 ∧ 𝑥 = 𝐴) → 𝐵 = 𝐶)    ⇒   ⊢ (𝜑 → (𝐹 = (𝑥 ∈ 𝐷 ↦ 𝐵) → (𝐹‘𝐴) = 𝐶)) | 
|   | 
| Theorem | mpteqb 5652* | 
Bidirectional equality theorem for a mapping abstraction.  Equivalent to
       eqfnfv 5659.  (Contributed by Mario Carneiro,
14-Nov-2014.)
 | 
| ⊢ (∀𝑥 ∈ 𝐴 𝐵 ∈ 𝑉 → ((𝑥 ∈ 𝐴 ↦ 𝐵) = (𝑥 ∈ 𝐴 ↦ 𝐶) ↔ ∀𝑥 ∈ 𝐴 𝐵 = 𝐶)) | 
|   | 
| Theorem | fvmptt 5653* | 
Closed theorem form of fvmpt 5638.  (Contributed by Scott Fenton,
       21-Feb-2013.)  (Revised by Mario Carneiro, 11-Sep-2015.)
 | 
| ⊢ ((∀𝑥(𝑥 = 𝐴 → 𝐵 = 𝐶) ∧ 𝐹 = (𝑥 ∈ 𝐷 ↦ 𝐵) ∧ (𝐴 ∈ 𝐷 ∧ 𝐶 ∈ 𝑉)) → (𝐹‘𝐴) = 𝐶) | 
|   | 
| Theorem | fvmptf 5654* | 
Value of a function given by an ordered-pair class abstraction.  This
       version of fvmptg 5637 uses bound-variable hypotheses instead of
distinct
       variable conditions.  (Contributed by NM, 8-Nov-2005.)  (Revised by
       Mario Carneiro, 15-Oct-2016.)
 | 
| ⊢ Ⅎ𝑥𝐴   
 &   ⊢ Ⅎ𝑥𝐶   
 &   ⊢ (𝑥 = 𝐴 → 𝐵 = 𝐶)   
 &   ⊢ 𝐹 = (𝑥 ∈ 𝐷 ↦ 𝐵)    ⇒   ⊢ ((𝐴 ∈ 𝐷 ∧ 𝐶 ∈ 𝑉) → (𝐹‘𝐴) = 𝐶) | 
|   | 
| Theorem | fvmptd3 5655* | 
Deduction version of fvmpt 5638.  (Contributed by Glauco Siliprandi,
       23-Oct-2021.)
 | 
| ⊢ 𝐹 = (𝑥 ∈ 𝐷 ↦ 𝐵)   
 &   ⊢ (𝑥 = 𝐴 → 𝐵 = 𝐶)   
 &   ⊢ (𝜑 → 𝐴 ∈ 𝐷)   
 &   ⊢ (𝜑 → 𝐶 ∈ 𝑉)    ⇒   ⊢ (𝜑 → (𝐹‘𝐴) = 𝐶) | 
|   | 
| Theorem | elfvmptrab1 5656* | 
Implications for the value of a function defined by the maps-to notation
       with a class abstraction as a result having an element.  Here, the base
       set of the class abstraction depends on the argument of the function.
       (Contributed by Alexander van der Vekens, 15-Jul-2018.)
 | 
| ⊢ 𝐹 = (𝑥 ∈ 𝑉 ↦ {𝑦 ∈ ⦋𝑥 / 𝑚⦌𝑀 ∣ 𝜑})    &   ⊢ (𝑋 ∈ 𝑉 → ⦋𝑋 / 𝑚⦌𝑀 ∈ V)    ⇒   ⊢ (𝑌 ∈ (𝐹‘𝑋) → (𝑋 ∈ 𝑉 ∧ 𝑌 ∈ ⦋𝑋 / 𝑚⦌𝑀)) | 
|   | 
| Theorem | elfvmptrab 5657* | 
Implications for the value of a function defined by the maps-to notation
       with a class abstraction as a result having an element.  (Contributed by
       Alexander van der Vekens, 15-Jul-2018.)
 | 
| ⊢ 𝐹 = (𝑥 ∈ 𝑉 ↦ {𝑦 ∈ 𝑀 ∣ 𝜑})    &   ⊢ (𝑋 ∈ 𝑉 → 𝑀 ∈ V)    ⇒   ⊢ (𝑌 ∈ (𝐹‘𝑋) → (𝑋 ∈ 𝑉 ∧ 𝑌 ∈ 𝑀)) | 
|   | 
| Theorem | fvopab6 5658* | 
Value of a function given by ordered-pair class abstraction.
       (Contributed by Jeff Madsen, 2-Sep-2009.)  (Revised by Mario Carneiro,
       11-Sep-2015.)
 | 
| ⊢ 𝐹 = {〈𝑥, 𝑦〉 ∣ (𝜑 ∧ 𝑦 = 𝐵)}    &   ⊢ (𝑥 = 𝐴 → (𝜑 ↔ 𝜓))    &   ⊢ (𝑥 = 𝐴 → 𝐵 = 𝐶)    ⇒   ⊢ ((𝐴 ∈ 𝐷 ∧ 𝐶 ∈ 𝑅 ∧ 𝜓) → (𝐹‘𝐴) = 𝐶) | 
|   | 
| Theorem | eqfnfv 5659* | 
Equality of functions is determined by their values.  Special case of
       Exercise 4 of [TakeutiZaring] p.
28 (with domain equality omitted).
       (Contributed by NM, 3-Aug-1994.)  (Proof shortened by Andrew Salmon,
       22-Oct-2011.)  (Proof shortened by Mario Carneiro, 31-Aug-2015.)
 | 
| ⊢ ((𝐹 Fn 𝐴 ∧ 𝐺 Fn 𝐴) → (𝐹 = 𝐺 ↔ ∀𝑥 ∈ 𝐴 (𝐹‘𝑥) = (𝐺‘𝑥))) | 
|   | 
| Theorem | eqfnfv2 5660* | 
Equality of functions is determined by their values.  Exercise 4 of
       [TakeutiZaring] p. 28. 
(Contributed by NM, 3-Aug-1994.)  (Revised by
       Mario Carneiro, 31-Aug-2015.)
 | 
| ⊢ ((𝐹 Fn 𝐴 ∧ 𝐺 Fn 𝐵) → (𝐹 = 𝐺 ↔ (𝐴 = 𝐵 ∧ ∀𝑥 ∈ 𝐴 (𝐹‘𝑥) = (𝐺‘𝑥)))) | 
|   | 
| Theorem | eqfnfv3 5661* | 
Derive equality of functions from equality of their values.
       (Contributed by Jeff Madsen, 2-Sep-2009.)
 | 
| ⊢ ((𝐹 Fn 𝐴 ∧ 𝐺 Fn 𝐵) → (𝐹 = 𝐺 ↔ (𝐵 ⊆ 𝐴 ∧ ∀𝑥 ∈ 𝐴 (𝑥 ∈ 𝐵 ∧ (𝐹‘𝑥) = (𝐺‘𝑥))))) | 
|   | 
| Theorem | eqfnfvd 5662* | 
Deduction for equality of functions.  (Contributed by Mario Carneiro,
       24-Jul-2014.)
 | 
| ⊢ (𝜑 → 𝐹 Fn 𝐴)   
 &   ⊢ (𝜑 → 𝐺 Fn 𝐴)   
 &   ⊢ ((𝜑 ∧ 𝑥 ∈ 𝐴) → (𝐹‘𝑥) = (𝐺‘𝑥))    ⇒   ⊢ (𝜑 → 𝐹 = 𝐺) | 
|   | 
| Theorem | eqfnfv2f 5663* | 
Equality of functions is determined by their values.  Special case of
       Exercise 4 of [TakeutiZaring] p.
28 (with domain equality omitted).
       This version of eqfnfv 5659 uses bound-variable hypotheses instead of
       distinct variable conditions.  (Contributed by NM, 29-Jan-2004.)
 | 
| ⊢ Ⅎ𝑥𝐹   
 &   ⊢ Ⅎ𝑥𝐺    ⇒   ⊢ ((𝐹 Fn 𝐴 ∧ 𝐺 Fn 𝐴) → (𝐹 = 𝐺 ↔ ∀𝑥 ∈ 𝐴 (𝐹‘𝑥) = (𝐺‘𝑥))) | 
|   | 
| Theorem | eqfunfv 5664* | 
Equality of functions is determined by their values.  (Contributed by
       Scott Fenton, 19-Jun-2011.)
 | 
| ⊢ ((Fun 𝐹 ∧ Fun 𝐺) → (𝐹 = 𝐺 ↔ (dom 𝐹 = dom 𝐺 ∧ ∀𝑥 ∈ dom 𝐹(𝐹‘𝑥) = (𝐺‘𝑥)))) | 
|   | 
| Theorem | fvreseq 5665* | 
Equality of restricted functions is determined by their values.
       (Contributed by NM, 3-Aug-1994.)
 | 
| ⊢ (((𝐹 Fn 𝐴 ∧ 𝐺 Fn 𝐴) ∧ 𝐵 ⊆ 𝐴) → ((𝐹 ↾ 𝐵) = (𝐺 ↾ 𝐵) ↔ ∀𝑥 ∈ 𝐵 (𝐹‘𝑥) = (𝐺‘𝑥))) | 
|   | 
| Theorem | fnmptfvd 5666* | 
A function with a given domain is a mapping defined by its function
       values.  (Contributed by AV, 1-Mar-2019.)
 | 
| ⊢ (𝜑 → 𝑀 Fn 𝐴)   
 &   ⊢ (𝑖 = 𝑎 → 𝐷 = 𝐶)   
 &   ⊢ ((𝜑 ∧ 𝑖 ∈ 𝐴) → 𝐷 ∈ 𝑈)   
 &   ⊢ ((𝜑 ∧ 𝑎 ∈ 𝐴) → 𝐶 ∈ 𝑉)    ⇒   ⊢ (𝜑 → (𝑀 = (𝑎 ∈ 𝐴 ↦ 𝐶) ↔ ∀𝑖 ∈ 𝐴 (𝑀‘𝑖) = 𝐷)) | 
|   | 
| Theorem | fndmdif 5667* | 
Two ways to express the locus of differences between two functions.
       (Contributed by Stefan O'Rear, 17-Jan-2015.)
 | 
| ⊢ ((𝐹 Fn 𝐴 ∧ 𝐺 Fn 𝐴) → dom (𝐹 ∖ 𝐺) = {𝑥 ∈ 𝐴 ∣ (𝐹‘𝑥) ≠ (𝐺‘𝑥)}) | 
|   | 
| Theorem | fndmdifcom 5668 | 
The difference set between two functions is commutative.  (Contributed
       by Stefan O'Rear, 17-Jan-2015.)
 | 
| ⊢ ((𝐹 Fn 𝐴 ∧ 𝐺 Fn 𝐴) → dom (𝐹 ∖ 𝐺) = dom (𝐺 ∖ 𝐹)) | 
|   | 
| Theorem | fndmin 5669* | 
Two ways to express the locus of equality between two functions.
       (Contributed by Stefan O'Rear, 17-Jan-2015.)
 | 
| ⊢ ((𝐹 Fn 𝐴 ∧ 𝐺 Fn 𝐴) → dom (𝐹 ∩ 𝐺) = {𝑥 ∈ 𝐴 ∣ (𝐹‘𝑥) = (𝐺‘𝑥)}) | 
|   | 
| Theorem | fneqeql 5670 | 
Two functions are equal iff their equalizer is the whole domain.
       (Contributed by Stefan O'Rear, 7-Mar-2015.)
 | 
| ⊢ ((𝐹 Fn 𝐴 ∧ 𝐺 Fn 𝐴) → (𝐹 = 𝐺 ↔ dom (𝐹 ∩ 𝐺) = 𝐴)) | 
|   | 
| Theorem | fneqeql2 5671 | 
Two functions are equal iff their equalizer contains the whole domain.
       (Contributed by Stefan O'Rear, 9-Mar-2015.)
 | 
| ⊢ ((𝐹 Fn 𝐴 ∧ 𝐺 Fn 𝐴) → (𝐹 = 𝐺 ↔ 𝐴 ⊆ dom (𝐹 ∩ 𝐺))) | 
|   | 
| Theorem | fnreseql 5672 | 
Two functions are equal on a subset iff their equalizer contains that
       subset.  (Contributed by Stefan O'Rear, 7-Mar-2015.)
 | 
| ⊢ ((𝐹 Fn 𝐴 ∧ 𝐺 Fn 𝐴 ∧ 𝑋 ⊆ 𝐴) → ((𝐹 ↾ 𝑋) = (𝐺 ↾ 𝑋) ↔ 𝑋 ⊆ dom (𝐹 ∩ 𝐺))) | 
|   | 
| Theorem | chfnrn 5673* | 
The range of a choice function (a function that chooses an element from
       each member of its domain) is included in the union of its domain.
       (Contributed by NM, 31-Aug-1999.)
 | 
| ⊢ ((𝐹 Fn 𝐴 ∧ ∀𝑥 ∈ 𝐴 (𝐹‘𝑥) ∈ 𝑥) → ran 𝐹 ⊆ ∪ 𝐴) | 
|   | 
| Theorem | funfvop 5674 | 
Ordered pair with function value.  Part of Theorem 4.3(i) of [Monk1]
     p. 41.  (Contributed by NM, 14-Oct-1996.)
 | 
| ⊢ ((Fun 𝐹 ∧ 𝐴 ∈ dom 𝐹) → 〈𝐴, (𝐹‘𝐴)〉 ∈ 𝐹) | 
|   | 
| Theorem | funfvbrb 5675 | 
Two ways to say that 𝐴 is in the domain of 𝐹. 
(Contributed by
     Mario Carneiro, 1-May-2014.)
 | 
| ⊢ (Fun 𝐹 → (𝐴 ∈ dom 𝐹 ↔ 𝐴𝐹(𝐹‘𝐴))) | 
|   | 
| Theorem | fvimacnvi 5676 | 
A member of a preimage is a function value argument.  (Contributed by NM,
     4-May-2007.)
 | 
| ⊢ ((Fun 𝐹 ∧ 𝐴 ∈ (◡𝐹 “ 𝐵)) → (𝐹‘𝐴) ∈ 𝐵) | 
|   | 
| Theorem | fvimacnv 5677 | 
The argument of a function value belongs to the preimage of any class
     containing the function value.  Raph Levien remarks:  "This proof is
     unsatisfying, because it seems to me that funimass2 5336 could probably be
     strengthened to a biconditional."  (Contributed by Raph Levien,
     20-Nov-2006.)
 | 
| ⊢ ((Fun 𝐹 ∧ 𝐴 ∈ dom 𝐹) → ((𝐹‘𝐴) ∈ 𝐵 ↔ 𝐴 ∈ (◡𝐹 “ 𝐵))) | 
|   | 
| Theorem | funimass3 5678 | 
A kind of contraposition law that infers an image subclass from a
       subclass of a preimage.  Raph Levien remarks:  "Likely this could
be
       proved directly, and fvimacnv 5677 would be the special case of 𝐴 being
       a singleton, but it works this way round too."  (Contributed by
Raph
       Levien, 20-Nov-2006.)
 | 
| ⊢ ((Fun 𝐹 ∧ 𝐴 ⊆ dom 𝐹) → ((𝐹 “ 𝐴) ⊆ 𝐵 ↔ 𝐴 ⊆ (◡𝐹 “ 𝐵))) | 
|   | 
| Theorem | funimass5 5679* | 
A subclass of a preimage in terms of function values.  (Contributed by
       NM, 15-May-2007.)
 | 
| ⊢ ((Fun 𝐹 ∧ 𝐴 ⊆ dom 𝐹) → (𝐴 ⊆ (◡𝐹 “ 𝐵) ↔ ∀𝑥 ∈ 𝐴 (𝐹‘𝑥) ∈ 𝐵)) | 
|   | 
| Theorem | funconstss 5680* | 
Two ways of specifying that a function is constant on a subdomain.
       (Contributed by NM, 8-Mar-2007.)
 | 
| ⊢ ((Fun 𝐹 ∧ 𝐴 ⊆ dom 𝐹) → (∀𝑥 ∈ 𝐴 (𝐹‘𝑥) = 𝐵 ↔ 𝐴 ⊆ (◡𝐹 “ {𝐵}))) | 
|   | 
| Theorem | elpreima 5681 | 
Membership in the preimage of a set under a function.  (Contributed by
     Jeff Madsen, 2-Sep-2009.)
 | 
| ⊢ (𝐹 Fn 𝐴 → (𝐵 ∈ (◡𝐹 “ 𝐶) ↔ (𝐵 ∈ 𝐴 ∧ (𝐹‘𝐵) ∈ 𝐶))) | 
|   | 
| Theorem | fniniseg 5682 | 
Membership in the preimage of a singleton, under a function.  (Contributed
     by Mario Carneiro, 12-May-2014.)  (Proof shortened by Mario Carneiro,
     28-Apr-2015.)
 | 
| ⊢ (𝐹 Fn 𝐴 → (𝐶 ∈ (◡𝐹 “ {𝐵}) ↔ (𝐶 ∈ 𝐴 ∧ (𝐹‘𝐶) = 𝐵))) | 
|   | 
| Theorem | fncnvima2 5683* | 
Inverse images under functions expressed as abstractions.  (Contributed
       by Stefan O'Rear, 1-Feb-2015.)
 | 
| ⊢ (𝐹 Fn 𝐴 → (◡𝐹 “ 𝐵) = {𝑥 ∈ 𝐴 ∣ (𝐹‘𝑥) ∈ 𝐵}) | 
|   | 
| Theorem | fniniseg2 5684* | 
Inverse point images under functions expressed as abstractions.
       (Contributed by Stefan O'Rear, 1-Feb-2015.)
 | 
| ⊢ (𝐹 Fn 𝐴 → (◡𝐹 “ {𝐵}) = {𝑥 ∈ 𝐴 ∣ (𝐹‘𝑥) = 𝐵}) | 
|   | 
| Theorem | fnniniseg2 5685* | 
Support sets of functions expressed as abstractions.  (Contributed by
       Stefan O'Rear, 1-Feb-2015.)
 | 
| ⊢ (𝐹 Fn 𝐴 → (◡𝐹 “ (V ∖ {𝐵})) = {𝑥 ∈ 𝐴 ∣ (𝐹‘𝑥) ≠ 𝐵}) | 
|   | 
| Theorem | rexsupp 5686* | 
Existential quantification restricted to a support.  (Contributed by
       Stefan O'Rear, 23-Mar-2015.)
 | 
| ⊢ (𝐹 Fn 𝐴 → (∃𝑥 ∈ (◡𝐹 “ (V ∖ {𝑍}))𝜑 ↔ ∃𝑥 ∈ 𝐴 ((𝐹‘𝑥) ≠ 𝑍 ∧ 𝜑))) | 
|   | 
| Theorem | unpreima 5687 | 
Preimage of a union.  (Contributed by Jeff Madsen, 2-Sep-2009.)
 | 
| ⊢ (Fun 𝐹 → (◡𝐹 “ (𝐴 ∪ 𝐵)) = ((◡𝐹 “ 𝐴) ∪ (◡𝐹 “ 𝐵))) | 
|   | 
| Theorem | inpreima 5688 | 
Preimage of an intersection.  (Contributed by Jeff Madsen, 2-Sep-2009.)
       (Proof shortened by Mario Carneiro, 14-Jun-2016.)
 | 
| ⊢ (Fun 𝐹 → (◡𝐹 “ (𝐴 ∩ 𝐵)) = ((◡𝐹 “ 𝐴) ∩ (◡𝐹 “ 𝐵))) | 
|   | 
| Theorem | difpreima 5689 | 
Preimage of a difference.  (Contributed by Mario Carneiro,
       14-Jun-2016.)
 | 
| ⊢ (Fun 𝐹 → (◡𝐹 “ (𝐴 ∖ 𝐵)) = ((◡𝐹 “ 𝐴) ∖ (◡𝐹 “ 𝐵))) | 
|   | 
| Theorem | respreima 5690 | 
The preimage of a restricted function.  (Contributed by Jeff Madsen,
       2-Sep-2009.)
 | 
| ⊢ (Fun 𝐹 → (◡(𝐹 ↾ 𝐵) “ 𝐴) = ((◡𝐹 “ 𝐴) ∩ 𝐵)) | 
|   | 
| Theorem | fimacnv 5691 | 
The preimage of the codomain of a mapping is the mapping's domain.
     (Contributed by FL, 25-Jan-2007.)
 | 
| ⊢ (𝐹:𝐴⟶𝐵 → (◡𝐹 “ 𝐵) = 𝐴) | 
|   | 
| Theorem | fnopfv 5692 | 
Ordered pair with function value.  Part of Theorem 4.3(i) of [Monk1]
     p. 41.  (Contributed by NM, 30-Sep-2004.)
 | 
| ⊢ ((𝐹 Fn 𝐴 ∧ 𝐵 ∈ 𝐴) → 〈𝐵, (𝐹‘𝐵)〉 ∈ 𝐹) | 
|   | 
| Theorem | fvelrn 5693 | 
A function's value belongs to its range.  (Contributed by NM,
       14-Oct-1996.)
 | 
| ⊢ ((Fun 𝐹 ∧ 𝐴 ∈ dom 𝐹) → (𝐹‘𝐴) ∈ ran 𝐹) | 
|   | 
| Theorem | fnfvelrn 5694 | 
A function's value belongs to its range.  (Contributed by NM,
     15-Oct-1996.)
 | 
| ⊢ ((𝐹 Fn 𝐴 ∧ 𝐵 ∈ 𝐴) → (𝐹‘𝐵) ∈ ran 𝐹) | 
|   | 
| Theorem | ffvelcdm 5695 | 
A function's value belongs to its codomain.  (Contributed by NM,
     12-Aug-1999.)
 | 
| ⊢ ((𝐹:𝐴⟶𝐵 ∧ 𝐶 ∈ 𝐴) → (𝐹‘𝐶) ∈ 𝐵) | 
|   | 
| Theorem | ffvelcdmi 5696 | 
A function's value belongs to its codomain.  (Contributed by NM,
       6-Apr-2005.)
 | 
| ⊢ 𝐹:𝐴⟶𝐵    ⇒   ⊢ (𝐶 ∈ 𝐴 → (𝐹‘𝐶) ∈ 𝐵) | 
|   | 
| Theorem | ffvelcdmda 5697 | 
A function's value belongs to its codomain.  (Contributed by Mario
       Carneiro, 29-Dec-2016.)
 | 
| ⊢ (𝜑 → 𝐹:𝐴⟶𝐵)    ⇒   ⊢ ((𝜑 ∧ 𝐶 ∈ 𝐴) → (𝐹‘𝐶) ∈ 𝐵) | 
|   | 
| Theorem | ffvelcdmd 5698 | 
A function's value belongs to its codomain.  (Contributed by Mario
       Carneiro, 29-Dec-2016.)
 | 
| ⊢ (𝜑 → 𝐹:𝐴⟶𝐵)   
 &   ⊢ (𝜑 → 𝐶 ∈ 𝐴)    ⇒   ⊢ (𝜑 → (𝐹‘𝐶) ∈ 𝐵) | 
|   | 
| Theorem | rexrn 5699* | 
Restricted existential quantification over the range of a function.
       (Contributed by Mario Carneiro, 24-Dec-2013.)  (Revised by Mario
       Carneiro, 20-Aug-2014.)
 | 
| ⊢ (𝑥 = (𝐹‘𝑦) → (𝜑 ↔ 𝜓))    ⇒   ⊢ (𝐹 Fn 𝐴 → (∃𝑥 ∈ ran 𝐹𝜑 ↔ ∃𝑦 ∈ 𝐴 𝜓)) | 
|   | 
| Theorem | ralrn 5700* | 
Restricted universal quantification over the range of a function.
       (Contributed by Mario Carneiro, 24-Dec-2013.)  (Revised by Mario
       Carneiro, 20-Aug-2014.)
 | 
| ⊢ (𝑥 = (𝐹‘𝑦) → (𝜑 ↔ 𝜓))    ⇒   ⊢ (𝐹 Fn 𝐴 → (∀𝑥 ∈ ran 𝐹𝜑 ↔ ∀𝑦 ∈ 𝐴 𝜓)) |