HomeHome Intuitionistic Logic Explorer
Theorem List (p. 57 of 133)
< Previous  Next >
Bad symbols? Try the
GIF version.

Mirrors  >  Metamath Home Page  >  ILE Home Page  >  Theorem List Contents  >  Recent Proofs       This page: Page List

Theorem List for Intuitionistic Logic Explorer - 5601-5700   *Has distinct variable group(s)
TypeLabelDescription
Statement
 
Theoremressnop0 5601 If 𝐴 is not in 𝐶, then the restriction of a singleton of 𝐴, 𝐵 to 𝐶 is null. (Contributed by Scott Fenton, 15-Apr-2011.)
𝐴𝐶 → ({⟨𝐴, 𝐵⟩} ↾ 𝐶) = ∅)
 
Theoremfpr 5602 A function with a domain of two elements. (Contributed by Jeff Madsen, 20-Jun-2010.) (Proof shortened by Andrew Salmon, 22-Oct-2011.)
𝐴 ∈ V    &   𝐵 ∈ V    &   𝐶 ∈ V    &   𝐷 ∈ V       (𝐴𝐵 → {⟨𝐴, 𝐶⟩, ⟨𝐵, 𝐷⟩}:{𝐴, 𝐵}⟶{𝐶, 𝐷})
 
Theoremfprg 5603 A function with a domain of two elements. (Contributed by FL, 2-Feb-2014.)
(((𝐴𝐸𝐵𝐹) ∧ (𝐶𝐺𝐷𝐻) ∧ 𝐴𝐵) → {⟨𝐴, 𝐶⟩, ⟨𝐵, 𝐷⟩}:{𝐴, 𝐵}⟶{𝐶, 𝐷})
 
Theoremftpg 5604 A function with a domain of three elements. (Contributed by Alexander van der Vekens, 4-Dec-2017.)
(((𝑋𝑈𝑌𝑉𝑍𝑊) ∧ (𝐴𝐹𝐵𝐺𝐶𝐻) ∧ (𝑋𝑌𝑋𝑍𝑌𝑍)) → {⟨𝑋, 𝐴⟩, ⟨𝑌, 𝐵⟩, ⟨𝑍, 𝐶⟩}:{𝑋, 𝑌, 𝑍}⟶{𝐴, 𝐵, 𝐶})
 
Theoremftp 5605 A function with a domain of three elements. (Contributed by Stefan O'Rear, 17-Oct-2014.) (Proof shortened by Alexander van der Vekens, 23-Jan-2018.)
𝐴 ∈ V    &   𝐵 ∈ V    &   𝐶 ∈ V    &   𝑋 ∈ V    &   𝑌 ∈ V    &   𝑍 ∈ V    &   𝐴𝐵    &   𝐴𝐶    &   𝐵𝐶       {⟨𝐴, 𝑋⟩, ⟨𝐵, 𝑌⟩, ⟨𝐶, 𝑍⟩}:{𝐴, 𝐵, 𝐶}⟶{𝑋, 𝑌, 𝑍}
 
Theoremfnressn 5606 A function restricted to a singleton. (Contributed by NM, 9-Oct-2004.)
((𝐹 Fn 𝐴𝐵𝐴) → (𝐹 ↾ {𝐵}) = {⟨𝐵, (𝐹𝐵)⟩})
 
Theoremfressnfv 5607 The value of a function restricted to a singleton. (Contributed by NM, 9-Oct-2004.)
((𝐹 Fn 𝐴𝐵𝐴) → ((𝐹 ↾ {𝐵}):{𝐵}⟶𝐶 ↔ (𝐹𝐵) ∈ 𝐶))
 
Theoremfvconst 5608 The value of a constant function. (Contributed by NM, 30-May-1999.)
((𝐹:𝐴⟶{𝐵} ∧ 𝐶𝐴) → (𝐹𝐶) = 𝐵)
 
Theoremfmptsn 5609* Express a singleton function in maps-to notation. (Contributed by NM, 6-Jun-2006.) (Proof shortened by Andrew Salmon, 22-Oct-2011.) (Revised by Stefan O'Rear, 28-Feb-2015.)
((𝐴𝑉𝐵𝑊) → {⟨𝐴, 𝐵⟩} = (𝑥 ∈ {𝐴} ↦ 𝐵))
 
Theoremfmptap 5610* Append an additional value to a function. (Contributed by NM, 6-Jun-2006.) (Revised by Mario Carneiro, 31-Aug-2015.)
𝐴 ∈ V    &   𝐵 ∈ V    &   (𝑅 ∪ {𝐴}) = 𝑆    &   (𝑥 = 𝐴𝐶 = 𝐵)       ((𝑥𝑅𝐶) ∪ {⟨𝐴, 𝐵⟩}) = (𝑥𝑆𝐶)
 
Theoremfmptapd 5611* Append an additional value to a function. (Contributed by Thierry Arnoux, 3-Jan-2017.)
(𝜑𝐴 ∈ V)    &   (𝜑𝐵 ∈ V)    &   (𝜑 → (𝑅 ∪ {𝐴}) = 𝑆)    &   ((𝜑𝑥 = 𝐴) → 𝐶 = 𝐵)       (𝜑 → ((𝑥𝑅𝐶) ∪ {⟨𝐴, 𝐵⟩}) = (𝑥𝑆𝐶))
 
Theoremfmptpr 5612* Express a pair function in maps-to notation. (Contributed by Thierry Arnoux, 3-Jan-2017.)
(𝜑𝐴𝑉)    &   (𝜑𝐵𝑊)    &   (𝜑𝐶𝑋)    &   (𝜑𝐷𝑌)    &   ((𝜑𝑥 = 𝐴) → 𝐸 = 𝐶)    &   ((𝜑𝑥 = 𝐵) → 𝐸 = 𝐷)       (𝜑 → {⟨𝐴, 𝐶⟩, ⟨𝐵, 𝐷⟩} = (𝑥 ∈ {𝐴, 𝐵} ↦ 𝐸))
 
Theoremfvresi 5613 The value of a restricted identity function. (Contributed by NM, 19-May-2004.)
(𝐵𝐴 → (( I ↾ 𝐴)‘𝐵) = 𝐵)
 
Theoremfvunsng 5614 Remove an ordered pair not participating in a function value. (Contributed by Jim Kingdon, 7-Jan-2019.)
((𝐷𝑉𝐵𝐷) → ((𝐴 ∪ {⟨𝐵, 𝐶⟩})‘𝐷) = (𝐴𝐷))
 
Theoremfvsn 5615 The value of a singleton of an ordered pair is the second member. (Contributed by NM, 12-Aug-1994.)
𝐴 ∈ V    &   𝐵 ∈ V       ({⟨𝐴, 𝐵⟩}‘𝐴) = 𝐵
 
Theoremfvsng 5616 The value of a singleton of an ordered pair is the second member. (Contributed by NM, 26-Oct-2012.)
((𝐴𝑉𝐵𝑊) → ({⟨𝐴, 𝐵⟩}‘𝐴) = 𝐵)
 
Theoremfvsnun1 5617 The value of a function with one of its ordered pairs replaced, at the replaced ordered pair. See also fvsnun2 5618. (Contributed by NM, 23-Sep-2007.)
𝐴 ∈ V    &   𝐵 ∈ V    &   𝐺 = ({⟨𝐴, 𝐵⟩} ∪ (𝐹 ↾ (𝐶 ∖ {𝐴})))       (𝐺𝐴) = 𝐵
 
Theoremfvsnun2 5618 The value of a function with one of its ordered pairs replaced, at arguments other than the replaced one. See also fvsnun1 5617. (Contributed by NM, 23-Sep-2007.)
𝐴 ∈ V    &   𝐵 ∈ V    &   𝐺 = ({⟨𝐴, 𝐵⟩} ∪ (𝐹 ↾ (𝐶 ∖ {𝐴})))       (𝐷 ∈ (𝐶 ∖ {𝐴}) → (𝐺𝐷) = (𝐹𝐷))
 
Theoremfnsnsplitss 5619 Split a function into a single point and all the rest. (Contributed by Stefan O'Rear, 27-Feb-2015.) (Revised by Jim Kingdon, 20-Jan-2023.)
((𝐹 Fn 𝐴𝑋𝐴) → ((𝐹 ↾ (𝐴 ∖ {𝑋})) ∪ {⟨𝑋, (𝐹𝑋)⟩}) ⊆ 𝐹)
 
Theoremfsnunf 5620 Adjoining a point to a function gives a function. (Contributed by Stefan O'Rear, 28-Feb-2015.)
((𝐹:𝑆𝑇 ∧ (𝑋𝑉 ∧ ¬ 𝑋𝑆) ∧ 𝑌𝑇) → (𝐹 ∪ {⟨𝑋, 𝑌⟩}):(𝑆 ∪ {𝑋})⟶𝑇)
 
Theoremfsnunfv 5621 Recover the added point from a point-added function. (Contributed by Stefan O'Rear, 28-Feb-2015.) (Revised by NM, 18-May-2017.)
((𝑋𝑉𝑌𝑊 ∧ ¬ 𝑋 ∈ dom 𝐹) → ((𝐹 ∪ {⟨𝑋, 𝑌⟩})‘𝑋) = 𝑌)
 
Theoremfsnunres 5622 Recover the original function from a point-added function. (Contributed by Stefan O'Rear, 28-Feb-2015.)
((𝐹 Fn 𝑆 ∧ ¬ 𝑋𝑆) → ((𝐹 ∪ {⟨𝑋, 𝑌⟩}) ↾ 𝑆) = 𝐹)
 
Theoremfunresdfunsnss 5623 Restricting a function to a domain without one element of the domain of the function, and adding a pair of this element and the function value of the element results in a subset of the function itself. (Contributed by AV, 2-Dec-2018.) (Revised by Jim Kingdon, 21-Jan-2023.)
((Fun 𝐹𝑋 ∈ dom 𝐹) → ((𝐹 ↾ (V ∖ {𝑋})) ∪ {⟨𝑋, (𝐹𝑋)⟩}) ⊆ 𝐹)
 
Theoremfvpr1 5624 The value of a function with a domain of two elements. (Contributed by Jeff Madsen, 20-Jun-2010.)
𝐴 ∈ V    &   𝐶 ∈ V       (𝐴𝐵 → ({⟨𝐴, 𝐶⟩, ⟨𝐵, 𝐷⟩}‘𝐴) = 𝐶)
 
Theoremfvpr2 5625 The value of a function with a domain of two elements. (Contributed by Jeff Madsen, 20-Jun-2010.)
𝐵 ∈ V    &   𝐷 ∈ V       (𝐴𝐵 → ({⟨𝐴, 𝐶⟩, ⟨𝐵, 𝐷⟩}‘𝐵) = 𝐷)
 
Theoremfvpr1g 5626 The value of a function with a domain of (at most) two elements. (Contributed by Alexander van der Vekens, 3-Dec-2017.)
((𝐴𝑉𝐶𝑊𝐴𝐵) → ({⟨𝐴, 𝐶⟩, ⟨𝐵, 𝐷⟩}‘𝐴) = 𝐶)
 
Theoremfvpr2g 5627 The value of a function with a domain of (at most) two elements. (Contributed by Alexander van der Vekens, 3-Dec-2017.)
((𝐵𝑉𝐷𝑊𝐴𝐵) → ({⟨𝐴, 𝐶⟩, ⟨𝐵, 𝐷⟩}‘𝐵) = 𝐷)
 
Theoremfvtp1g 5628 The value of a function with a domain of (at most) three elements. (Contributed by Alexander van der Vekens, 4-Dec-2017.)
(((𝐴𝑉𝐷𝑊) ∧ (𝐴𝐵𝐴𝐶)) → ({⟨𝐴, 𝐷⟩, ⟨𝐵, 𝐸⟩, ⟨𝐶, 𝐹⟩}‘𝐴) = 𝐷)
 
Theoremfvtp2g 5629 The value of a function with a domain of (at most) three elements. (Contributed by Alexander van der Vekens, 4-Dec-2017.)
(((𝐵𝑉𝐸𝑊) ∧ (𝐴𝐵𝐵𝐶)) → ({⟨𝐴, 𝐷⟩, ⟨𝐵, 𝐸⟩, ⟨𝐶, 𝐹⟩}‘𝐵) = 𝐸)
 
Theoremfvtp3g 5630 The value of a function with a domain of (at most) three elements. (Contributed by Alexander van der Vekens, 4-Dec-2017.)
(((𝐶𝑉𝐹𝑊) ∧ (𝐴𝐶𝐵𝐶)) → ({⟨𝐴, 𝐷⟩, ⟨𝐵, 𝐸⟩, ⟨𝐶, 𝐹⟩}‘𝐶) = 𝐹)
 
Theoremfvtp1 5631 The first value of a function with a domain of three elements. (Contributed by NM, 14-Sep-2011.)
𝐴 ∈ V    &   𝐷 ∈ V       ((𝐴𝐵𝐴𝐶) → ({⟨𝐴, 𝐷⟩, ⟨𝐵, 𝐸⟩, ⟨𝐶, 𝐹⟩}‘𝐴) = 𝐷)
 
Theoremfvtp2 5632 The second value of a function with a domain of three elements. (Contributed by NM, 14-Sep-2011.)
𝐵 ∈ V    &   𝐸 ∈ V       ((𝐴𝐵𝐵𝐶) → ({⟨𝐴, 𝐷⟩, ⟨𝐵, 𝐸⟩, ⟨𝐶, 𝐹⟩}‘𝐵) = 𝐸)
 
Theoremfvtp3 5633 The third value of a function with a domain of three elements. (Contributed by NM, 14-Sep-2011.)
𝐶 ∈ V    &   𝐹 ∈ V       ((𝐴𝐶𝐵𝐶) → ({⟨𝐴, 𝐷⟩, ⟨𝐵, 𝐸⟩, ⟨𝐶, 𝐹⟩}‘𝐶) = 𝐹)
 
Theoremfvconst2g 5634 The value of a constant function. (Contributed by NM, 20-Aug-2005.)
((𝐵𝐷𝐶𝐴) → ((𝐴 × {𝐵})‘𝐶) = 𝐵)
 
Theoremfconst2g 5635 A constant function expressed as a cross product. (Contributed by NM, 27-Nov-2007.)
(𝐵𝐶 → (𝐹:𝐴⟶{𝐵} ↔ 𝐹 = (𝐴 × {𝐵})))
 
Theoremfvconst2 5636 The value of a constant function. (Contributed by NM, 16-Apr-2005.)
𝐵 ∈ V       (𝐶𝐴 → ((𝐴 × {𝐵})‘𝐶) = 𝐵)
 
Theoremfconst2 5637 A constant function expressed as a cross product. (Contributed by NM, 20-Aug-1999.)
𝐵 ∈ V       (𝐹:𝐴⟶{𝐵} ↔ 𝐹 = (𝐴 × {𝐵}))
 
Theoremfconstfvm 5638* A constant function expressed in terms of its functionality, domain, and value. See also fconst2 5637. (Contributed by Jim Kingdon, 8-Jan-2019.)
(∃𝑦 𝑦𝐴 → (𝐹:𝐴⟶{𝐵} ↔ (𝐹 Fn 𝐴 ∧ ∀𝑥𝐴 (𝐹𝑥) = 𝐵)))
 
Theoremfconst3m 5639* Two ways to express a constant function. (Contributed by Jim Kingdon, 8-Jan-2019.)
(∃𝑥 𝑥𝐴 → (𝐹:𝐴⟶{𝐵} ↔ (𝐹 Fn 𝐴𝐴 ⊆ (𝐹 “ {𝐵}))))
 
Theoremfconst4m 5640* Two ways to express a constant function. (Contributed by NM, 8-Mar-2007.)
(∃𝑥 𝑥𝐴 → (𝐹:𝐴⟶{𝐵} ↔ (𝐹 Fn 𝐴 ∧ (𝐹 “ {𝐵}) = 𝐴)))
 
Theoremresfunexg 5641 The restriction of a function to a set exists. Compare Proposition 6.17 of [TakeutiZaring] p. 28. (Contributed by NM, 7-Apr-1995.) (Revised by Mario Carneiro, 22-Jun-2013.)
((Fun 𝐴𝐵𝐶) → (𝐴𝐵) ∈ V)
 
Theoremfnex 5642 If the domain of a function is a set, the function is a set. Theorem 6.16(1) of [TakeutiZaring] p. 28. This theorem is derived using the Axiom of Replacement in the form of resfunexg 5641. (Contributed by NM, 14-Aug-1994.) (Proof shortened by Andrew Salmon, 17-Sep-2011.)
((𝐹 Fn 𝐴𝐴𝐵) → 𝐹 ∈ V)
 
Theoremfunex 5643 If the domain of a function exists, so does the function. Part of Theorem 4.15(v) of [Monk1] p. 46. This theorem is derived using the Axiom of Replacement in the form of fnex 5642. (Note: Any resemblance between F.U.N.E.X. and "Have You Any Eggs" is purely a coincidence originated by Swedish chefs.) (Contributed by NM, 11-Nov-1995.)
((Fun 𝐹 ∧ dom 𝐹𝐵) → 𝐹 ∈ V)
 
Theoremopabex 5644* Existence of a function expressed as class of ordered pairs. (Contributed by NM, 21-Jul-1996.)
𝐴 ∈ V    &   (𝑥𝐴 → ∃*𝑦𝜑)       {⟨𝑥, 𝑦⟩ ∣ (𝑥𝐴𝜑)} ∈ V
 
Theoremmptexg 5645* If the domain of a function given by maps-to notation is a set, the function is a set. (Contributed by FL, 6-Jun-2011.) (Revised by Mario Carneiro, 31-Aug-2015.)
(𝐴𝑉 → (𝑥𝐴𝐵) ∈ V)
 
Theoremmptex 5646* If the domain of a function given by maps-to notation is a set, the function is a set. (Contributed by NM, 22-Apr-2005.) (Revised by Mario Carneiro, 20-Dec-2013.)
𝐴 ∈ V       (𝑥𝐴𝐵) ∈ V
 
Theoremfex 5647 If the domain of a mapping is a set, the function is a set. (Contributed by NM, 3-Oct-1999.)
((𝐹:𝐴𝐵𝐴𝐶) → 𝐹 ∈ V)
 
Theoremeufnfv 5648* A function is uniquely determined by its values. (Contributed by NM, 31-Aug-2011.)
𝐴 ∈ V    &   𝐵 ∈ V       ∃!𝑓(𝑓 Fn 𝐴 ∧ ∀𝑥𝐴 (𝑓𝑥) = 𝐵)
 
Theoremfunfvima 5649 A function's value in a preimage belongs to the image. (Contributed by NM, 23-Sep-2003.)
((Fun 𝐹𝐵 ∈ dom 𝐹) → (𝐵𝐴 → (𝐹𝐵) ∈ (𝐹𝐴)))
 
Theoremfunfvima2 5650 A function's value in an included preimage belongs to the image. (Contributed by NM, 3-Feb-1997.)
((Fun 𝐹𝐴 ⊆ dom 𝐹) → (𝐵𝐴 → (𝐹𝐵) ∈ (𝐹𝐴)))
 
Theoremfunfvima3 5651 A class including a function contains the function's value in the image of the singleton of the argument. (Contributed by NM, 23-Mar-2004.)
((Fun 𝐹𝐹𝐺) → (𝐴 ∈ dom 𝐹 → (𝐹𝐴) ∈ (𝐺 “ {𝐴})))
 
Theoremfnfvima 5652 The function value of an operand in a set is contained in the image of that set, using the Fn abbreviation. (Contributed by Stefan O'Rear, 10-Mar-2015.)
((𝐹 Fn 𝐴𝑆𝐴𝑋𝑆) → (𝐹𝑋) ∈ (𝐹𝑆))
 
Theoremfoima2 5653* Given an onto function, an element is in its codomain if and only if it is the image of an element of its domain (see foima 5350). (Contributed by BJ, 6-Jul-2022.)
(𝐹:𝐴onto𝐵 → (𝑌𝐵 ↔ ∃𝑥𝐴 𝑌 = (𝐹𝑥)))
 
Theoremfoelrn 5654* Property of a surjective function. (Contributed by Jeff Madsen, 4-Jan-2011.) (Proof shortened by BJ, 6-Jul-2022.)
((𝐹:𝐴onto𝐵𝐶𝐵) → ∃𝑥𝐴 𝐶 = (𝐹𝑥))
 
Theoremfoco2 5655 If a composition of two functions is surjective, then the function on the left is surjective. (Contributed by Jeff Madsen, 16-Jun-2011.)
((𝐹:𝐵𝐶𝐺:𝐴𝐵 ∧ (𝐹𝐺):𝐴onto𝐶) → 𝐹:𝐵onto𝐶)
 
Theoremrexima 5656* Existential quantification under an image in terms of the base set. (Contributed by Stefan O'Rear, 21-Jan-2015.)
(𝑥 = (𝐹𝑦) → (𝜑𝜓))       ((𝐹 Fn 𝐴𝐵𝐴) → (∃𝑥 ∈ (𝐹𝐵)𝜑 ↔ ∃𝑦𝐵 𝜓))
 
Theoremralima 5657* Universal quantification under an image in terms of the base set. (Contributed by Stefan O'Rear, 21-Jan-2015.)
(𝑥 = (𝐹𝑦) → (𝜑𝜓))       ((𝐹 Fn 𝐴𝐵𝐴) → (∀𝑥 ∈ (𝐹𝐵)𝜑 ↔ ∀𝑦𝐵 𝜓))
 
Theoremidref 5658* TODO: This is the same as issref 4921 (which has a much longer proof). Should we replace issref 4921 with this one? - NM 9-May-2016.

Two ways to state a relation is reflexive. (Adapted from Tarski.) (Contributed by FL, 15-Jan-2012.) (Proof shortened by Mario Carneiro, 3-Nov-2015.) (Proof modification is discouraged.)

(( I ↾ 𝐴) ⊆ 𝑅 ↔ ∀𝑥𝐴 𝑥𝑅𝑥)
 
Theoremelabrex 5659* Elementhood in an image set. (Contributed by Mario Carneiro, 14-Jan-2014.)
𝐵 ∈ V       (𝑥𝐴𝐵 ∈ {𝑦 ∣ ∃𝑥𝐴 𝑦 = 𝐵})
 
Theoremabrexco 5660* Composition of two image maps 𝐶(𝑦) and 𝐵(𝑤). (Contributed by NM, 27-May-2013.)
𝐵 ∈ V    &   (𝑦 = 𝐵𝐶 = 𝐷)       {𝑥 ∣ ∃𝑦 ∈ {𝑧 ∣ ∃𝑤𝐴 𝑧 = 𝐵}𝑥 = 𝐶} = {𝑥 ∣ ∃𝑤𝐴 𝑥 = 𝐷}
 
Theoremimaiun 5661* The image of an indexed union is the indexed union of the images. (Contributed by Mario Carneiro, 18-Jun-2014.)
(𝐴 𝑥𝐵 𝐶) = 𝑥𝐵 (𝐴𝐶)
 
Theoremimauni 5662* The image of a union is the indexed union of the images. Theorem 3K(a) of [Enderton] p. 50. (Contributed by NM, 9-Aug-2004.) (Proof shortened by Mario Carneiro, 18-Jun-2014.)
(𝐴 𝐵) = 𝑥𝐵 (𝐴𝑥)
 
Theoremfniunfv 5663* The indexed union of a function's values is the union of its range. Compare Definition 5.4 of [Monk1] p. 50. (Contributed by NM, 27-Sep-2004.)
(𝐹 Fn 𝐴 𝑥𝐴 (𝐹𝑥) = ran 𝐹)
 
Theoremfuniunfvdm 5664* The indexed union of a function's values is the union of its image under the index class. This theorem is a slight variation of fniunfv 5663. (Contributed by Jim Kingdon, 10-Jan-2019.)
(𝐹 Fn 𝐴 𝑥𝐴 (𝐹𝑥) = (𝐹𝐴))
 
Theoremfuniunfvdmf 5665* The indexed union of a function's values is the union of its image under the index class. This version of funiunfvdm 5664 uses a bound-variable hypothesis in place of a distinct variable condition. (Contributed by Jim Kingdon, 10-Jan-2019.)
𝑥𝐹       (𝐹 Fn 𝐴 𝑥𝐴 (𝐹𝑥) = (𝐹𝐴))
 
Theoremeluniimadm 5666* Membership in the union of an image of a function. (Contributed by Jim Kingdon, 10-Jan-2019.)
(𝐹 Fn 𝐴 → (𝐵 (𝐹𝐴) ↔ ∃𝑥𝐴 𝐵 ∈ (𝐹𝑥)))
 
Theoremelunirn 5667* Membership in the union of the range of a function. (Contributed by NM, 24-Sep-2006.)
(Fun 𝐹 → (𝐴 ran 𝐹 ↔ ∃𝑥 ∈ dom 𝐹 𝐴 ∈ (𝐹𝑥)))
 
Theoremfnunirn 5668* Membership in a union of some function-defined family of sets. (Contributed by Stefan O'Rear, 30-Jan-2015.)
(𝐹 Fn 𝐼 → (𝐴 ran 𝐹 ↔ ∃𝑥𝐼 𝐴 ∈ (𝐹𝑥)))
 
Theoremdff13 5669* A one-to-one function in terms of function values. Compare Theorem 4.8(iv) of [Monk1] p. 43. (Contributed by NM, 29-Oct-1996.)
(𝐹:𝐴1-1𝐵 ↔ (𝐹:𝐴𝐵 ∧ ∀𝑥𝐴𝑦𝐴 ((𝐹𝑥) = (𝐹𝑦) → 𝑥 = 𝑦)))
 
Theoremf1veqaeq 5670 If the values of a one-to-one function for two arguments are equal, the arguments themselves must be equal. (Contributed by Alexander van der Vekens, 12-Nov-2017.)
((𝐹:𝐴1-1𝐵 ∧ (𝐶𝐴𝐷𝐴)) → ((𝐹𝐶) = (𝐹𝐷) → 𝐶 = 𝐷))
 
Theoremdff13f 5671* A one-to-one function in terms of function values. Compare Theorem 4.8(iv) of [Monk1] p. 43. (Contributed by NM, 31-Jul-2003.)
𝑥𝐹    &   𝑦𝐹       (𝐹:𝐴1-1𝐵 ↔ (𝐹:𝐴𝐵 ∧ ∀𝑥𝐴𝑦𝐴 ((𝐹𝑥) = (𝐹𝑦) → 𝑥 = 𝑦)))
 
Theoremf1mpt 5672* Express injection for a mapping operation. (Contributed by Mario Carneiro, 2-Jan-2017.)
𝐹 = (𝑥𝐴𝐶)    &   (𝑥 = 𝑦𝐶 = 𝐷)       (𝐹:𝐴1-1𝐵 ↔ (∀𝑥𝐴 𝐶𝐵 ∧ ∀𝑥𝐴𝑦𝐴 (𝐶 = 𝐷𝑥 = 𝑦)))
 
Theoremf1fveq 5673 Equality of function values for a one-to-one function. (Contributed by NM, 11-Feb-1997.)
((𝐹:𝐴1-1𝐵 ∧ (𝐶𝐴𝐷𝐴)) → ((𝐹𝐶) = (𝐹𝐷) ↔ 𝐶 = 𝐷))
 
Theoremf1elima 5674 Membership in the image of a 1-1 map. (Contributed by Jeff Madsen, 2-Sep-2009.)
((𝐹:𝐴1-1𝐵𝑋𝐴𝑌𝐴) → ((𝐹𝑋) ∈ (𝐹𝑌) ↔ 𝑋𝑌))
 
Theoremf1imass 5675 Taking images under a one-to-one function preserves subsets. (Contributed by Stefan O'Rear, 30-Oct-2014.)
((𝐹:𝐴1-1𝐵 ∧ (𝐶𝐴𝐷𝐴)) → ((𝐹𝐶) ⊆ (𝐹𝐷) ↔ 𝐶𝐷))
 
Theoremf1imaeq 5676 Taking images under a one-to-one function preserves equality. (Contributed by Stefan O'Rear, 30-Oct-2014.)
((𝐹:𝐴1-1𝐵 ∧ (𝐶𝐴𝐷𝐴)) → ((𝐹𝐶) = (𝐹𝐷) ↔ 𝐶 = 𝐷))
 
Theoremdff1o6 5677* A one-to-one onto function in terms of function values. (Contributed by NM, 29-Mar-2008.)
(𝐹:𝐴1-1-onto𝐵 ↔ (𝐹 Fn 𝐴 ∧ ran 𝐹 = 𝐵 ∧ ∀𝑥𝐴𝑦𝐴 ((𝐹𝑥) = (𝐹𝑦) → 𝑥 = 𝑦)))
 
Theoremf1ocnvfv1 5678 The converse value of the value of a one-to-one onto function. (Contributed by NM, 20-May-2004.)
((𝐹:𝐴1-1-onto𝐵𝐶𝐴) → (𝐹‘(𝐹𝐶)) = 𝐶)
 
Theoremf1ocnvfv2 5679 The value of the converse value of a one-to-one onto function. (Contributed by NM, 20-May-2004.)
((𝐹:𝐴1-1-onto𝐵𝐶𝐵) → (𝐹‘(𝐹𝐶)) = 𝐶)
 
Theoremf1ocnvfv 5680 Relationship between the value of a one-to-one onto function and the value of its converse. (Contributed by Raph Levien, 10-Apr-2004.)
((𝐹:𝐴1-1-onto𝐵𝐶𝐴) → ((𝐹𝐶) = 𝐷 → (𝐹𝐷) = 𝐶))
 
Theoremf1ocnvfvb 5681 Relationship between the value of a one-to-one onto function and the value of its converse. (Contributed by NM, 20-May-2004.)
((𝐹:𝐴1-1-onto𝐵𝐶𝐴𝐷𝐵) → ((𝐹𝐶) = 𝐷 ↔ (𝐹𝐷) = 𝐶))
 
Theoremf1ocnvdm 5682 The value of the converse of a one-to-one onto function belongs to its domain. (Contributed by NM, 26-May-2006.)
((𝐹:𝐴1-1-onto𝐵𝐶𝐵) → (𝐹𝐶) ∈ 𝐴)
 
Theoremf1ocnvfvrneq 5683 If the values of a one-to-one function for two arguments from the range of the function are equal, the arguments themselves must be equal. (Contributed by Alexander van der Vekens, 12-Nov-2017.)
((𝐹:𝐴1-1𝐵 ∧ (𝐶 ∈ ran 𝐹𝐷 ∈ ran 𝐹)) → ((𝐹𝐶) = (𝐹𝐷) → 𝐶 = 𝐷))
 
Theoremfcof1 5684 An application is injective if a retraction exists. Proposition 8 of [BourbakiEns] p. E.II.18. (Contributed by FL, 11-Nov-2011.) (Revised by Mario Carneiro, 27-Dec-2014.)
((𝐹:𝐴𝐵 ∧ (𝑅𝐹) = ( I ↾ 𝐴)) → 𝐹:𝐴1-1𝐵)
 
Theoremfcofo 5685 An application is surjective if a section exists. Proposition 8 of [BourbakiEns] p. E.II.18. (Contributed by FL, 17-Nov-2011.) (Proof shortened by Mario Carneiro, 27-Dec-2014.)
((𝐹:𝐴𝐵𝑆:𝐵𝐴 ∧ (𝐹𝑆) = ( I ↾ 𝐵)) → 𝐹:𝐴onto𝐵)
 
Theoremcbvfo 5686* Change bound variable between domain and range of function. (Contributed by NM, 23-Feb-1997.) (Proof shortened by Mario Carneiro, 21-Mar-2015.)
((𝐹𝑥) = 𝑦 → (𝜑𝜓))       (𝐹:𝐴onto𝐵 → (∀𝑥𝐴 𝜑 ↔ ∀𝑦𝐵 𝜓))
 
Theoremcbvexfo 5687* Change bound variable between domain and range of function. (Contributed by NM, 23-Feb-1997.)
((𝐹𝑥) = 𝑦 → (𝜑𝜓))       (𝐹:𝐴onto𝐵 → (∃𝑥𝐴 𝜑 ↔ ∃𝑦𝐵 𝜓))
 
Theoremcocan1 5688 An injection is left-cancelable. (Contributed by FL, 2-Aug-2009.) (Revised by Mario Carneiro, 21-Mar-2015.)
((𝐹:𝐵1-1𝐶𝐻:𝐴𝐵𝐾:𝐴𝐵) → ((𝐹𝐻) = (𝐹𝐾) ↔ 𝐻 = 𝐾))
 
Theoremcocan2 5689 A surjection is right-cancelable. (Contributed by FL, 21-Nov-2011.) (Proof shortened by Mario Carneiro, 21-Mar-2015.)
((𝐹:𝐴onto𝐵𝐻 Fn 𝐵𝐾 Fn 𝐵) → ((𝐻𝐹) = (𝐾𝐹) ↔ 𝐻 = 𝐾))
 
Theoremfcof1o 5690 Show that two functions are inverse to each other by computing their compositions. (Contributed by Mario Carneiro, 21-Mar-2015.)
(((𝐹:𝐴𝐵𝐺:𝐵𝐴) ∧ ((𝐹𝐺) = ( I ↾ 𝐵) ∧ (𝐺𝐹) = ( I ↾ 𝐴))) → (𝐹:𝐴1-1-onto𝐵𝐹 = 𝐺))
 
Theoremfoeqcnvco 5691 Condition for function equality in terms of vanishing of the composition with the converse. EDITORIAL: Is there a relation-algebraic proof of this? (Contributed by Stefan O'Rear, 12-Feb-2015.)
((𝐹:𝐴onto𝐵𝐺:𝐴onto𝐵) → (𝐹 = 𝐺 ↔ (𝐹𝐺) = ( I ↾ 𝐵)))
 
Theoremf1eqcocnv 5692 Condition for function equality in terms of vanishing of the composition with the inverse. (Contributed by Stefan O'Rear, 12-Feb-2015.)
((𝐹:𝐴1-1𝐵𝐺:𝐴1-1𝐵) → (𝐹 = 𝐺 ↔ (𝐹𝐺) = ( I ↾ 𝐴)))
 
Theoremfliftrel 5693* 𝐹, a function lift, is a subset of 𝑅 × 𝑆. (Contributed by Mario Carneiro, 23-Dec-2016.)
𝐹 = ran (𝑥𝑋 ↦ ⟨𝐴, 𝐵⟩)    &   ((𝜑𝑥𝑋) → 𝐴𝑅)    &   ((𝜑𝑥𝑋) → 𝐵𝑆)       (𝜑𝐹 ⊆ (𝑅 × 𝑆))
 
Theoremfliftel 5694* Elementhood in the relation 𝐹. (Contributed by Mario Carneiro, 23-Dec-2016.)
𝐹 = ran (𝑥𝑋 ↦ ⟨𝐴, 𝐵⟩)    &   ((𝜑𝑥𝑋) → 𝐴𝑅)    &   ((𝜑𝑥𝑋) → 𝐵𝑆)       (𝜑 → (𝐶𝐹𝐷 ↔ ∃𝑥𝑋 (𝐶 = 𝐴𝐷 = 𝐵)))
 
Theoremfliftel1 5695* Elementhood in the relation 𝐹. (Contributed by Mario Carneiro, 23-Dec-2016.)
𝐹 = ran (𝑥𝑋 ↦ ⟨𝐴, 𝐵⟩)    &   ((𝜑𝑥𝑋) → 𝐴𝑅)    &   ((𝜑𝑥𝑋) → 𝐵𝑆)       ((𝜑𝑥𝑋) → 𝐴𝐹𝐵)
 
Theoremfliftcnv 5696* Converse of the relation 𝐹. (Contributed by Mario Carneiro, 23-Dec-2016.)
𝐹 = ran (𝑥𝑋 ↦ ⟨𝐴, 𝐵⟩)    &   ((𝜑𝑥𝑋) → 𝐴𝑅)    &   ((𝜑𝑥𝑋) → 𝐵𝑆)       (𝜑𝐹 = ran (𝑥𝑋 ↦ ⟨𝐵, 𝐴⟩))
 
Theoremfliftfun 5697* The function 𝐹 is the unique function defined by 𝐹𝐴 = 𝐵, provided that the well-definedness condition holds. (Contributed by Mario Carneiro, 23-Dec-2016.)
𝐹 = ran (𝑥𝑋 ↦ ⟨𝐴, 𝐵⟩)    &   ((𝜑𝑥𝑋) → 𝐴𝑅)    &   ((𝜑𝑥𝑋) → 𝐵𝑆)    &   (𝑥 = 𝑦𝐴 = 𝐶)    &   (𝑥 = 𝑦𝐵 = 𝐷)       (𝜑 → (Fun 𝐹 ↔ ∀𝑥𝑋𝑦𝑋 (𝐴 = 𝐶𝐵 = 𝐷)))
 
Theoremfliftfund 5698* The function 𝐹 is the unique function defined by 𝐹𝐴 = 𝐵, provided that the well-definedness condition holds. (Contributed by Mario Carneiro, 23-Dec-2016.)
𝐹 = ran (𝑥𝑋 ↦ ⟨𝐴, 𝐵⟩)    &   ((𝜑𝑥𝑋) → 𝐴𝑅)    &   ((𝜑𝑥𝑋) → 𝐵𝑆)    &   (𝑥 = 𝑦𝐴 = 𝐶)    &   (𝑥 = 𝑦𝐵 = 𝐷)    &   ((𝜑 ∧ (𝑥𝑋𝑦𝑋𝐴 = 𝐶)) → 𝐵 = 𝐷)       (𝜑 → Fun 𝐹)
 
Theoremfliftfuns 5699* The function 𝐹 is the unique function defined by 𝐹𝐴 = 𝐵, provided that the well-definedness condition holds. (Contributed by Mario Carneiro, 23-Dec-2016.)
𝐹 = ran (𝑥𝑋 ↦ ⟨𝐴, 𝐵⟩)    &   ((𝜑𝑥𝑋) → 𝐴𝑅)    &   ((𝜑𝑥𝑋) → 𝐵𝑆)       (𝜑 → (Fun 𝐹 ↔ ∀𝑦𝑋𝑧𝑋 (𝑦 / 𝑥𝐴 = 𝑧 / 𝑥𝐴𝑦 / 𝑥𝐵 = 𝑧 / 𝑥𝐵)))
 
Theoremfliftf 5700* The domain and range of the function 𝐹. (Contributed by Mario Carneiro, 23-Dec-2016.)
𝐹 = ran (𝑥𝑋 ↦ ⟨𝐴, 𝐵⟩)    &   ((𝜑𝑥𝑋) → 𝐴𝑅)    &   ((𝜑𝑥𝑋) → 𝐵𝑆)       (𝜑 → (Fun 𝐹𝐹:ran (𝑥𝑋𝐴)⟶𝑆))
    < Previous  Next >

Page List
Jump to page: Contents  1 1-100 2 101-200 3 201-300 4 301-400 5 401-500 6 501-600 7 601-700 8 701-800 9 801-900 10 901-1000 11 1001-1100 12 1101-1200 13 1201-1300 14 1301-1400 15 1401-1500 16 1501-1600 17 1601-1700 18 1701-1800 19 1801-1900 20 1901-2000 21 2001-2100 22 2101-2200 23 2201-2300 24 2301-2400 25 2401-2500 26 2501-2600 27 2601-2700 28 2701-2800 29 2801-2900 30 2901-3000 31 3001-3100 32 3101-3200 33 3201-3300 34 3301-3400 35 3401-3500 36 3501-3600 37 3601-3700 38 3701-3800 39 3801-3900 40 3901-4000 41 4001-4100 42 4101-4200 43 4201-4300 44 4301-4400 45 4401-4500 46 4501-4600 47 4601-4700 48 4701-4800 49 4801-4900 50 4901-5000 51 5001-5100 52 5101-5200 53 5201-5300 54 5301-5400 55 5401-5500 56 5501-5600 57 5601-5700 58 5701-5800 59 5801-5900 60 5901-6000 61 6001-6100 62 6101-6200 63 6201-6300 64 6301-6400 65 6401-6500 66 6501-6600 67 6601-6700 68 6701-6800 69 6801-6900 70 6901-7000 71 7001-7100 72 7101-7200 73 7201-7300 74 7301-7400 75 7401-7500 76 7501-7600 77 7601-7700 78 7701-7800 79 7801-7900 80 7901-8000 81 8001-8100 82 8101-8200 83 8201-8300 84 8301-8400 85 8401-8500 86 8501-8600 87 8601-8700 88 8701-8800 89 8801-8900 90 8901-9000 91 9001-9100 92 9101-9200 93 9201-9300 94 9301-9400 95 9401-9500 96 9501-9600 97 9601-9700 98 9701-9800 99 9801-9900 100 9901-10000 101 10001-10100 102 10101-10200 103 10201-10300 104 10301-10400 105 10401-10500 106 10501-10600 107 10601-10700 108 10701-10800 109 10801-10900 110 10901-11000 111 11001-11100 112 11101-11200 113 11201-11300 114 11301-11400 115 11401-11500 116 11501-11600 117 11601-11700 118 11701-11800 119 11801-11900 120 11901-12000 121 12001-12100 122 12101-12200 123 12201-12300 124 12301-12400 125 12401-12500 126 12501-12600 127 12601-12700 128 12701-12800 129 12801-12900 130 12901-13000 131 13001-13100 132 13101-13200 133 13201-13250
  Copyright terms: Public domain < Previous  Next >