Type | Label | Description |
Statement |
|
Theorem | offveqb 6101* |
Equivalent expressions for equality with a function operation.
(Contributed by NM, 9-Oct-2014.) (Proof shortened by Mario Carneiro,
5-Dec-2016.)
|
⊢ (𝜑 → 𝐴 ∈ 𝑉)
& ⊢ (𝜑 → 𝐹 Fn 𝐴)
& ⊢ (𝜑 → 𝐺 Fn 𝐴)
& ⊢ (𝜑 → 𝐻 Fn 𝐴)
& ⊢ ((𝜑 ∧ 𝑥 ∈ 𝐴) → (𝐹‘𝑥) = 𝐵)
& ⊢ ((𝜑 ∧ 𝑥 ∈ 𝐴) → (𝐺‘𝑥) = 𝐶) ⇒ ⊢ (𝜑 → (𝐻 = (𝐹 ∘𝑓 𝑅𝐺) ↔ ∀𝑥 ∈ 𝐴 (𝐻‘𝑥) = (𝐵𝑅𝐶))) |
|
Theorem | ofc12 6102 |
Function operation on two constant functions. (Contributed by Mario
Carneiro, 28-Jul-2014.)
|
⊢ (𝜑 → 𝐴 ∈ 𝑉)
& ⊢ (𝜑 → 𝐵 ∈ 𝑊)
& ⊢ (𝜑 → 𝐶 ∈ 𝑋) ⇒ ⊢ (𝜑 → ((𝐴 × {𝐵}) ∘𝑓 𝑅(𝐴 × {𝐶})) = (𝐴 × {(𝐵𝑅𝐶)})) |
|
Theorem | caofref 6103* |
Transfer a reflexive law to the function relation. (Contributed by
Mario Carneiro, 28-Jul-2014.)
|
⊢ (𝜑 → 𝐴 ∈ 𝑉)
& ⊢ (𝜑 → 𝐹:𝐴⟶𝑆)
& ⊢ ((𝜑 ∧ 𝑥 ∈ 𝑆) → 𝑥𝑅𝑥) ⇒ ⊢ (𝜑 → 𝐹 ∘𝑟 𝑅𝐹) |
|
Theorem | caofinvl 6104* |
Transfer a left inverse law to the function operation. (Contributed
by NM, 22-Oct-2014.)
|
⊢ (𝜑 → 𝐴 ∈ 𝑉)
& ⊢ (𝜑 → 𝐹:𝐴⟶𝑆)
& ⊢ (𝜑 → 𝐵 ∈ 𝑊)
& ⊢ (𝜑 → 𝑁:𝑆⟶𝑆)
& ⊢ (𝜑 → 𝐺 = (𝑣 ∈ 𝐴 ↦ (𝑁‘(𝐹‘𝑣)))) & ⊢ ((𝜑 ∧ 𝑥 ∈ 𝑆) → ((𝑁‘𝑥)𝑅𝑥) = 𝐵) ⇒ ⊢ (𝜑 → (𝐺 ∘𝑓 𝑅𝐹) = (𝐴 × {𝐵})) |
|
Theorem | caofcom 6105* |
Transfer a commutative law to the function operation. (Contributed by
Mario Carneiro, 26-Jul-2014.)
|
⊢ (𝜑 → 𝐴 ∈ 𝑉)
& ⊢ (𝜑 → 𝐹:𝐴⟶𝑆)
& ⊢ (𝜑 → 𝐺:𝐴⟶𝑆)
& ⊢ ((𝜑 ∧ (𝑥 ∈ 𝑆 ∧ 𝑦 ∈ 𝑆)) → (𝑥𝑅𝑦) = (𝑦𝑅𝑥)) ⇒ ⊢ (𝜑 → (𝐹 ∘𝑓 𝑅𝐺) = (𝐺 ∘𝑓 𝑅𝐹)) |
|
Theorem | caofrss 6106* |
Transfer a relation subset law to the function relation. (Contributed
by Mario Carneiro, 28-Jul-2014.)
|
⊢ (𝜑 → 𝐴 ∈ 𝑉)
& ⊢ (𝜑 → 𝐹:𝐴⟶𝑆)
& ⊢ (𝜑 → 𝐺:𝐴⟶𝑆)
& ⊢ ((𝜑 ∧ (𝑥 ∈ 𝑆 ∧ 𝑦 ∈ 𝑆)) → (𝑥𝑅𝑦 → 𝑥𝑇𝑦)) ⇒ ⊢ (𝜑 → (𝐹 ∘𝑟 𝑅𝐺 → 𝐹 ∘𝑟 𝑇𝐺)) |
|
Theorem | caoftrn 6107* |
Transfer a transitivity law to the function relation. (Contributed by
Mario Carneiro, 28-Jul-2014.)
|
⊢ (𝜑 → 𝐴 ∈ 𝑉)
& ⊢ (𝜑 → 𝐹:𝐴⟶𝑆)
& ⊢ (𝜑 → 𝐺:𝐴⟶𝑆)
& ⊢ (𝜑 → 𝐻:𝐴⟶𝑆)
& ⊢ ((𝜑 ∧ (𝑥 ∈ 𝑆 ∧ 𝑦 ∈ 𝑆 ∧ 𝑧 ∈ 𝑆)) → ((𝑥𝑅𝑦 ∧ 𝑦𝑇𝑧) → 𝑥𝑈𝑧)) ⇒ ⊢ (𝜑 → ((𝐹 ∘𝑟 𝑅𝐺 ∧ 𝐺 ∘𝑟 𝑇𝐻) → 𝐹 ∘𝑟 𝑈𝐻)) |
|
2.6.14 Functions (continued)
|
|
Theorem | resfunexgALT 6108 |
The restriction of a function to a set exists. Compare Proposition 6.17
of [TakeutiZaring] p. 28. This
version has a shorter proof than
resfunexg 5737 but requires ax-pow 4174 and ax-un 4433. (Contributed by NM,
7-Apr-1995.) (Proof modification is discouraged.)
(New usage is discouraged.)
|
⊢ ((Fun 𝐴 ∧ 𝐵 ∈ 𝐶) → (𝐴 ↾ 𝐵) ∈ V) |
|
Theorem | cofunexg 6109 |
Existence of a composition when the first member is a function.
(Contributed by NM, 8-Oct-2007.)
|
⊢ ((Fun 𝐴 ∧ 𝐵 ∈ 𝐶) → (𝐴 ∘ 𝐵) ∈ V) |
|
Theorem | cofunex2g 6110 |
Existence of a composition when the second member is one-to-one.
(Contributed by NM, 8-Oct-2007.)
|
⊢ ((𝐴 ∈ 𝑉 ∧ Fun ◡𝐵) → (𝐴 ∘ 𝐵) ∈ V) |
|
Theorem | fnexALT 6111 |
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 funimaexg 5300. This version of fnex 5738
uses
ax-pow 4174 and ax-un 4433, whereas fnex 5738
does not. (Contributed by NM,
14-Aug-1994.) (Proof modification is discouraged.)
(New usage is discouraged.)
|
⊢ ((𝐹 Fn 𝐴 ∧ 𝐴 ∈ 𝐵) → 𝐹 ∈ V) |
|
Theorem | funexw 6112 |
Weak version of funex 5739 that holds without ax-coll 4118. If the domain and
codomain of a function exist, so does the function. (Contributed by Rohan
Ridenour, 13-Aug-2023.)
|
⊢ ((Fun 𝐹 ∧ dom 𝐹 ∈ 𝐵 ∧ ran 𝐹 ∈ 𝐶) → 𝐹 ∈ V) |
|
Theorem | mptexw 6113* |
Weak version of mptex 5742 that holds without ax-coll 4118. If the domain
and codomain of a function given by maps-to notation are sets, the
function is a set. (Contributed by Rohan Ridenour, 13-Aug-2023.)
|
⊢ 𝐴 ∈ V & ⊢ 𝐶 ∈ V & ⊢ ∀𝑥 ∈ 𝐴 𝐵 ∈ 𝐶 ⇒ ⊢ (𝑥 ∈ 𝐴 ↦ 𝐵) ∈ V |
|
Theorem | funrnex 6114 |
If the domain of a function exists, so does its range. Part of Theorem
4.15(v) of [Monk1] p. 46. This theorem is
derived using the Axiom of
Replacement in the form of funex 5739. (Contributed by NM, 11-Nov-1995.)
|
⊢ (dom 𝐹 ∈ 𝐵 → (Fun 𝐹 → ran 𝐹 ∈ V)) |
|
Theorem | focdmex 6115 |
If the domain of an onto function exists, so does its codomain.
(Contributed by NM, 23-Jul-2004.)
|
⊢ (𝐴 ∈ 𝐶 → (𝐹:𝐴–onto→𝐵 → 𝐵 ∈ V)) |
|
Theorem | f1dmex 6116 |
If the codomain of a one-to-one function exists, so does its domain. This
can be thought of as a form of the Axiom of Replacement. (Contributed by
NM, 4-Sep-2004.)
|
⊢ ((𝐹:𝐴–1-1→𝐵 ∧ 𝐵 ∈ 𝐶) → 𝐴 ∈ V) |
|
Theorem | abrexex 6117* |
Existence of a class abstraction of existentially restricted sets. 𝑥
is normally a free-variable parameter in the class expression
substituted for 𝐵, which can be thought of as 𝐵(𝑥). This
simple-looking theorem is actually quite powerful and appears to involve
the Axiom of Replacement in an intrinsic way, as can be seen by tracing
back through the path mptexg 5741, funex 5739, fnex 5738, resfunexg 5737, and
funimaexg 5300. See also abrexex2 6124. (Contributed by NM, 16-Oct-2003.)
(Proof shortened by Mario Carneiro, 31-Aug-2015.)
|
⊢ 𝐴 ∈ V ⇒ ⊢ {𝑦 ∣ ∃𝑥 ∈ 𝐴 𝑦 = 𝐵} ∈ V |
|
Theorem | abrexexg 6118* |
Existence of a class abstraction of existentially restricted sets. 𝑥
is normally a free-variable parameter in 𝐵. The antecedent assures
us that 𝐴 is a set. (Contributed by NM,
3-Nov-2003.)
|
⊢ (𝐴 ∈ 𝑉 → {𝑦 ∣ ∃𝑥 ∈ 𝐴 𝑦 = 𝐵} ∈ V) |
|
Theorem | iunexg 6119* |
The existence of an indexed union. 𝑥 is normally a free-variable
parameter in 𝐵. (Contributed by NM, 23-Mar-2006.)
|
⊢ ((𝐴 ∈ 𝑉 ∧ ∀𝑥 ∈ 𝐴 𝐵 ∈ 𝑊) → ∪ 𝑥 ∈ 𝐴 𝐵 ∈ V) |
|
Theorem | abrexex2g 6120* |
Existence of an existentially restricted class abstraction.
(Contributed by Jeff Madsen, 2-Sep-2009.)
|
⊢ ((𝐴 ∈ 𝑉 ∧ ∀𝑥 ∈ 𝐴 {𝑦 ∣ 𝜑} ∈ 𝑊) → {𝑦 ∣ ∃𝑥 ∈ 𝐴 𝜑} ∈ V) |
|
Theorem | opabex3d 6121* |
Existence of an ordered pair abstraction, deduction version.
(Contributed by Alexander van der Vekens, 19-Oct-2017.)
|
⊢ (𝜑 → 𝐴 ∈ V) & ⊢ ((𝜑 ∧ 𝑥 ∈ 𝐴) → {𝑦 ∣ 𝜓} ∈ V) ⇒ ⊢ (𝜑 → {⟨𝑥, 𝑦⟩ ∣ (𝑥 ∈ 𝐴 ∧ 𝜓)} ∈ V) |
|
Theorem | opabex3 6122* |
Existence of an ordered pair abstraction. (Contributed by Jeff Madsen,
2-Sep-2009.)
|
⊢ 𝐴 ∈ V & ⊢ (𝑥 ∈ 𝐴 → {𝑦 ∣ 𝜑} ∈ V) ⇒ ⊢ {⟨𝑥, 𝑦⟩ ∣ (𝑥 ∈ 𝐴 ∧ 𝜑)} ∈ V |
|
Theorem | iunex 6123* |
The existence of an indexed union. 𝑥 is normally a free-variable
parameter in the class expression substituted for 𝐵, which can be
read informally as 𝐵(𝑥). (Contributed by NM, 13-Oct-2003.)
|
⊢ 𝐴 ∈ V & ⊢ 𝐵 ∈
V ⇒ ⊢ ∪ 𝑥 ∈ 𝐴 𝐵 ∈ V |
|
Theorem | abrexex2 6124* |
Existence of an existentially restricted class abstraction. 𝜑 is
normally has free-variable parameters 𝑥 and 𝑦. See
also
abrexex 6117. (Contributed by NM, 12-Sep-2004.)
|
⊢ 𝐴 ∈ V & ⊢ {𝑦 ∣ 𝜑} ∈ V ⇒ ⊢ {𝑦 ∣ ∃𝑥 ∈ 𝐴 𝜑} ∈ V |
|
Theorem | abexssex 6125* |
Existence of a class abstraction with an existentially quantified
expression. Both 𝑥 and 𝑦 can be free in 𝜑.
(Contributed
by NM, 29-Jul-2006.)
|
⊢ 𝐴 ∈ V & ⊢ {𝑦 ∣ 𝜑} ∈ V ⇒ ⊢ {𝑦 ∣ ∃𝑥(𝑥 ⊆ 𝐴 ∧ 𝜑)} ∈ V |
|
Theorem | abexex 6126* |
A condition where a class builder continues to exist after its wff is
existentially quantified. (Contributed by NM, 4-Mar-2007.)
|
⊢ 𝐴 ∈ V & ⊢ (𝜑 → 𝑥 ∈ 𝐴)
& ⊢ {𝑦 ∣ 𝜑} ∈ V ⇒ ⊢ {𝑦 ∣ ∃𝑥𝜑} ∈ V |
|
Theorem | oprabexd 6127* |
Existence of an operator abstraction. (Contributed by Jeff Madsen,
2-Sep-2009.)
|
⊢ (𝜑 → 𝐴 ∈ V) & ⊢ (𝜑 → 𝐵 ∈ V) & ⊢ ((𝜑 ∧ (𝑥 ∈ 𝐴 ∧ 𝑦 ∈ 𝐵)) → ∃*𝑧𝜓)
& ⊢ (𝜑 → 𝐹 = {⟨⟨𝑥, 𝑦⟩, 𝑧⟩ ∣ ((𝑥 ∈ 𝐴 ∧ 𝑦 ∈ 𝐵) ∧ 𝜓)}) ⇒ ⊢ (𝜑 → 𝐹 ∈ V) |
|
Theorem | oprabex 6128* |
Existence of an operation class abstraction. (Contributed by NM,
19-Oct-2004.)
|
⊢ 𝐴 ∈ V & ⊢ 𝐵 ∈ V & ⊢ ((𝑥 ∈ 𝐴 ∧ 𝑦 ∈ 𝐵) → ∃*𝑧𝜑)
& ⊢ 𝐹 = {⟨⟨𝑥, 𝑦⟩, 𝑧⟩ ∣ ((𝑥 ∈ 𝐴 ∧ 𝑦 ∈ 𝐵) ∧ 𝜑)} ⇒ ⊢ 𝐹 ∈ V |
|
Theorem | oprabex3 6129* |
Existence of an operation class abstraction (special case).
(Contributed by NM, 19-Oct-2004.)
|
⊢ 𝐻 ∈ V & ⊢ 𝐹 = {⟨⟨𝑥, 𝑦⟩, 𝑧⟩ ∣ ((𝑥 ∈ (𝐻 × 𝐻) ∧ 𝑦 ∈ (𝐻 × 𝐻)) ∧ ∃𝑤∃𝑣∃𝑢∃𝑓((𝑥 = ⟨𝑤, 𝑣⟩ ∧ 𝑦 = ⟨𝑢, 𝑓⟩) ∧ 𝑧 = 𝑅))} ⇒ ⊢ 𝐹 ∈ V |
|
Theorem | oprabrexex2 6130* |
Existence of an existentially restricted operation abstraction.
(Contributed by Jeff Madsen, 11-Jun-2010.)
|
⊢ 𝐴 ∈ V & ⊢
{⟨⟨𝑥,
𝑦⟩, 𝑧⟩ ∣ 𝜑} ∈ V ⇒ ⊢ {⟨⟨𝑥, 𝑦⟩, 𝑧⟩ ∣ ∃𝑤 ∈ 𝐴 𝜑} ∈ V |
|
Theorem | ab2rexex 6131* |
Existence of a class abstraction of existentially restricted sets.
Variables 𝑥 and 𝑦 are normally
free-variable parameters in the
class expression substituted for 𝐶, which can be thought of as
𝐶(𝑥, 𝑦). See comments for abrexex 6117. (Contributed by NM,
20-Sep-2011.)
|
⊢ 𝐴 ∈ V & ⊢ 𝐵 ∈
V ⇒ ⊢ {𝑧 ∣ ∃𝑥 ∈ 𝐴 ∃𝑦 ∈ 𝐵 𝑧 = 𝐶} ∈ V |
|
Theorem | ab2rexex2 6132* |
Existence of an existentially restricted class abstraction. 𝜑
normally has free-variable parameters 𝑥, 𝑦, and 𝑧.
Compare abrexex2 6124. (Contributed by NM, 20-Sep-2011.)
|
⊢ 𝐴 ∈ V & ⊢ 𝐵 ∈ V & ⊢ {𝑧 ∣ 𝜑} ∈ V ⇒ ⊢ {𝑧 ∣ ∃𝑥 ∈ 𝐴 ∃𝑦 ∈ 𝐵 𝜑} ∈ V |
|
Theorem | xpexgALT 6133 |
The cross product of two sets is a set. Proposition 6.2 of
[TakeutiZaring] p. 23. This
version is proven using Replacement; see
xpexg 4740 for a version that uses the Power Set axiom
instead.
(Contributed by Mario Carneiro, 20-May-2013.)
(Proof modification is discouraged.) (New usage is discouraged.)
|
⊢ ((𝐴 ∈ 𝑉 ∧ 𝐵 ∈ 𝑊) → (𝐴 × 𝐵) ∈ V) |
|
Theorem | offval3 6134* |
General value of (𝐹 ∘𝑓 𝑅𝐺) with no assumptions on
functionality
of 𝐹 and 𝐺. (Contributed by Stefan
O'Rear, 24-Jan-2015.)
|
⊢ ((𝐹 ∈ 𝑉 ∧ 𝐺 ∈ 𝑊) → (𝐹 ∘𝑓 𝑅𝐺) = (𝑥 ∈ (dom 𝐹 ∩ dom 𝐺) ↦ ((𝐹‘𝑥)𝑅(𝐺‘𝑥)))) |
|
Theorem | offres 6135 |
Pointwise combination commutes with restriction. (Contributed by Stefan
O'Rear, 24-Jan-2015.)
|
⊢ ((𝐹 ∈ 𝑉 ∧ 𝐺 ∈ 𝑊) → ((𝐹 ∘𝑓 𝑅𝐺) ↾ 𝐷) = ((𝐹 ↾ 𝐷) ∘𝑓 𝑅(𝐺 ↾ 𝐷))) |
|
Theorem | ofmres 6136* |
Equivalent expressions for a restriction of the function operation map.
Unlike ∘𝑓 𝑅 which is a proper class, ( ∘𝑓 𝑅 ↾ (𝐴 × 𝐵)) can
be a set by ofmresex 6137, allowing it to be used as a function or
structure argument. By ofmresval 6093, the restricted operation map
values are the same as the original values, allowing theorems for
∘𝑓 𝑅 to be reused. (Contributed by NM,
20-Oct-2014.)
|
⊢ ( ∘𝑓 𝑅 ↾ (𝐴 × 𝐵)) = (𝑓 ∈ 𝐴, 𝑔 ∈ 𝐵 ↦ (𝑓 ∘𝑓 𝑅𝑔)) |
|
Theorem | ofmresex 6137 |
Existence of a restriction of the function operation map. (Contributed
by NM, 20-Oct-2014.)
|
⊢ (𝜑 → 𝐴 ∈ 𝑉)
& ⊢ (𝜑 → 𝐵 ∈ 𝑊) ⇒ ⊢ (𝜑 → ( ∘𝑓 𝑅 ↾ (𝐴 × 𝐵)) ∈ V) |
|
2.6.15 First and second members of an ordered
pair
|
|
Syntax | c1st 6138 |
Extend the definition of a class to include the first member an ordered
pair function.
|
class 1st |
|
Syntax | c2nd 6139 |
Extend the definition of a class to include the second member an ordered
pair function.
|
class 2nd |
|
Definition | df-1st 6140 |
Define a function that extracts the first member, or abscissa, of an
ordered pair. Theorem op1st 6146 proves that it does this. For example,
(1st ‘⟨ 3 , 4 ⟩) = 3 . Equivalent to Definition 5.13 (i) of
[Monk1] p. 52 (compare op1sta 5110 and op1stb 4478). The notation is the same
as Monk's. (Contributed by NM, 9-Oct-2004.)
|
⊢ 1st = (𝑥 ∈ V ↦ ∪ dom {𝑥}) |
|
Definition | df-2nd 6141 |
Define a function that extracts the second member, or ordinate, of an
ordered pair. Theorem op2nd 6147 proves that it does this. For example,
(2nd ‘⟨ 3 , 4 ⟩) = 4 . Equivalent to Definition 5.13 (ii)
of [Monk1] p. 52 (compare op2nda 5113 and op2ndb 5112). The notation is the
same as Monk's. (Contributed by NM, 9-Oct-2004.)
|
⊢ 2nd = (𝑥 ∈ V ↦ ∪ ran {𝑥}) |
|
Theorem | 1stvalg 6142 |
The value of the function that extracts the first member of an ordered
pair. (Contributed by NM, 9-Oct-2004.) (Revised by Mario Carneiro,
8-Sep-2013.)
|
⊢ (𝐴 ∈ V → (1st
‘𝐴) = ∪ dom {𝐴}) |
|
Theorem | 2ndvalg 6143 |
The value of the function that extracts the second member of an ordered
pair. (Contributed by NM, 9-Oct-2004.) (Revised by Mario Carneiro,
8-Sep-2013.)
|
⊢ (𝐴 ∈ V → (2nd
‘𝐴) = ∪ ran {𝐴}) |
|
Theorem | 1st0 6144 |
The value of the first-member function at the empty set. (Contributed by
NM, 23-Apr-2007.)
|
⊢ (1st ‘∅) =
∅ |
|
Theorem | 2nd0 6145 |
The value of the second-member function at the empty set. (Contributed by
NM, 23-Apr-2007.)
|
⊢ (2nd ‘∅) =
∅ |
|
Theorem | op1st 6146 |
Extract the first member of an ordered pair. (Contributed by NM,
5-Oct-2004.)
|
⊢ 𝐴 ∈ V & ⊢ 𝐵 ∈
V ⇒ ⊢ (1st
‘⟨𝐴, 𝐵⟩) = 𝐴 |
|
Theorem | op2nd 6147 |
Extract the second member of an ordered pair. (Contributed by NM,
5-Oct-2004.)
|
⊢ 𝐴 ∈ V & ⊢ 𝐵 ∈
V ⇒ ⊢ (2nd
‘⟨𝐴, 𝐵⟩) = 𝐵 |
|
Theorem | op1std 6148 |
Extract the first member of an ordered pair. (Contributed by Mario
Carneiro, 31-Aug-2015.)
|
⊢ 𝐴 ∈ V & ⊢ 𝐵 ∈
V ⇒ ⊢ (𝐶 = ⟨𝐴, 𝐵⟩ → (1st ‘𝐶) = 𝐴) |
|
Theorem | op2ndd 6149 |
Extract the second member of an ordered pair. (Contributed by Mario
Carneiro, 31-Aug-2015.)
|
⊢ 𝐴 ∈ V & ⊢ 𝐵 ∈
V ⇒ ⊢ (𝐶 = ⟨𝐴, 𝐵⟩ → (2nd ‘𝐶) = 𝐵) |
|
Theorem | op1stg 6150 |
Extract the first member of an ordered pair. (Contributed by NM,
19-Jul-2005.)
|
⊢ ((𝐴 ∈ 𝑉 ∧ 𝐵 ∈ 𝑊) → (1st ‘⟨𝐴, 𝐵⟩) = 𝐴) |
|
Theorem | op2ndg 6151 |
Extract the second member of an ordered pair. (Contributed by NM,
19-Jul-2005.)
|
⊢ ((𝐴 ∈ 𝑉 ∧ 𝐵 ∈ 𝑊) → (2nd ‘⟨𝐴, 𝐵⟩) = 𝐵) |
|
Theorem | ot1stg 6152 |
Extract the first member of an ordered triple. (Due to infrequent
usage, it isn't worthwhile at this point to define special extractors
for triples, so we reuse the ordered pair extractors for ot1stg 6152,
ot2ndg 6153, ot3rdgg 6154.) (Contributed by NM, 3-Apr-2015.) (Revised
by
Mario Carneiro, 2-May-2015.)
|
⊢ ((𝐴 ∈ 𝑉 ∧ 𝐵 ∈ 𝑊 ∧ 𝐶 ∈ 𝑋) → (1st
‘(1st ‘⟨𝐴, 𝐵, 𝐶⟩)) = 𝐴) |
|
Theorem | ot2ndg 6153 |
Extract the second member of an ordered triple. (See ot1stg 6152 comment.)
(Contributed by NM, 3-Apr-2015.) (Revised by Mario Carneiro,
2-May-2015.)
|
⊢ ((𝐴 ∈ 𝑉 ∧ 𝐵 ∈ 𝑊 ∧ 𝐶 ∈ 𝑋) → (2nd
‘(1st ‘⟨𝐴, 𝐵, 𝐶⟩)) = 𝐵) |
|
Theorem | ot3rdgg 6154 |
Extract the third member of an ordered triple. (See ot1stg 6152 comment.)
(Contributed by NM, 3-Apr-2015.)
|
⊢ ((𝐴 ∈ 𝑉 ∧ 𝐵 ∈ 𝑊 ∧ 𝐶 ∈ 𝑋) → (2nd ‘⟨𝐴, 𝐵, 𝐶⟩) = 𝐶) |
|
Theorem | 1stval2 6155 |
Alternate value of the function that extracts the first member of an
ordered pair. Definition 5.13 (i) of [Monk1] p. 52. (Contributed by
NM, 18-Aug-2006.)
|
⊢ (𝐴 ∈ (V × V) →
(1st ‘𝐴)
= ∩ ∩ 𝐴) |
|
Theorem | 2ndval2 6156 |
Alternate value of the function that extracts the second member of an
ordered pair. Definition 5.13 (ii) of [Monk1] p. 52. (Contributed by
NM, 18-Aug-2006.)
|
⊢ (𝐴 ∈ (V × V) →
(2nd ‘𝐴)
= ∩ ∩ ∩ ◡{𝐴}) |
|
Theorem | fo1st 6157 |
The 1st function maps the universe onto the
universe. (Contributed
by NM, 14-Oct-2004.) (Revised by Mario Carneiro, 8-Sep-2013.)
|
⊢ 1st :V–onto→V |
|
Theorem | fo2nd 6158 |
The 2nd function maps the universe onto the
universe. (Contributed
by NM, 14-Oct-2004.) (Revised by Mario Carneiro, 8-Sep-2013.)
|
⊢ 2nd :V–onto→V |
|
Theorem | f1stres 6159 |
Mapping of a restriction of the 1st (first
member of an ordered
pair) function. (Contributed by NM, 11-Oct-2004.) (Revised by Mario
Carneiro, 8-Sep-2013.)
|
⊢ (1st ↾ (𝐴 × 𝐵)):(𝐴 × 𝐵)⟶𝐴 |
|
Theorem | f2ndres 6160 |
Mapping of a restriction of the 2nd (second
member of an ordered
pair) function. (Contributed by NM, 7-Aug-2006.) (Revised by Mario
Carneiro, 8-Sep-2013.)
|
⊢ (2nd ↾ (𝐴 × 𝐵)):(𝐴 × 𝐵)⟶𝐵 |
|
Theorem | fo1stresm 6161* |
Onto mapping of a restriction of the 1st
(first member of an ordered
pair) function. (Contributed by Jim Kingdon, 24-Jan-2019.)
|
⊢ (∃𝑦 𝑦 ∈ 𝐵 → (1st ↾ (𝐴 × 𝐵)):(𝐴 × 𝐵)–onto→𝐴) |
|
Theorem | fo2ndresm 6162* |
Onto mapping of a restriction of the 2nd
(second member of an
ordered pair) function. (Contributed by Jim Kingdon, 24-Jan-2019.)
|
⊢ (∃𝑥 𝑥 ∈ 𝐴 → (2nd ↾ (𝐴 × 𝐵)):(𝐴 × 𝐵)–onto→𝐵) |
|
Theorem | 1stcof 6163 |
Composition of the first member function with another function.
(Contributed by NM, 12-Oct-2007.)
|
⊢ (𝐹:𝐴⟶(𝐵 × 𝐶) → (1st ∘ 𝐹):𝐴⟶𝐵) |
|
Theorem | 2ndcof 6164 |
Composition of the second member function with another function.
(Contributed by FL, 15-Oct-2012.)
|
⊢ (𝐹:𝐴⟶(𝐵 × 𝐶) → (2nd ∘ 𝐹):𝐴⟶𝐶) |
|
Theorem | xp1st 6165 |
Location of the first element of a Cartesian product. (Contributed by
Jeff Madsen, 2-Sep-2009.)
|
⊢ (𝐴 ∈ (𝐵 × 𝐶) → (1st ‘𝐴) ∈ 𝐵) |
|
Theorem | xp2nd 6166 |
Location of the second element of a Cartesian product. (Contributed by
Jeff Madsen, 2-Sep-2009.)
|
⊢ (𝐴 ∈ (𝐵 × 𝐶) → (2nd ‘𝐴) ∈ 𝐶) |
|
Theorem | 1stexg 6167 |
Existence of the first member of a set. (Contributed by Jim Kingdon,
26-Jan-2019.)
|
⊢ (𝐴 ∈ 𝑉 → (1st ‘𝐴) ∈ V) |
|
Theorem | 2ndexg 6168 |
Existence of the first member of a set. (Contributed by Jim Kingdon,
26-Jan-2019.)
|
⊢ (𝐴 ∈ 𝑉 → (2nd ‘𝐴) ∈ V) |
|
Theorem | elxp6 6169 |
Membership in a cross product. This version requires no quantifiers or
dummy variables. See also elxp4 5116. (Contributed by NM, 9-Oct-2004.)
|
⊢ (𝐴 ∈ (𝐵 × 𝐶) ↔ (𝐴 = ⟨(1st ‘𝐴), (2nd ‘𝐴)⟩ ∧ ((1st
‘𝐴) ∈ 𝐵 ∧ (2nd
‘𝐴) ∈ 𝐶))) |
|
Theorem | elxp7 6170 |
Membership in a cross product. This version requires no quantifiers or
dummy variables. See also elxp4 5116. (Contributed by NM, 19-Aug-2006.)
|
⊢ (𝐴 ∈ (𝐵 × 𝐶) ↔ (𝐴 ∈ (V × V) ∧
((1st ‘𝐴)
∈ 𝐵 ∧
(2nd ‘𝐴)
∈ 𝐶))) |
|
Theorem | oprssdmm 6171* |
Domain of closure of an operation. (Contributed by Jim Kingdon,
23-Oct-2023.)
|
⊢ ((𝜑 ∧ 𝑢 ∈ 𝑆) → ∃𝑣 𝑣 ∈ 𝑢)
& ⊢ ((𝜑 ∧ (𝑥 ∈ 𝑆 ∧ 𝑦 ∈ 𝑆)) → (𝑥𝐹𝑦) ∈ 𝑆)
& ⊢ (𝜑 → Rel 𝐹) ⇒ ⊢ (𝜑 → (𝑆 × 𝑆) ⊆ dom 𝐹) |
|
Theorem | eqopi 6172 |
Equality with an ordered pair. (Contributed by NM, 15-Dec-2008.)
(Revised by Mario Carneiro, 23-Feb-2014.)
|
⊢ ((𝐴 ∈ (𝑉 × 𝑊) ∧ ((1st ‘𝐴) = 𝐵 ∧ (2nd ‘𝐴) = 𝐶)) → 𝐴 = ⟨𝐵, 𝐶⟩) |
|
Theorem | xp2 6173* |
Representation of cross product based on ordered pair component
functions. (Contributed by NM, 16-Sep-2006.)
|
⊢ (𝐴 × 𝐵) = {𝑥 ∈ (V × V) ∣
((1st ‘𝑥)
∈ 𝐴 ∧
(2nd ‘𝑥)
∈ 𝐵)} |
|
Theorem | unielxp 6174 |
The membership relation for a cross product is inherited by union.
(Contributed by NM, 16-Sep-2006.)
|
⊢ (𝐴 ∈ (𝐵 × 𝐶) → ∪ 𝐴 ∈ ∪ (𝐵
× 𝐶)) |
|
Theorem | 1st2nd2 6175 |
Reconstruction of a member of a cross product in terms of its ordered pair
components. (Contributed by NM, 20-Oct-2013.)
|
⊢ (𝐴 ∈ (𝐵 × 𝐶) → 𝐴 = ⟨(1st ‘𝐴), (2nd ‘𝐴)⟩) |
|
Theorem | xpopth 6176 |
An ordered pair theorem for members of cross products. (Contributed by
NM, 20-Jun-2007.)
|
⊢ ((𝐴 ∈ (𝐶 × 𝐷) ∧ 𝐵 ∈ (𝑅 × 𝑆)) → (((1st ‘𝐴) = (1st
‘𝐵) ∧
(2nd ‘𝐴)
= (2nd ‘𝐵)) ↔ 𝐴 = 𝐵)) |
|
Theorem | eqop 6177 |
Two ways to express equality with an ordered pair. (Contributed by NM,
3-Sep-2007.) (Proof shortened by Mario Carneiro, 26-Apr-2015.)
|
⊢ (𝐴 ∈ (𝑉 × 𝑊) → (𝐴 = ⟨𝐵, 𝐶⟩ ↔ ((1st ‘𝐴) = 𝐵 ∧ (2nd ‘𝐴) = 𝐶))) |
|
Theorem | eqop2 6178 |
Two ways to express equality with an ordered pair. (Contributed by NM,
25-Feb-2014.)
|
⊢ 𝐵 ∈ V & ⊢ 𝐶 ∈
V ⇒ ⊢ (𝐴 = ⟨𝐵, 𝐶⟩ ↔ (𝐴 ∈ (V × V) ∧
((1st ‘𝐴)
= 𝐵 ∧ (2nd
‘𝐴) = 𝐶))) |
|
Theorem | op1steq 6179* |
Two ways of expressing that an element is the first member of an ordered
pair. (Contributed by NM, 22-Sep-2013.) (Revised by Mario Carneiro,
23-Feb-2014.)
|
⊢ (𝐴 ∈ (𝑉 × 𝑊) → ((1st ‘𝐴) = 𝐵 ↔ ∃𝑥 𝐴 = ⟨𝐵, 𝑥⟩)) |
|
Theorem | 2nd1st 6180 |
Swap the members of an ordered pair. (Contributed by NM, 31-Dec-2014.)
|
⊢ (𝐴 ∈ (𝐵 × 𝐶) → ∪ ◡{𝐴} = ⟨(2nd ‘𝐴), (1st ‘𝐴)⟩) |
|
Theorem | 1st2nd 6181 |
Reconstruction of a member of a relation in terms of its ordered pair
components. (Contributed by NM, 29-Aug-2006.)
|
⊢ ((Rel 𝐵 ∧ 𝐴 ∈ 𝐵) → 𝐴 = ⟨(1st ‘𝐴), (2nd ‘𝐴)⟩) |
|
Theorem | 1stdm 6182 |
The first ordered pair component of a member of a relation belongs to the
domain of the relation. (Contributed by NM, 17-Sep-2006.)
|
⊢ ((Rel 𝑅 ∧ 𝐴 ∈ 𝑅) → (1st ‘𝐴) ∈ dom 𝑅) |
|
Theorem | 2ndrn 6183 |
The second ordered pair component of a member of a relation belongs to the
range of the relation. (Contributed by NM, 17-Sep-2006.)
|
⊢ ((Rel 𝑅 ∧ 𝐴 ∈ 𝑅) → (2nd ‘𝐴) ∈ ran 𝑅) |
|
Theorem | 1st2ndbr 6184 |
Express an element of a relation as a relationship between first and
second components. (Contributed by Mario Carneiro, 22-Jun-2016.)
|
⊢ ((Rel 𝐵 ∧ 𝐴 ∈ 𝐵) → (1st ‘𝐴)𝐵(2nd ‘𝐴)) |
|
Theorem | releldm2 6185* |
Two ways of expressing membership in the domain of a relation.
(Contributed by NM, 22-Sep-2013.)
|
⊢ (Rel 𝐴 → (𝐵 ∈ dom 𝐴 ↔ ∃𝑥 ∈ 𝐴 (1st ‘𝑥) = 𝐵)) |
|
Theorem | reldm 6186* |
An expression for the domain of a relation. (Contributed by NM,
22-Sep-2013.)
|
⊢ (Rel 𝐴 → dom 𝐴 = ran (𝑥 ∈ 𝐴 ↦ (1st ‘𝑥))) |
|
Theorem | sbcopeq1a 6187 |
Equality theorem for substitution of a class for an ordered pair (analog
of sbceq1a 2972 that avoids the existential quantifiers of copsexg 4244).
(Contributed by NM, 19-Aug-2006.) (Revised by Mario Carneiro,
31-Aug-2015.)
|
⊢ (𝐴 = ⟨𝑥, 𝑦⟩ → ([(1st
‘𝐴) / 𝑥][(2nd
‘𝐴) / 𝑦]𝜑 ↔ 𝜑)) |
|
Theorem | csbopeq1a 6188 |
Equality theorem for substitution of a class 𝐴 for an ordered pair
⟨𝑥, 𝑦⟩ in 𝐵 (analog of csbeq1a 3066). (Contributed by NM,
19-Aug-2006.) (Revised by Mario Carneiro, 31-Aug-2015.)
|
⊢ (𝐴 = ⟨𝑥, 𝑦⟩ → ⦋(1st
‘𝐴) / 𝑥⦌⦋(2nd
‘𝐴) / 𝑦⦌𝐵 = 𝐵) |
|
Theorem | dfopab2 6189* |
A way to define an ordered-pair class abstraction without using
existential quantifiers. (Contributed by NM, 18-Aug-2006.) (Revised by
Mario Carneiro, 31-Aug-2015.)
|
⊢ {⟨𝑥, 𝑦⟩ ∣ 𝜑} = {𝑧 ∈ (V × V) ∣
[(1st ‘𝑧) / 𝑥][(2nd ‘𝑧) / 𝑦]𝜑} |
|
Theorem | dfoprab3s 6190* |
A way to define an operation class abstraction without using existential
quantifiers. (Contributed by NM, 18-Aug-2006.) (Revised by Mario
Carneiro, 31-Aug-2015.)
|
⊢ {⟨⟨𝑥, 𝑦⟩, 𝑧⟩ ∣ 𝜑} = {⟨𝑤, 𝑧⟩ ∣ (𝑤 ∈ (V × V) ∧
[(1st ‘𝑤) / 𝑥][(2nd ‘𝑤) / 𝑦]𝜑)} |
|
Theorem | dfoprab3 6191* |
Operation class abstraction expressed without existential quantifiers.
(Contributed by NM, 16-Dec-2008.)
|
⊢ (𝑤 = ⟨𝑥, 𝑦⟩ → (𝜑 ↔ 𝜓)) ⇒ ⊢ {⟨𝑤, 𝑧⟩ ∣ (𝑤 ∈ (V × V) ∧ 𝜑)} = {⟨⟨𝑥, 𝑦⟩, 𝑧⟩ ∣ 𝜓} |
|
Theorem | dfoprab4 6192* |
Operation class abstraction expressed without existential quantifiers.
(Contributed by NM, 3-Sep-2007.) (Revised by Mario Carneiro,
31-Aug-2015.)
|
⊢ (𝑤 = ⟨𝑥, 𝑦⟩ → (𝜑 ↔ 𝜓)) ⇒ ⊢ {⟨𝑤, 𝑧⟩ ∣ (𝑤 ∈ (𝐴 × 𝐵) ∧ 𝜑)} = {⟨⟨𝑥, 𝑦⟩, 𝑧⟩ ∣ ((𝑥 ∈ 𝐴 ∧ 𝑦 ∈ 𝐵) ∧ 𝜓)} |
|
Theorem | dfoprab4f 6193* |
Operation class abstraction expressed without existential quantifiers.
(Unnecessary distinct variable restrictions were removed by David
Abernethy, 19-Jun-2012.) (Contributed by NM, 20-Dec-2008.) (Revised by
Mario Carneiro, 31-Aug-2015.)
|
⊢ Ⅎ𝑥𝜑
& ⊢ Ⅎ𝑦𝜑
& ⊢ (𝑤 = ⟨𝑥, 𝑦⟩ → (𝜑 ↔ 𝜓)) ⇒ ⊢ {⟨𝑤, 𝑧⟩ ∣ (𝑤 ∈ (𝐴 × 𝐵) ∧ 𝜑)} = {⟨⟨𝑥, 𝑦⟩, 𝑧⟩ ∣ ((𝑥 ∈ 𝐴 ∧ 𝑦 ∈ 𝐵) ∧ 𝜓)} |
|
Theorem | dfxp3 6194* |
Define the cross product of three classes. Compare df-xp 4632.
(Contributed by FL, 6-Nov-2013.) (Proof shortened by Mario Carneiro,
3-Nov-2015.)
|
⊢ ((𝐴 × 𝐵) × 𝐶) = {⟨⟨𝑥, 𝑦⟩, 𝑧⟩ ∣ (𝑥 ∈ 𝐴 ∧ 𝑦 ∈ 𝐵 ∧ 𝑧 ∈ 𝐶)} |
|
Theorem | elopabi 6195* |
A consequence of membership in an ordered-pair class abstraction, using
ordered pair extractors. (Contributed by NM, 29-Aug-2006.)
|
⊢ (𝑥 = (1st ‘𝐴) → (𝜑 ↔ 𝜓)) & ⊢ (𝑦 = (2nd ‘𝐴) → (𝜓 ↔ 𝜒)) ⇒ ⊢ (𝐴 ∈ {⟨𝑥, 𝑦⟩ ∣ 𝜑} → 𝜒) |
|
Theorem | eloprabi 6196* |
A consequence of membership in an operation class abstraction, using
ordered pair extractors. (Contributed by NM, 6-Nov-2006.) (Revised by
David Abernethy, 19-Jun-2012.)
|
⊢ (𝑥 = (1st ‘(1st
‘𝐴)) → (𝜑 ↔ 𝜓)) & ⊢ (𝑦 = (2nd
‘(1st ‘𝐴)) → (𝜓 ↔ 𝜒)) & ⊢ (𝑧 = (2nd ‘𝐴) → (𝜒 ↔ 𝜃)) ⇒ ⊢ (𝐴 ∈ {⟨⟨𝑥, 𝑦⟩, 𝑧⟩ ∣ 𝜑} → 𝜃) |
|
Theorem | mpomptsx 6197* |
Express a two-argument function as a one-argument function, or
vice-versa. (Contributed by Mario Carneiro, 24-Dec-2016.)
|
⊢ (𝑥 ∈ 𝐴, 𝑦 ∈ 𝐵 ↦ 𝐶) = (𝑧 ∈ ∪
𝑥 ∈ 𝐴 ({𝑥} × 𝐵) ↦ ⦋(1st
‘𝑧) / 𝑥⦌⦋(2nd
‘𝑧) / 𝑦⦌𝐶) |
|
Theorem | mpompts 6198* |
Express a two-argument function as a one-argument function, or
vice-versa. (Contributed by Mario Carneiro, 24-Sep-2015.)
|
⊢ (𝑥 ∈ 𝐴, 𝑦 ∈ 𝐵 ↦ 𝐶) = (𝑧 ∈ (𝐴 × 𝐵) ↦ ⦋(1st
‘𝑧) / 𝑥⦌⦋(2nd
‘𝑧) / 𝑦⦌𝐶) |
|
Theorem | dmmpossx 6199* |
The domain of a mapping is a subset of its base class. (Contributed by
Mario Carneiro, 9-Feb-2015.)
|
⊢ 𝐹 = (𝑥 ∈ 𝐴, 𝑦 ∈ 𝐵 ↦ 𝐶) ⇒ ⊢ dom 𝐹 ⊆ ∪ 𝑥 ∈ 𝐴 ({𝑥} × 𝐵) |
|
Theorem | fmpox 6200* |
Functionality, domain and codomain of a class given by the maps-to
notation, where 𝐵(𝑥) is not constant but depends on 𝑥.
(Contributed by NM, 29-Dec-2014.)
|
⊢ 𝐹 = (𝑥 ∈ 𝐴, 𝑦 ∈ 𝐵 ↦ 𝐶) ⇒ ⊢ (∀𝑥 ∈ 𝐴 ∀𝑦 ∈ 𝐵 𝐶 ∈ 𝐷 ↔ 𝐹:∪ 𝑥 ∈ 𝐴 ({𝑥} × 𝐵)⟶𝐷) |