Theorem List for Intuitionistic Logic Explorer - 5501-5600 *Has distinct variable
group(s)
Type | Label | Description |
Statement |
|
Theorem | fvssunirng 5501 |
The result of a function value is always a subset of the union of the
range, if the input is a set. (Contributed by Stefan O'Rear,
2-Nov-2014.) (Revised by Mario Carneiro, 24-May-2019.)
|
⊢ (𝐴 ∈ V → (𝐹‘𝐴) ⊆ ∪ ran
𝐹) |
|
Theorem | relfvssunirn 5502 |
The result of a function value is always a subset of the union of the
range, even if it is invalid and thus empty. (Contributed by Stefan
O'Rear, 2-Nov-2014.) (Revised by Mario Carneiro, 24-May-2019.)
|
⊢ (Rel 𝐹 → (𝐹‘𝐴) ⊆ ∪ ran
𝐹) |
|
Theorem | funfvex 5503 |
The value of a function exists. A special case of Corollary 6.13 of
[TakeutiZaring] p. 27.
(Contributed by Jim Kingdon, 29-Dec-2018.)
|
⊢ ((Fun 𝐹 ∧ 𝐴 ∈ dom 𝐹) → (𝐹‘𝐴) ∈ V) |
|
Theorem | relrnfvex 5504 |
If a function has a set range, then the function value exists
unconditional on the domain. (Contributed by Mario Carneiro,
24-May-2019.)
|
⊢ ((Rel 𝐹 ∧ ran 𝐹 ∈ V) → (𝐹‘𝐴) ∈ V) |
|
Theorem | fvexg 5505 |
Evaluating a set function at a set exists. (Contributed by Mario
Carneiro and Jim Kingdon, 28-May-2019.)
|
⊢ ((𝐹 ∈ 𝑉 ∧ 𝐴 ∈ 𝑊) → (𝐹‘𝐴) ∈ V) |
|
Theorem | fvex 5506 |
Evaluating a set function at a set exists. (Contributed by Mario
Carneiro and Jim Kingdon, 28-May-2019.)
|
⊢ 𝐹 ∈ 𝑉
& ⊢ 𝐴 ∈ 𝑊 ⇒ ⊢ (𝐹‘𝐴) ∈ V |
|
Theorem | sefvex 5507 |
If a function is set-like, then the function value exists if the input
does. (Contributed by Mario Carneiro, 24-May-2019.)
|
⊢ ((◡𝐹 Se V ∧ 𝐴 ∈ V) → (𝐹‘𝐴) ∈ V) |
|
Theorem | fvifdc 5508 |
Move a conditional outside of a function. (Contributed by Jim Kingdon,
1-Jan-2022.)
|
⊢ (DECID 𝜑 → (𝐹‘if(𝜑, 𝐴, 𝐵)) = if(𝜑, (𝐹‘𝐴), (𝐹‘𝐵))) |
|
Theorem | fv3 5509* |
Alternate definition of the value of a function. Definition 6.11 of
[TakeutiZaring] p. 26.
(Contributed by NM, 30-Apr-2004.) (Revised by
Mario Carneiro, 31-Aug-2015.)
|
⊢ (𝐹‘𝐴) = {𝑥 ∣ (∃𝑦(𝑥 ∈ 𝑦 ∧ 𝐴𝐹𝑦) ∧ ∃!𝑦 𝐴𝐹𝑦)} |
|
Theorem | fvres 5510 |
The value of a restricted function. (Contributed by NM, 2-Aug-1994.)
|
⊢ (𝐴 ∈ 𝐵 → ((𝐹 ↾ 𝐵)‘𝐴) = (𝐹‘𝐴)) |
|
Theorem | fvresd 5511 |
The value of a restricted function, deduction version of fvres 5510.
(Contributed by Glauco Siliprandi, 8-Apr-2021.)
|
⊢ (𝜑 → 𝐴 ∈ 𝐵) ⇒ ⊢ (𝜑 → ((𝐹 ↾ 𝐵)‘𝐴) = (𝐹‘𝐴)) |
|
Theorem | funssfv 5512 |
The value of a member of the domain of a subclass of a function.
(Contributed by NM, 15-Aug-1994.)
|
⊢ ((Fun 𝐹 ∧ 𝐺 ⊆ 𝐹 ∧ 𝐴 ∈ dom 𝐺) → (𝐹‘𝐴) = (𝐺‘𝐴)) |
|
Theorem | tz6.12-1 5513* |
Function value. Theorem 6.12(1) of [TakeutiZaring] p. 27. (Contributed
by NM, 30-Apr-2004.)
|
⊢ ((𝐴𝐹𝑦 ∧ ∃!𝑦 𝐴𝐹𝑦) → (𝐹‘𝐴) = 𝑦) |
|
Theorem | tz6.12 5514* |
Function value. Theorem 6.12(1) of [TakeutiZaring] p. 27. (Contributed
by NM, 10-Jul-1994.)
|
⊢ ((〈𝐴, 𝑦〉 ∈ 𝐹 ∧ ∃!𝑦〈𝐴, 𝑦〉 ∈ 𝐹) → (𝐹‘𝐴) = 𝑦) |
|
Theorem | tz6.12f 5515* |
Function value, using bound-variable hypotheses instead of distinct
variable conditions. (Contributed by NM, 30-Aug-1999.)
|
⊢ Ⅎ𝑦𝐹 ⇒ ⊢ ((〈𝐴, 𝑦〉 ∈ 𝐹 ∧ ∃!𝑦〈𝐴, 𝑦〉 ∈ 𝐹) → (𝐹‘𝐴) = 𝑦) |
|
Theorem | tz6.12c 5516* |
Corollary of Theorem 6.12(1) of [TakeutiZaring] p. 27. (Contributed by
NM, 30-Apr-2004.)
|
⊢ (∃!𝑦 𝐴𝐹𝑦 → ((𝐹‘𝐴) = 𝑦 ↔ 𝐴𝐹𝑦)) |
|
Theorem | ndmfvg 5517 |
The value of a class outside its domain is the empty set. (Contributed
by Jim Kingdon, 15-Jan-2019.)
|
⊢ ((𝐴 ∈ V ∧ ¬ 𝐴 ∈ dom 𝐹) → (𝐹‘𝐴) = ∅) |
|
Theorem | relelfvdm 5518 |
If a function value has a member, the argument belongs to the domain.
(Contributed by Jim Kingdon, 22-Jan-2019.)
|
⊢ ((Rel 𝐹 ∧ 𝐴 ∈ (𝐹‘𝐵)) → 𝐵 ∈ dom 𝐹) |
|
Theorem | nfvres 5519 |
The value of a non-member of a restriction is the empty set.
(Contributed by NM, 13-Nov-1995.)
|
⊢ (¬ 𝐴 ∈ 𝐵 → ((𝐹 ↾ 𝐵)‘𝐴) = ∅) |
|
Theorem | nfunsn 5520 |
If the restriction of a class to a singleton is not a function, its
value is the empty set. (Contributed by NM, 8-Aug-2010.) (Proof
shortened by Andrew Salmon, 22-Oct-2011.)
|
⊢ (¬ Fun (𝐹 ↾ {𝐴}) → (𝐹‘𝐴) = ∅) |
|
Theorem | 0fv 5521 |
Function value of the empty set. (Contributed by Stefan O'Rear,
26-Nov-2014.)
|
⊢ (∅‘𝐴) = ∅ |
|
Theorem | csbfv12g 5522 |
Move class substitution in and out of a function value. (Contributed by
NM, 11-Nov-2005.)
|
⊢ (𝐴 ∈ 𝐶 → ⦋𝐴 / 𝑥⦌(𝐹‘𝐵) = (⦋𝐴 / 𝑥⦌𝐹‘⦋𝐴 / 𝑥⦌𝐵)) |
|
Theorem | csbfv2g 5523* |
Move class substitution in and out of a function value. (Contributed by
NM, 10-Nov-2005.)
|
⊢ (𝐴 ∈ 𝐶 → ⦋𝐴 / 𝑥⦌(𝐹‘𝐵) = (𝐹‘⦋𝐴 / 𝑥⦌𝐵)) |
|
Theorem | csbfvg 5524* |
Substitution for a function value. (Contributed by NM, 1-Jan-2006.)
|
⊢ (𝐴 ∈ 𝐶 → ⦋𝐴 / 𝑥⦌(𝐹‘𝑥) = (𝐹‘𝐴)) |
|
Theorem | funbrfv 5525 |
The second argument of a binary relation on a function is the function's
value. (Contributed by NM, 30-Apr-2004.) (Revised by Mario Carneiro,
28-Apr-2015.)
|
⊢ (Fun 𝐹 → (𝐴𝐹𝐵 → (𝐹‘𝐴) = 𝐵)) |
|
Theorem | funopfv 5526 |
The second element in an ordered pair member of a function is the
function's value. (Contributed by NM, 19-Jul-1996.)
|
⊢ (Fun 𝐹 → (〈𝐴, 𝐵〉 ∈ 𝐹 → (𝐹‘𝐴) = 𝐵)) |
|
Theorem | fnbrfvb 5527 |
Equivalence of function value and binary relation. (Contributed by NM,
19-Apr-2004.) (Revised by Mario Carneiro, 28-Apr-2015.)
|
⊢ ((𝐹 Fn 𝐴 ∧ 𝐵 ∈ 𝐴) → ((𝐹‘𝐵) = 𝐶 ↔ 𝐵𝐹𝐶)) |
|
Theorem | fnopfvb 5528 |
Equivalence of function value and ordered pair membership. (Contributed
by NM, 7-Nov-1995.)
|
⊢ ((𝐹 Fn 𝐴 ∧ 𝐵 ∈ 𝐴) → ((𝐹‘𝐵) = 𝐶 ↔ 〈𝐵, 𝐶〉 ∈ 𝐹)) |
|
Theorem | funbrfvb 5529 |
Equivalence of function value and binary relation. (Contributed by NM,
26-Mar-2006.)
|
⊢ ((Fun 𝐹 ∧ 𝐴 ∈ dom 𝐹) → ((𝐹‘𝐴) = 𝐵 ↔ 𝐴𝐹𝐵)) |
|
Theorem | funopfvb 5530 |
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 5531 |
Function value in terms of a binary relation. (Contributed by Mario
Carneiro, 19-Mar-2014.)
|
⊢ (Fun 𝐹 → (𝐴𝐹𝐵 ↔ (𝐴 ∈ dom 𝐹 ∧ (𝐹‘𝐴) = 𝐵))) |
|
Theorem | dffn5im 5532* |
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 5226 and dmmptss 5100. (Contributed by Jim Kingdon,
31-Dec-2018.)
|
⊢ (𝐹 Fn 𝐴 → 𝐹 = (𝑥 ∈ 𝐴 ↦ (𝐹‘𝑥))) |
|
Theorem | fnrnfv 5533* |
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 5534* |
A member of a function's range is a value of the function. (Contributed
by NM, 31-Oct-1995.)
|
⊢ (𝐹 Fn 𝐴 → (𝐵 ∈ ran 𝐹 ↔ ∃𝑥 ∈ 𝐴 (𝐹‘𝑥) = 𝐵)) |
|
Theorem | dfimafn 5535* |
Alternate definition of the image of a function. (Contributed by Raph
Levien, 20-Nov-2006.)
|
⊢ ((Fun 𝐹 ∧ 𝐴 ⊆ dom 𝐹) → (𝐹 “ 𝐴) = {𝑦 ∣ ∃𝑥 ∈ 𝐴 (𝐹‘𝑥) = 𝑦}) |
|
Theorem | dfimafn2 5536* |
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 5537* |
Membership relation for the values of a function whose image is a
subclass. (Contributed by Raph Levien, 20-Nov-2006.)
|
⊢ ((Fun 𝐹 ∧ 𝐴 ⊆ dom 𝐹) → ((𝐹 “ 𝐴) ⊆ 𝐵 ↔ ∀𝑥 ∈ 𝐴 (𝐹‘𝑥) ∈ 𝐵)) |
|
Theorem | fvelima 5538* |
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 | feqmptd 5539* |
Deduction form of dffn5im 5532. (Contributed by Mario Carneiro,
8-Jan-2015.)
|
⊢ (𝜑 → 𝐹:𝐴⟶𝐵) ⇒ ⊢ (𝜑 → 𝐹 = (𝑥 ∈ 𝐴 ↦ (𝐹‘𝑥))) |
|
Theorem | feqresmpt 5540* |
Express a restricted function as a mapping. (Contributed by Mario
Carneiro, 18-May-2016.)
|
⊢ (𝜑 → 𝐹:𝐴⟶𝐵)
& ⊢ (𝜑 → 𝐶 ⊆ 𝐴) ⇒ ⊢ (𝜑 → (𝐹 ↾ 𝐶) = (𝑥 ∈ 𝐶 ↦ (𝐹‘𝑥))) |
|
Theorem | dffn5imf 5541* |
Representation of a function in terms of its values. (Contributed by
Jim Kingdon, 31-Dec-2018.)
|
⊢ Ⅎ𝑥𝐹 ⇒ ⊢ (𝐹 Fn 𝐴 → 𝐹 = (𝑥 ∈ 𝐴 ↦ (𝐹‘𝑥))) |
|
Theorem | fvelimab 5542* |
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 5543 |
The value of the identity function. (Contributed by NM, 1-May-2004.)
(Revised by Mario Carneiro, 28-Apr-2015.)
|
⊢ (𝐴 ∈ 𝑉 → ( I ‘𝐴) = 𝐴) |
|
Theorem | fniinfv 5544* |
The indexed intersection of a function's values is the intersection of
its range. (Contributed by NM, 20-Oct-2005.)
|
⊢ (𝐹 Fn 𝐴 → ∩
𝑥 ∈ 𝐴 (𝐹‘𝑥) = ∩ ran 𝐹) |
|
Theorem | fnsnfv 5545 |
Singleton of function value. (Contributed by NM, 22-May-1998.)
|
⊢ ((𝐹 Fn 𝐴 ∧ 𝐵 ∈ 𝐴) → {(𝐹‘𝐵)} = (𝐹 “ {𝐵})) |
|
Theorem | fnimapr 5546 |
The image of a pair under a function. (Contributed by Jeff Madsen,
6-Jan-2011.)
|
⊢ ((𝐹 Fn 𝐴 ∧ 𝐵 ∈ 𝐴 ∧ 𝐶 ∈ 𝐴) → (𝐹 “ {𝐵, 𝐶}) = {(𝐹‘𝐵), (𝐹‘𝐶)}) |
|
Theorem | ssimaex 5547* |
The existence of a subimage. (Contributed by NM, 8-Apr-2007.)
|
⊢ 𝐴 ∈ V ⇒ ⊢ ((Fun 𝐹 ∧ 𝐵 ⊆ (𝐹 “ 𝐴)) → ∃𝑥(𝑥 ⊆ 𝐴 ∧ 𝐵 = (𝐹 “ 𝑥))) |
|
Theorem | ssimaexg 5548* |
The existence of a subimage. (Contributed by FL, 15-Apr-2007.)
|
⊢ ((𝐴 ∈ 𝐶 ∧ Fun 𝐹 ∧ 𝐵 ⊆ (𝐹 “ 𝐴)) → ∃𝑥(𝑥 ⊆ 𝐴 ∧ 𝐵 = (𝐹 “ 𝑥))) |
|
Theorem | funfvdm 5549 |
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 5550* |
The value of a function. Definition of function value in [Enderton]
p. 43. (Contributed by Jim Kingdon, 1-Jan-2019.)
|
⊢ ((Fun 𝐹 ∧ 𝐴 ∈ dom 𝐹) → (𝐹‘𝐴) = ∪ {𝑦 ∣ 𝐴𝐹𝑦}) |
|
Theorem | funfvdm2f 5551 |
The value of a function. Version of funfvdm2 5550 using a bound-variable
hypotheses instead of distinct variable conditions. (Contributed by Jim
Kingdon, 1-Jan-2019.)
|
⊢ Ⅎ𝑦𝐴
& ⊢ Ⅎ𝑦𝐹 ⇒ ⊢ ((Fun 𝐹 ∧ 𝐴 ∈ dom 𝐹) → (𝐹‘𝐴) = ∪ {𝑦 ∣ 𝐴𝐹𝑦}) |
|
Theorem | fvun1 5552 |
The value of a union when the argument is in the first domain.
(Contributed by Scott Fenton, 29-Jun-2013.)
|
⊢ ((𝐹 Fn 𝐴 ∧ 𝐺 Fn 𝐵 ∧ ((𝐴 ∩ 𝐵) = ∅ ∧ 𝑋 ∈ 𝐴)) → ((𝐹 ∪ 𝐺)‘𝑋) = (𝐹‘𝑋)) |
|
Theorem | fvun2 5553 |
The value of a union when the argument is in the second domain.
(Contributed by Scott Fenton, 29-Jun-2013.)
|
⊢ ((𝐹 Fn 𝐴 ∧ 𝐺 Fn 𝐵 ∧ ((𝐴 ∩ 𝐵) = ∅ ∧ 𝑋 ∈ 𝐵)) → ((𝐹 ∪ 𝐺)‘𝑋) = (𝐺‘𝑋)) |
|
Theorem | dmfco 5554 |
Domains of a function composition. (Contributed by NM, 27-Jan-1997.)
|
⊢ ((Fun 𝐺 ∧ 𝐴 ∈ dom 𝐺) → (𝐴 ∈ dom (𝐹 ∘ 𝐺) ↔ (𝐺‘𝐴) ∈ dom 𝐹)) |
|
Theorem | fvco2 5555 |
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 5556 |
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 5557 |
Value of a function composition. (Contributed by NM, 3-Jan-2004.)
(Revised by Mario Carneiro, 26-Dec-2014.)
|
⊢ ((𝐺:𝐴⟶𝐵 ∧ 𝐶 ∈ 𝐴) → ((𝐹 ∘ 𝐺)‘𝐶) = (𝐹‘(𝐺‘𝐶))) |
|
Theorem | fvco4 5558 |
Value of a composition. (Contributed by BJ, 7-Jul-2022.)
|
⊢ (((𝐾:𝐴⟶𝑋 ∧ (𝐻 ∘ 𝐾) = 𝐹) ∧ (𝑢 ∈ 𝐴 ∧ 𝑥 = (𝐾‘𝑢))) → (𝐻‘𝑥) = (𝐹‘𝑢)) |
|
Theorem | fvopab3g 5559* |
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 5560* |
Value of a function given by ordered-pair class abstraction.
(Contributed by NM, 23-Oct-1999.)
|
⊢ (𝑥 = 𝐴 → (𝜑 ↔ 𝜓)) & ⊢ (𝑦 = 𝐵 → (𝜓 ↔ 𝜒)) & ⊢ (𝑥 ∈ 𝐶 → ∃*𝑦𝜑)
& ⊢ 𝐹 = {〈𝑥, 𝑦〉 ∣ (𝑥 ∈ 𝐶 ∧ 𝜑)} ⇒ ⊢ ((𝐴 ∈ 𝐶 ∧ 𝐵 ∈ 𝐷) → (𝜒 → (𝐹‘𝐴) = 𝐵)) |
|
Theorem | fvmptss2 5561* |
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 5562* |
Value of a function given in maps-to notation. (Contributed by NM,
2-Oct-2007.) (Revised by Mario Carneiro, 31-Aug-2015.)
|
⊢ (𝑥 = 𝐴 → 𝐵 = 𝐶)
& ⊢ 𝐹 = (𝑥 ∈ 𝐷 ↦ 𝐵) ⇒ ⊢ ((𝐴 ∈ 𝐷 ∧ 𝐶 ∈ 𝑅) → (𝐹‘𝐴) = 𝐶) |
|
Theorem | fvmpt 5563* |
Value of a function given in maps-to notation. (Contributed by NM,
17-Aug-2011.)
|
⊢ (𝑥 = 𝐴 → 𝐵 = 𝐶)
& ⊢ 𝐹 = (𝑥 ∈ 𝐷 ↦ 𝐵)
& ⊢ 𝐶 ∈ V ⇒ ⊢ (𝐴 ∈ 𝐷 → (𝐹‘𝐴) = 𝐶) |
|
Theorem | fvmpts 5564* |
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 5565* |
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 5566* |
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 5567* |
Deduction version of fvmpt 5563. (Contributed by Scott Fenton,
18-Feb-2013.) (Revised by Mario Carneiro, 31-Aug-2015.)
|
⊢ (𝜑 → 𝐹 = (𝑥 ∈ 𝐷 ↦ 𝐵)) & ⊢ ((𝜑 ∧ 𝑥 = 𝐴) → 𝐵 = 𝐶)
& ⊢ (𝜑 → 𝐴 ∈ 𝐷)
& ⊢ (𝜑 → 𝐶 ∈ 𝑉) ⇒ ⊢ (𝜑 → (𝐹‘𝐴) = 𝐶) |
|
Theorem | mptrcl 5568* |
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 5569* |
Value of a function given by the maps-to notation. (Contributed by FL,
21-Jun-2010.)
|
⊢ 𝐹 = (𝑥 ∈ 𝐴 ↦ 𝐵) ⇒ ⊢ ((𝑥 ∈ 𝐴 ∧ 𝐵 ∈ 𝐶) → (𝐹‘𝑥) = 𝐵) |
|
Theorem | fvmptssdm 5570* |
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 5571* |
Sufficient condition for a maps-to notation to be set-like.
(Contributed by Mario Carneiro, 3-Jul-2019.)
|
⊢ 𝐹 = (𝑥 ∈ 𝐴 ↦ 𝐵) ⇒ ⊢ ((∀𝑥 𝐵 ∈ 𝑉 ∧ 𝐶 ∈ 𝑊) → (𝐹‘𝐶) ∈ V) |
|
Theorem | fvmpt2d 5572* |
Deduction version of fvmpt2 5569. (Contributed by Thierry Arnoux,
8-Dec-2016.)
|
⊢ (𝜑 → 𝐹 = (𝑥 ∈ 𝐴 ↦ 𝐵)) & ⊢ ((𝜑 ∧ 𝑥 ∈ 𝐴) → 𝐵 ∈ 𝑉) ⇒ ⊢ ((𝜑 ∧ 𝑥 ∈ 𝐴) → (𝐹‘𝑥) = 𝐵) |
|
Theorem | fvmptdf 5573* |
Alternate deduction version of fvmpt 5563, suitable for iteration.
(Contributed by Mario Carneiro, 7-Jan-2017.)
|
⊢ (𝜑 → 𝐴 ∈ 𝐷)
& ⊢ ((𝜑 ∧ 𝑥 = 𝐴) → 𝐵 ∈ 𝑉)
& ⊢ ((𝜑 ∧ 𝑥 = 𝐴) → ((𝐹‘𝐴) = 𝐵 → 𝜓)) & ⊢
Ⅎ𝑥𝐹
& ⊢ Ⅎ𝑥𝜓 ⇒ ⊢ (𝜑 → (𝐹 = (𝑥 ∈ 𝐷 ↦ 𝐵) → 𝜓)) |
|
Theorem | fvmptdv 5574* |
Alternate deduction version of fvmpt 5563, suitable for iteration.
(Contributed by Mario Carneiro, 7-Jan-2017.)
|
⊢ (𝜑 → 𝐴 ∈ 𝐷)
& ⊢ ((𝜑 ∧ 𝑥 = 𝐴) → 𝐵 ∈ 𝑉)
& ⊢ ((𝜑 ∧ 𝑥 = 𝐴) → ((𝐹‘𝐴) = 𝐵 → 𝜓)) ⇒ ⊢ (𝜑 → (𝐹 = (𝑥 ∈ 𝐷 ↦ 𝐵) → 𝜓)) |
|
Theorem | fvmptdv2 5575* |
Alternate deduction version of fvmpt 5563, suitable for iteration.
(Contributed by Mario Carneiro, 7-Jan-2017.)
|
⊢ (𝜑 → 𝐴 ∈ 𝐷)
& ⊢ ((𝜑 ∧ 𝑥 = 𝐴) → 𝐵 ∈ 𝑉)
& ⊢ ((𝜑 ∧ 𝑥 = 𝐴) → 𝐵 = 𝐶) ⇒ ⊢ (𝜑 → (𝐹 = (𝑥 ∈ 𝐷 ↦ 𝐵) → (𝐹‘𝐴) = 𝐶)) |
|
Theorem | mpteqb 5576* |
Bidirectional equality theorem for a mapping abstraction. Equivalent to
eqfnfv 5583. (Contributed by Mario Carneiro,
14-Nov-2014.)
|
⊢ (∀𝑥 ∈ 𝐴 𝐵 ∈ 𝑉 → ((𝑥 ∈ 𝐴 ↦ 𝐵) = (𝑥 ∈ 𝐴 ↦ 𝐶) ↔ ∀𝑥 ∈ 𝐴 𝐵 = 𝐶)) |
|
Theorem | fvmptt 5577* |
Closed theorem form of fvmpt 5563. (Contributed by Scott Fenton,
21-Feb-2013.) (Revised by Mario Carneiro, 11-Sep-2015.)
|
⊢ ((∀𝑥(𝑥 = 𝐴 → 𝐵 = 𝐶) ∧ 𝐹 = (𝑥 ∈ 𝐷 ↦ 𝐵) ∧ (𝐴 ∈ 𝐷 ∧ 𝐶 ∈ 𝑉)) → (𝐹‘𝐴) = 𝐶) |
|
Theorem | fvmptf 5578* |
Value of a function given by an ordered-pair class abstraction. This
version of fvmptg 5562 uses bound-variable hypotheses instead of
distinct
variable conditions. (Contributed by NM, 8-Nov-2005.) (Revised by
Mario Carneiro, 15-Oct-2016.)
|
⊢ Ⅎ𝑥𝐴
& ⊢ Ⅎ𝑥𝐶
& ⊢ (𝑥 = 𝐴 → 𝐵 = 𝐶)
& ⊢ 𝐹 = (𝑥 ∈ 𝐷 ↦ 𝐵) ⇒ ⊢ ((𝐴 ∈ 𝐷 ∧ 𝐶 ∈ 𝑉) → (𝐹‘𝐴) = 𝐶) |
|
Theorem | fvmptd3 5579* |
Deduction version of fvmpt 5563. (Contributed by Glauco Siliprandi,
23-Oct-2021.)
|
⊢ 𝐹 = (𝑥 ∈ 𝐷 ↦ 𝐵)
& ⊢ (𝑥 = 𝐴 → 𝐵 = 𝐶)
& ⊢ (𝜑 → 𝐴 ∈ 𝐷)
& ⊢ (𝜑 → 𝐶 ∈ 𝑉) ⇒ ⊢ (𝜑 → (𝐹‘𝐴) = 𝐶) |
|
Theorem | elfvmptrab1 5580* |
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 5581* |
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 5582* |
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 5583* |
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 5584* |
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 5585* |
Derive equality of functions from equality of their values.
(Contributed by Jeff Madsen, 2-Sep-2009.)
|
⊢ ((𝐹 Fn 𝐴 ∧ 𝐺 Fn 𝐵) → (𝐹 = 𝐺 ↔ (𝐵 ⊆ 𝐴 ∧ ∀𝑥 ∈ 𝐴 (𝑥 ∈ 𝐵 ∧ (𝐹‘𝑥) = (𝐺‘𝑥))))) |
|
Theorem | eqfnfvd 5586* |
Deduction for equality of functions. (Contributed by Mario Carneiro,
24-Jul-2014.)
|
⊢ (𝜑 → 𝐹 Fn 𝐴)
& ⊢ (𝜑 → 𝐺 Fn 𝐴)
& ⊢ ((𝜑 ∧ 𝑥 ∈ 𝐴) → (𝐹‘𝑥) = (𝐺‘𝑥)) ⇒ ⊢ (𝜑 → 𝐹 = 𝐺) |
|
Theorem | eqfnfv2f 5587* |
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 5583 uses bound-variable hypotheses instead of
distinct variable conditions. (Contributed by NM, 29-Jan-2004.)
|
⊢ Ⅎ𝑥𝐹
& ⊢ Ⅎ𝑥𝐺 ⇒ ⊢ ((𝐹 Fn 𝐴 ∧ 𝐺 Fn 𝐴) → (𝐹 = 𝐺 ↔ ∀𝑥 ∈ 𝐴 (𝐹‘𝑥) = (𝐺‘𝑥))) |
|
Theorem | eqfunfv 5588* |
Equality of functions is determined by their values. (Contributed by
Scott Fenton, 19-Jun-2011.)
|
⊢ ((Fun 𝐹 ∧ Fun 𝐺) → (𝐹 = 𝐺 ↔ (dom 𝐹 = dom 𝐺 ∧ ∀𝑥 ∈ dom 𝐹(𝐹‘𝑥) = (𝐺‘𝑥)))) |
|
Theorem | fvreseq 5589* |
Equality of restricted functions is determined by their values.
(Contributed by NM, 3-Aug-1994.)
|
⊢ (((𝐹 Fn 𝐴 ∧ 𝐺 Fn 𝐴) ∧ 𝐵 ⊆ 𝐴) → ((𝐹 ↾ 𝐵) = (𝐺 ↾ 𝐵) ↔ ∀𝑥 ∈ 𝐵 (𝐹‘𝑥) = (𝐺‘𝑥))) |
|
Theorem | fndmdif 5590* |
Two ways to express the locus of differences between two functions.
(Contributed by Stefan O'Rear, 17-Jan-2015.)
|
⊢ ((𝐹 Fn 𝐴 ∧ 𝐺 Fn 𝐴) → dom (𝐹 ∖ 𝐺) = {𝑥 ∈ 𝐴 ∣ (𝐹‘𝑥) ≠ (𝐺‘𝑥)}) |
|
Theorem | fndmdifcom 5591 |
The difference set between two functions is commutative. (Contributed
by Stefan O'Rear, 17-Jan-2015.)
|
⊢ ((𝐹 Fn 𝐴 ∧ 𝐺 Fn 𝐴) → dom (𝐹 ∖ 𝐺) = dom (𝐺 ∖ 𝐹)) |
|
Theorem | fndmin 5592* |
Two ways to express the locus of equality between two functions.
(Contributed by Stefan O'Rear, 17-Jan-2015.)
|
⊢ ((𝐹 Fn 𝐴 ∧ 𝐺 Fn 𝐴) → dom (𝐹 ∩ 𝐺) = {𝑥 ∈ 𝐴 ∣ (𝐹‘𝑥) = (𝐺‘𝑥)}) |
|
Theorem | fneqeql 5593 |
Two functions are equal iff their equalizer is the whole domain.
(Contributed by Stefan O'Rear, 7-Mar-2015.)
|
⊢ ((𝐹 Fn 𝐴 ∧ 𝐺 Fn 𝐴) → (𝐹 = 𝐺 ↔ dom (𝐹 ∩ 𝐺) = 𝐴)) |
|
Theorem | fneqeql2 5594 |
Two functions are equal iff their equalizer contains the whole domain.
(Contributed by Stefan O'Rear, 9-Mar-2015.)
|
⊢ ((𝐹 Fn 𝐴 ∧ 𝐺 Fn 𝐴) → (𝐹 = 𝐺 ↔ 𝐴 ⊆ dom (𝐹 ∩ 𝐺))) |
|
Theorem | fnreseql 5595 |
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 5596* |
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 5597 |
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 5598 |
Two ways to say that 𝐴 is in the domain of 𝐹.
(Contributed by
Mario Carneiro, 1-May-2014.)
|
⊢ (Fun 𝐹 → (𝐴 ∈ dom 𝐹 ↔ 𝐴𝐹(𝐹‘𝐴))) |
|
Theorem | fvimacnvi 5599 |
A member of a preimage is a function value argument. (Contributed by NM,
4-May-2007.)
|
⊢ ((Fun 𝐹 ∧ 𝐴 ∈ (◡𝐹 “ 𝐵)) → (𝐹‘𝐴) ∈ 𝐵) |
|
Theorem | fvimacnv 5600 |
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 5266 could probably be
strengthened to a biconditional." (Contributed by Raph Levien,
20-Nov-2006.)
|
⊢ ((Fun 𝐹 ∧ 𝐴 ∈ dom 𝐹) → ((𝐹‘𝐴) ∈ 𝐵 ↔ 𝐴 ∈ (◡𝐹 “ 𝐵))) |