Theorem List for Intuitionistic Logic Explorer - 4901-5000 *Has distinct variable
group(s)
Type | Label | Description |
Statement |
|
Theorem | relssres 4901 |
Simplification law for restriction. (Contributed by NM,
16-Aug-1994.)
|
⊢ ((Rel 𝐴 ∧ dom 𝐴 ⊆ 𝐵) → (𝐴 ↾ 𝐵) = 𝐴) |
|
Theorem | resdm 4902 |
A relation restricted to its domain equals itself. (Contributed by NM,
12-Dec-2006.)
|
⊢ (Rel 𝐴 → (𝐴 ↾ dom 𝐴) = 𝐴) |
|
Theorem | resexg 4903 |
The restriction of a set is a set. (Contributed by NM, 28-Mar-1998.)
(Proof shortened by Andrew Salmon, 27-Aug-2011.)
|
⊢ (𝐴 ∈ 𝑉 → (𝐴 ↾ 𝐵) ∈ V) |
|
Theorem | resex 4904 |
The restriction of a set is a set. (Contributed by Jeff Madsen,
19-Jun-2011.)
|
⊢ 𝐴 ∈ V ⇒ ⊢ (𝐴 ↾ 𝐵) ∈ V |
|
Theorem | resindm 4905 |
When restricting a relation, intersecting with the domain of the relation
has no effect. (Contributed by FL, 6-Oct-2008.)
|
⊢ (Rel 𝐴 → (𝐴 ↾ (𝐵 ∩ dom 𝐴)) = (𝐴 ↾ 𝐵)) |
|
Theorem | resdmdfsn 4906 |
Restricting a relation to its domain without a set is the same as
restricting the relation to the universe without this set. (Contributed
by AV, 2-Dec-2018.)
|
⊢ (Rel 𝑅 → (𝑅 ↾ (V ∖ {𝑋})) = (𝑅 ↾ (dom 𝑅 ∖ {𝑋}))) |
|
Theorem | resopab 4907* |
Restriction of a class abstraction of ordered pairs. (Contributed by
NM, 5-Nov-2002.)
|
⊢ ({〈𝑥, 𝑦〉 ∣ 𝜑} ↾ 𝐴) = {〈𝑥, 𝑦〉 ∣ (𝑥 ∈ 𝐴 ∧ 𝜑)} |
|
Theorem | resiexg 4908 |
The existence of a restricted identity function, proved without using
the Axiom of Replacement. (Contributed by NM, 13-Jan-2007.)
|
⊢ (𝐴 ∈ 𝑉 → ( I ↾ 𝐴) ∈ V) |
|
Theorem | iss 4909 |
A subclass of the identity function is the identity function restricted
to its domain. (Contributed by NM, 13-Dec-2003.) (Proof shortened by
Andrew Salmon, 27-Aug-2011.)
|
⊢ (𝐴 ⊆ I ↔ 𝐴 = ( I ↾ dom 𝐴)) |
|
Theorem | resopab2 4910* |
Restriction of a class abstraction of ordered pairs. (Contributed by
NM, 24-Aug-2007.)
|
⊢ (𝐴 ⊆ 𝐵 → ({〈𝑥, 𝑦〉 ∣ (𝑥 ∈ 𝐵 ∧ 𝜑)} ↾ 𝐴) = {〈𝑥, 𝑦〉 ∣ (𝑥 ∈ 𝐴 ∧ 𝜑)}) |
|
Theorem | resmpt 4911* |
Restriction of the mapping operation. (Contributed by Mario Carneiro,
15-Jul-2013.)
|
⊢ (𝐵 ⊆ 𝐴 → ((𝑥 ∈ 𝐴 ↦ 𝐶) ↾ 𝐵) = (𝑥 ∈ 𝐵 ↦ 𝐶)) |
|
Theorem | resmpt3 4912* |
Unconditional restriction of the mapping operation. (Contributed by
Stefan O'Rear, 24-Jan-2015.) (Proof shortened by Mario Carneiro,
22-Mar-2015.)
|
⊢ ((𝑥 ∈ 𝐴 ↦ 𝐶) ↾ 𝐵) = (𝑥 ∈ (𝐴 ∩ 𝐵) ↦ 𝐶) |
|
Theorem | resmptf 4913 |
Restriction of the mapping operation. (Contributed by Thierry Arnoux,
28-Mar-2017.)
|
⊢ Ⅎ𝑥𝐴
& ⊢ Ⅎ𝑥𝐵 ⇒ ⊢ (𝐵 ⊆ 𝐴 → ((𝑥 ∈ 𝐴 ↦ 𝐶) ↾ 𝐵) = (𝑥 ∈ 𝐵 ↦ 𝐶)) |
|
Theorem | resmptd 4914* |
Restriction of the mapping operation, deduction form. (Contributed by
Glauco Siliprandi, 11-Dec-2019.)
|
⊢ (𝜑 → 𝐵 ⊆ 𝐴) ⇒ ⊢ (𝜑 → ((𝑥 ∈ 𝐴 ↦ 𝐶) ↾ 𝐵) = (𝑥 ∈ 𝐵 ↦ 𝐶)) |
|
Theorem | dfres2 4915* |
Alternate definition of the restriction operation. (Contributed by
Mario Carneiro, 5-Nov-2013.)
|
⊢ (𝑅 ↾ 𝐴) = {〈𝑥, 𝑦〉 ∣ (𝑥 ∈ 𝐴 ∧ 𝑥𝑅𝑦)} |
|
Theorem | opabresid 4916* |
The restricted identity expressed with the class builder. (Contributed
by FL, 25-Apr-2012.)
|
⊢ {〈𝑥, 𝑦〉 ∣ (𝑥 ∈ 𝐴 ∧ 𝑦 = 𝑥)} = ( I ↾ 𝐴) |
|
Theorem | mptresid 4917* |
The restricted identity expressed with the maps-to notation.
(Contributed by FL, 25-Apr-2012.)
|
⊢ (𝑥 ∈ 𝐴 ↦ 𝑥) = ( I ↾ 𝐴) |
|
Theorem | dmresi 4918 |
The domain of a restricted identity function. (Contributed by NM,
27-Aug-2004.)
|
⊢ dom ( I ↾ 𝐴) = 𝐴 |
|
Theorem | resid 4919 |
Any relation restricted to the universe is itself. (Contributed by NM,
16-Mar-2004.)
|
⊢ (Rel 𝐴 → (𝐴 ↾ V) = 𝐴) |
|
Theorem | imaeq1 4920 |
Equality theorem for image. (Contributed by NM, 14-Aug-1994.)
|
⊢ (𝐴 = 𝐵 → (𝐴 “ 𝐶) = (𝐵 “ 𝐶)) |
|
Theorem | imaeq2 4921 |
Equality theorem for image. (Contributed by NM, 14-Aug-1994.)
|
⊢ (𝐴 = 𝐵 → (𝐶 “ 𝐴) = (𝐶 “ 𝐵)) |
|
Theorem | imaeq1i 4922 |
Equality theorem for image. (Contributed by NM, 21-Dec-2008.)
|
⊢ 𝐴 = 𝐵 ⇒ ⊢ (𝐴 “ 𝐶) = (𝐵 “ 𝐶) |
|
Theorem | imaeq2i 4923 |
Equality theorem for image. (Contributed by NM, 21-Dec-2008.)
|
⊢ 𝐴 = 𝐵 ⇒ ⊢ (𝐶 “ 𝐴) = (𝐶 “ 𝐵) |
|
Theorem | imaeq1d 4924 |
Equality theorem for image. (Contributed by FL, 15-Dec-2006.)
|
⊢ (𝜑 → 𝐴 = 𝐵) ⇒ ⊢ (𝜑 → (𝐴 “ 𝐶) = (𝐵 “ 𝐶)) |
|
Theorem | imaeq2d 4925 |
Equality theorem for image. (Contributed by FL, 15-Dec-2006.)
|
⊢ (𝜑 → 𝐴 = 𝐵) ⇒ ⊢ (𝜑 → (𝐶 “ 𝐴) = (𝐶 “ 𝐵)) |
|
Theorem | imaeq12d 4926 |
Equality theorem for image. (Contributed by Mario Carneiro,
4-Dec-2016.)
|
⊢ (𝜑 → 𝐴 = 𝐵)
& ⊢ (𝜑 → 𝐶 = 𝐷) ⇒ ⊢ (𝜑 → (𝐴 “ 𝐶) = (𝐵 “ 𝐷)) |
|
Theorem | dfima2 4927* |
Alternate definition of image. Compare definition (d) of [Enderton]
p. 44. (Contributed by NM, 19-Apr-2004.) (Proof shortened by Andrew
Salmon, 27-Aug-2011.)
|
⊢ (𝐴 “ 𝐵) = {𝑦 ∣ ∃𝑥 ∈ 𝐵 𝑥𝐴𝑦} |
|
Theorem | dfima3 4928* |
Alternate definition of image. Compare definition (d) of [Enderton]
p. 44. (Contributed by NM, 14-Aug-1994.) (Proof shortened by Andrew
Salmon, 27-Aug-2011.)
|
⊢ (𝐴 “ 𝐵) = {𝑦 ∣ ∃𝑥(𝑥 ∈ 𝐵 ∧ 〈𝑥, 𝑦〉 ∈ 𝐴)} |
|
Theorem | elimag 4929* |
Membership in an image. Theorem 34 of [Suppes]
p. 65. (Contributed by
NM, 20-Jan-2007.)
|
⊢ (𝐴 ∈ 𝑉 → (𝐴 ∈ (𝐵 “ 𝐶) ↔ ∃𝑥 ∈ 𝐶 𝑥𝐵𝐴)) |
|
Theorem | elima 4930* |
Membership in an image. Theorem 34 of [Suppes]
p. 65. (Contributed by
NM, 19-Apr-2004.)
|
⊢ 𝐴 ∈ V ⇒ ⊢ (𝐴 ∈ (𝐵 “ 𝐶) ↔ ∃𝑥 ∈ 𝐶 𝑥𝐵𝐴) |
|
Theorem | elima2 4931* |
Membership in an image. Theorem 34 of [Suppes]
p. 65. (Contributed by
NM, 11-Aug-2004.)
|
⊢ 𝐴 ∈ V ⇒ ⊢ (𝐴 ∈ (𝐵 “ 𝐶) ↔ ∃𝑥(𝑥 ∈ 𝐶 ∧ 𝑥𝐵𝐴)) |
|
Theorem | elima3 4932* |
Membership in an image. Theorem 34 of [Suppes]
p. 65. (Contributed by
NM, 14-Aug-1994.)
|
⊢ 𝐴 ∈ V ⇒ ⊢ (𝐴 ∈ (𝐵 “ 𝐶) ↔ ∃𝑥(𝑥 ∈ 𝐶 ∧ 〈𝑥, 𝐴〉 ∈ 𝐵)) |
|
Theorem | nfima 4933 |
Bound-variable hypothesis builder for image. (Contributed by NM,
30-Dec-1996.) (Proof shortened by Andrew Salmon, 27-Aug-2011.)
|
⊢ Ⅎ𝑥𝐴
& ⊢ Ⅎ𝑥𝐵 ⇒ ⊢ Ⅎ𝑥(𝐴 “ 𝐵) |
|
Theorem | nfimad 4934 |
Deduction version of bound-variable hypothesis builder nfima 4933.
(Contributed by FL, 15-Dec-2006.) (Revised by Mario Carneiro,
15-Oct-2016.)
|
⊢ (𝜑 → Ⅎ𝑥𝐴)
& ⊢ (𝜑 → Ⅎ𝑥𝐵) ⇒ ⊢ (𝜑 → Ⅎ𝑥(𝐴 “ 𝐵)) |
|
Theorem | imadmrn 4935 |
The image of the domain of a class is the range of the class.
(Contributed by NM, 14-Aug-1994.)
|
⊢ (𝐴 “ dom 𝐴) = ran 𝐴 |
|
Theorem | imassrn 4936 |
The image of a class is a subset of its range. Theorem 3.16(xi) of
[Monk1] p. 39. (Contributed by NM,
31-Mar-1995.)
|
⊢ (𝐴 “ 𝐵) ⊆ ran 𝐴 |
|
Theorem | imaexg 4937 |
The image of a set is a set. Theorem 3.17 of [Monk1] p. 39. (Contributed
by NM, 24-Jul-1995.)
|
⊢ (𝐴 ∈ 𝑉 → (𝐴 “ 𝐵) ∈ V) |
|
Theorem | imaex 4938 |
The image of a set is a set. Theorem 3.17 of [Monk1] p. 39.
(Contributed by JJ, 24-Sep-2021.)
|
⊢ 𝐴 ∈ V ⇒ ⊢ (𝐴 “ 𝐵) ∈ V |
|
Theorem | imai 4939 |
Image under the identity relation. Theorem 3.16(viii) of [Monk1] p. 38.
(Contributed by NM, 30-Apr-1998.)
|
⊢ ( I “ 𝐴) = 𝐴 |
|
Theorem | rnresi 4940 |
The range of the restricted identity function. (Contributed by NM,
27-Aug-2004.)
|
⊢ ran ( I ↾ 𝐴) = 𝐴 |
|
Theorem | resiima 4941 |
The image of a restriction of the identity function. (Contributed by FL,
31-Dec-2006.)
|
⊢ (𝐵 ⊆ 𝐴 → (( I ↾ 𝐴) “ 𝐵) = 𝐵) |
|
Theorem | ima0 4942 |
Image of the empty set. Theorem 3.16(ii) of [Monk1] p. 38. (Contributed
by NM, 20-May-1998.)
|
⊢ (𝐴 “ ∅) =
∅ |
|
Theorem | 0ima 4943 |
Image under the empty relation. (Contributed by FL, 11-Jan-2007.)
|
⊢ (∅ “ 𝐴) = ∅ |
|
Theorem | csbima12g 4944 |
Move class substitution in and out of the image of a function.
(Contributed by FL, 15-Dec-2006.) (Proof shortened by Mario Carneiro,
4-Dec-2016.)
|
⊢ (𝐴 ∈ 𝐶 → ⦋𝐴 / 𝑥⦌(𝐹 “ 𝐵) = (⦋𝐴 / 𝑥⦌𝐹 “ ⦋𝐴 / 𝑥⦌𝐵)) |
|
Theorem | imadisj 4945 |
A class whose image under another is empty is disjoint with the other's
domain. (Contributed by FL, 24-Jan-2007.)
|
⊢ ((𝐴 “ 𝐵) = ∅ ↔ (dom 𝐴 ∩ 𝐵) = ∅) |
|
Theorem | cnvimass 4946 |
A preimage under any class is included in the domain of the class.
(Contributed by FL, 29-Jan-2007.)
|
⊢ (◡𝐴 “ 𝐵) ⊆ dom 𝐴 |
|
Theorem | cnvimarndm 4947 |
The preimage of the range of a class is the domain of the class.
(Contributed by Jeff Hankins, 15-Jul-2009.)
|
⊢ (◡𝐴 “ ran 𝐴) = dom 𝐴 |
|
Theorem | imasng 4948* |
The image of a singleton. (Contributed by NM, 8-May-2005.)
|
⊢ (𝐴 ∈ 𝐵 → (𝑅 “ {𝐴}) = {𝑦 ∣ 𝐴𝑅𝑦}) |
|
Theorem | elreimasng 4949 |
Elementhood in the image of a singleton. (Contributed by Jim Kingdon,
10-Dec-2018.)
|
⊢ ((Rel 𝑅 ∧ 𝐴 ∈ 𝑉) → (𝐵 ∈ (𝑅 “ {𝐴}) ↔ 𝐴𝑅𝐵)) |
|
Theorem | elimasn 4950 |
Membership in an image of a singleton. (Contributed by NM,
15-Mar-2004.) (Proof shortened by Andrew Salmon, 27-Aug-2011.)
|
⊢ 𝐵 ∈ V & ⊢ 𝐶 ∈
V ⇒ ⊢ (𝐶 ∈ (𝐴 “ {𝐵}) ↔ 〈𝐵, 𝐶〉 ∈ 𝐴) |
|
Theorem | elimasng 4951 |
Membership in an image of a singleton. (Contributed by Raph Levien,
21-Oct-2006.)
|
⊢ ((𝐵 ∈ 𝑉 ∧ 𝐶 ∈ 𝑊) → (𝐶 ∈ (𝐴 “ {𝐵}) ↔ 〈𝐵, 𝐶〉 ∈ 𝐴)) |
|
Theorem | args 4952* |
Two ways to express the class of unique-valued arguments of 𝐹,
which is the same as the domain of 𝐹 whenever 𝐹 is a function.
The left-hand side of the equality is from Definition 10.2 of [Quine]
p. 65. Quine uses the notation "arg 𝐹 " for this class
(for which
we have no separate notation). (Contributed by NM, 8-May-2005.)
|
⊢ {𝑥 ∣ ∃𝑦(𝐹 “ {𝑥}) = {𝑦}} = {𝑥 ∣ ∃!𝑦 𝑥𝐹𝑦} |
|
Theorem | eliniseg 4953 |
Membership in an initial segment. The idiom (◡𝐴 “ {𝐵}),
meaning {𝑥 ∣ 𝑥𝐴𝐵}, is used to specify an initial
segment in
(for example) Definition 6.21 of [TakeutiZaring] p. 30. (Contributed by
NM, 28-Apr-2004.) (Proof shortened by Andrew Salmon, 27-Aug-2011.)
|
⊢ 𝐶 ∈ V ⇒ ⊢ (𝐵 ∈ 𝑉 → (𝐶 ∈ (◡𝐴 “ {𝐵}) ↔ 𝐶𝐴𝐵)) |
|
Theorem | epini 4954 |
Any set is equal to its preimage under the converse epsilon relation.
(Contributed by Mario Carneiro, 9-Mar-2013.)
|
⊢ 𝐴 ∈ V ⇒ ⊢ (◡ E “ {𝐴}) = 𝐴 |
|
Theorem | iniseg 4955* |
An idiom that signifies an initial segment of an ordering, used, for
example, in Definition 6.21 of [TakeutiZaring] p. 30. (Contributed by
NM, 28-Apr-2004.)
|
⊢ (𝐵 ∈ 𝑉 → (◡𝐴 “ {𝐵}) = {𝑥 ∣ 𝑥𝐴𝐵}) |
|
Theorem | dfse2 4956* |
Alternate definition of set-like relation. (Contributed by Mario
Carneiro, 23-Jun-2015.)
|
⊢ (𝑅 Se 𝐴 ↔ ∀𝑥 ∈ 𝐴 (𝐴 ∩ (◡𝑅 “ {𝑥})) ∈ V) |
|
Theorem | exse2 4957 |
Any set relation is set-like. (Contributed by Mario Carneiro,
22-Jun-2015.)
|
⊢ (𝑅 ∈ 𝑉 → 𝑅 Se 𝐴) |
|
Theorem | imass1 4958 |
Subset theorem for image. (Contributed by NM, 16-Mar-2004.)
|
⊢ (𝐴 ⊆ 𝐵 → (𝐴 “ 𝐶) ⊆ (𝐵 “ 𝐶)) |
|
Theorem | imass2 4959 |
Subset theorem for image. Exercise 22(a) of [Enderton] p. 53.
(Contributed by NM, 22-Mar-1998.)
|
⊢ (𝐴 ⊆ 𝐵 → (𝐶 “ 𝐴) ⊆ (𝐶 “ 𝐵)) |
|
Theorem | ndmima 4960 |
The image of a singleton outside the domain is empty. (Contributed by NM,
22-May-1998.)
|
⊢ (¬ 𝐴 ∈ dom 𝐵 → (𝐵 “ {𝐴}) = ∅) |
|
Theorem | relcnv 4961 |
A converse is a relation. Theorem 12 of [Suppes] p. 62. (Contributed
by NM, 29-Oct-1996.)
|
⊢ Rel ◡𝐴 |
|
Theorem | relbrcnvg 4962 |
When 𝑅 is a relation, the sethood
assumptions on brcnv 4766 can be
omitted. (Contributed by Mario Carneiro, 28-Apr-2015.)
|
⊢ (Rel 𝑅 → (𝐴◡𝑅𝐵 ↔ 𝐵𝑅𝐴)) |
|
Theorem | relbrcnv 4963 |
When 𝑅 is a relation, the sethood
assumptions on brcnv 4766 can be
omitted. (Contributed by Mario Carneiro, 28-Apr-2015.)
|
⊢ Rel 𝑅 ⇒ ⊢ (𝐴◡𝑅𝐵 ↔ 𝐵𝑅𝐴) |
|
Theorem | cotr 4964* |
Two ways of saying a relation is transitive. Definition of transitivity
in [Schechter] p. 51. (Contributed by
NM, 27-Dec-1996.) (Proof
shortened by Andrew Salmon, 27-Aug-2011.)
|
⊢ ((𝑅 ∘ 𝑅) ⊆ 𝑅 ↔ ∀𝑥∀𝑦∀𝑧((𝑥𝑅𝑦 ∧ 𝑦𝑅𝑧) → 𝑥𝑅𝑧)) |
|
Theorem | issref 4965* |
Two ways to state a relation is reflexive. Adapted from Tarski.
(Contributed by FL, 15-Jan-2012.) (Revised by NM, 30-Mar-2016.)
|
⊢ (( I ↾ 𝐴) ⊆ 𝑅 ↔ ∀𝑥 ∈ 𝐴 𝑥𝑅𝑥) |
|
Theorem | cnvsym 4966* |
Two ways of saying a relation is symmetric. Similar to definition of
symmetry in [Schechter] p. 51.
(Contributed by NM, 28-Dec-1996.)
(Proof shortened by Andrew Salmon, 27-Aug-2011.)
|
⊢ (◡𝑅 ⊆ 𝑅 ↔ ∀𝑥∀𝑦(𝑥𝑅𝑦 → 𝑦𝑅𝑥)) |
|
Theorem | intasym 4967* |
Two ways of saying a relation is antisymmetric. Definition of
antisymmetry in [Schechter] p. 51.
(Contributed by NM, 9-Sep-2004.)
(Proof shortened by Andrew Salmon, 27-Aug-2011.)
|
⊢ ((𝑅 ∩ ◡𝑅) ⊆ I ↔ ∀𝑥∀𝑦((𝑥𝑅𝑦 ∧ 𝑦𝑅𝑥) → 𝑥 = 𝑦)) |
|
Theorem | asymref 4968* |
Two ways of saying a relation is antisymmetric and reflexive.
∪ ∪ 𝑅 is the field of a relation by relfld 5111. (Contributed by
NM, 6-May-2008.) (Proof shortened by Andrew Salmon, 27-Aug-2011.)
|
⊢ ((𝑅 ∩ ◡𝑅) = ( I ↾ ∪ ∪ 𝑅) ↔ ∀𝑥 ∈ ∪ ∪ 𝑅∀𝑦((𝑥𝑅𝑦 ∧ 𝑦𝑅𝑥) ↔ 𝑥 = 𝑦)) |
|
Theorem | intirr 4969* |
Two ways of saying a relation is irreflexive. Definition of
irreflexivity in [Schechter] p. 51.
(Contributed by NM, 9-Sep-2004.)
(Proof shortened by Andrew Salmon, 27-Aug-2011.)
|
⊢ ((𝑅 ∩ I ) = ∅ ↔ ∀𝑥 ¬ 𝑥𝑅𝑥) |
|
Theorem | brcodir 4970* |
Two ways of saying that two elements have an upper bound. (Contributed
by Mario Carneiro, 3-Nov-2015.)
|
⊢ ((𝐴 ∈ 𝑉 ∧ 𝐵 ∈ 𝑊) → (𝐴(◡𝑅 ∘ 𝑅)𝐵 ↔ ∃𝑧(𝐴𝑅𝑧 ∧ 𝐵𝑅𝑧))) |
|
Theorem | codir 4971* |
Two ways of saying a relation is directed. (Contributed by Mario
Carneiro, 22-Nov-2013.)
|
⊢ ((𝐴 × 𝐵) ⊆ (◡𝑅 ∘ 𝑅) ↔ ∀𝑥 ∈ 𝐴 ∀𝑦 ∈ 𝐵 ∃𝑧(𝑥𝑅𝑧 ∧ 𝑦𝑅𝑧)) |
|
Theorem | qfto 4972* |
A quantifier-free way of expressing the total order predicate.
(Contributed by Mario Carneiro, 22-Nov-2013.)
|
⊢ ((𝐴 × 𝐵) ⊆ (𝑅 ∪ ◡𝑅) ↔ ∀𝑥 ∈ 𝐴 ∀𝑦 ∈ 𝐵 (𝑥𝑅𝑦 ∨ 𝑦𝑅𝑥)) |
|
Theorem | xpidtr 4973 |
A square cross product (𝐴 × 𝐴) is a transitive relation.
(Contributed by FL, 31-Jul-2009.)
|
⊢ ((𝐴 × 𝐴) ∘ (𝐴 × 𝐴)) ⊆ (𝐴 × 𝐴) |
|
Theorem | trin2 4974 |
The intersection of two transitive classes is transitive. (Contributed
by FL, 31-Jul-2009.)
|
⊢ (((𝑅 ∘ 𝑅) ⊆ 𝑅 ∧ (𝑆 ∘ 𝑆) ⊆ 𝑆) → ((𝑅 ∩ 𝑆) ∘ (𝑅 ∩ 𝑆)) ⊆ (𝑅 ∩ 𝑆)) |
|
Theorem | poirr2 4975 |
A partial order relation is irreflexive. (Contributed by Mario
Carneiro, 2-Nov-2015.)
|
⊢ (𝑅 Po 𝐴 → (𝑅 ∩ ( I ↾ 𝐴)) = ∅) |
|
Theorem | trinxp 4976 |
The relation induced by a transitive relation on a part of its field is
transitive. (Taking the intersection of a relation with a square cross
product is a way to restrict it to a subset of its field.) (Contributed
by FL, 31-Jul-2009.)
|
⊢ ((𝑅 ∘ 𝑅) ⊆ 𝑅 → ((𝑅 ∩ (𝐴 × 𝐴)) ∘ (𝑅 ∩ (𝐴 × 𝐴))) ⊆ (𝑅 ∩ (𝐴 × 𝐴))) |
|
Theorem | soirri 4977 |
A strict order relation is irreflexive. (Contributed by NM,
10-Feb-1996.) (Revised by Mario Carneiro, 10-May-2013.)
|
⊢ 𝑅 Or 𝑆
& ⊢ 𝑅 ⊆ (𝑆 × 𝑆) ⇒ ⊢ ¬ 𝐴𝑅𝐴 |
|
Theorem | sotri 4978 |
A strict order relation is a transitive relation. (Contributed by NM,
10-Feb-1996.) (Revised by Mario Carneiro, 10-May-2013.)
|
⊢ 𝑅 Or 𝑆
& ⊢ 𝑅 ⊆ (𝑆 × 𝑆) ⇒ ⊢ ((𝐴𝑅𝐵 ∧ 𝐵𝑅𝐶) → 𝐴𝑅𝐶) |
|
Theorem | son2lpi 4979 |
A strict order relation has no 2-cycle loops. (Contributed by NM,
10-Feb-1996.) (Revised by Mario Carneiro, 10-May-2013.)
|
⊢ 𝑅 Or 𝑆
& ⊢ 𝑅 ⊆ (𝑆 × 𝑆) ⇒ ⊢ ¬ (𝐴𝑅𝐵 ∧ 𝐵𝑅𝐴) |
|
Theorem | sotri2 4980 |
A transitivity relation. (Read ¬ B < A and B
< C implies A < C .)
(Contributed by Mario Carneiro, 10-May-2013.)
|
⊢ 𝑅 Or 𝑆
& ⊢ 𝑅 ⊆ (𝑆 × 𝑆) ⇒ ⊢ ((𝐴 ∈ 𝑆 ∧ ¬ 𝐵𝑅𝐴 ∧ 𝐵𝑅𝐶) → 𝐴𝑅𝐶) |
|
Theorem | sotri3 4981 |
A transitivity relation. (Read A < B and ¬ C
< B implies A < C .)
(Contributed by Mario Carneiro, 10-May-2013.)
|
⊢ 𝑅 Or 𝑆
& ⊢ 𝑅 ⊆ (𝑆 × 𝑆) ⇒ ⊢ ((𝐶 ∈ 𝑆 ∧ 𝐴𝑅𝐵 ∧ ¬ 𝐶𝑅𝐵) → 𝐴𝑅𝐶) |
|
Theorem | poleloe 4982 |
Express "less than or equals" for general strict orders.
(Contributed by
Stefan O'Rear, 17-Jan-2015.)
|
⊢ (𝐵 ∈ 𝑉 → (𝐴(𝑅 ∪ I )𝐵 ↔ (𝐴𝑅𝐵 ∨ 𝐴 = 𝐵))) |
|
Theorem | poltletr 4983 |
Transitive law for general strict orders. (Contributed by Stefan O'Rear,
17-Jan-2015.)
|
⊢ ((𝑅 Po 𝑋 ∧ (𝐴 ∈ 𝑋 ∧ 𝐵 ∈ 𝑋 ∧ 𝐶 ∈ 𝑋)) → ((𝐴𝑅𝐵 ∧ 𝐵(𝑅 ∪ I )𝐶) → 𝐴𝑅𝐶)) |
|
Theorem | cnvopab 4984* |
The converse of a class abstraction of ordered pairs. (Contributed by
NM, 11-Dec-2003.) (Proof shortened by Andrew Salmon, 27-Aug-2011.)
|
⊢ ◡{〈𝑥, 𝑦〉 ∣ 𝜑} = {〈𝑦, 𝑥〉 ∣ 𝜑} |
|
Theorem | mptcnv 4985* |
The converse of a mapping function. (Contributed by Thierry Arnoux,
16-Jan-2017.)
|
⊢ (𝜑 → ((𝑥 ∈ 𝐴 ∧ 𝑦 = 𝐵) ↔ (𝑦 ∈ 𝐶 ∧ 𝑥 = 𝐷))) ⇒ ⊢ (𝜑 → ◡(𝑥 ∈ 𝐴 ↦ 𝐵) = (𝑦 ∈ 𝐶 ↦ 𝐷)) |
|
Theorem | cnv0 4986 |
The converse of the empty set. (Contributed by NM, 6-Apr-1998.)
|
⊢ ◡∅ = ∅ |
|
Theorem | cnvi 4987 |
The converse of the identity relation. Theorem 3.7(ii) of [Monk1]
p. 36. (Contributed by NM, 26-Apr-1998.) (Proof shortened by Andrew
Salmon, 27-Aug-2011.)
|
⊢ ◡ I
= I |
|
Theorem | cnvun 4988 |
The converse of a union is the union of converses. Theorem 16 of
[Suppes] p. 62. (Contributed by NM,
25-Mar-1998.) (Proof shortened by
Andrew Salmon, 27-Aug-2011.)
|
⊢ ◡(𝐴 ∪ 𝐵) = (◡𝐴 ∪ ◡𝐵) |
|
Theorem | cnvdif 4989 |
Distributive law for converse over set difference. (Contributed by
Mario Carneiro, 26-Jun-2014.)
|
⊢ ◡(𝐴 ∖ 𝐵) = (◡𝐴 ∖ ◡𝐵) |
|
Theorem | cnvin 4990 |
Distributive law for converse over intersection. Theorem 15 of [Suppes]
p. 62. (Contributed by NM, 25-Mar-1998.) (Revised by Mario Carneiro,
26-Jun-2014.)
|
⊢ ◡(𝐴 ∩ 𝐵) = (◡𝐴 ∩ ◡𝐵) |
|
Theorem | rnun 4991 |
Distributive law for range over union. Theorem 8 of [Suppes] p. 60.
(Contributed by NM, 24-Mar-1998.)
|
⊢ ran (𝐴 ∪ 𝐵) = (ran 𝐴 ∪ ran 𝐵) |
|
Theorem | rnin 4992 |
The range of an intersection belongs the intersection of ranges. Theorem
9 of [Suppes] p. 60. (Contributed by NM,
15-Sep-2004.)
|
⊢ ran (𝐴 ∩ 𝐵) ⊆ (ran 𝐴 ∩ ran 𝐵) |
|
Theorem | rniun 4993 |
The range of an indexed union. (Contributed by Mario Carneiro,
29-May-2015.)
|
⊢ ran ∪
𝑥 ∈ 𝐴 𝐵 = ∪
𝑥 ∈ 𝐴 ran 𝐵 |
|
Theorem | rnuni 4994* |
The range of a union. Part of Exercise 8 of [Enderton] p. 41.
(Contributed by NM, 17-Mar-2004.) (Revised by Mario Carneiro,
29-May-2015.)
|
⊢ ran ∪ 𝐴 = ∪ 𝑥 ∈ 𝐴 ran 𝑥 |
|
Theorem | imaundi 4995 |
Distributive law for image over union. Theorem 35 of [Suppes] p. 65.
(Contributed by NM, 30-Sep-2002.)
|
⊢ (𝐴 “ (𝐵 ∪ 𝐶)) = ((𝐴 “ 𝐵) ∪ (𝐴 “ 𝐶)) |
|
Theorem | imaundir 4996 |
The image of a union. (Contributed by Jeff Hoffman, 17-Feb-2008.)
|
⊢ ((𝐴 ∪ 𝐵) “ 𝐶) = ((𝐴 “ 𝐶) ∪ (𝐵 “ 𝐶)) |
|
Theorem | dminss 4997 |
An upper bound for intersection with a domain. Theorem 40 of [Suppes]
p. 66, who calls it "somewhat surprising." (Contributed by
NM,
11-Aug-2004.)
|
⊢ (dom 𝑅 ∩ 𝐴) ⊆ (◡𝑅 “ (𝑅 “ 𝐴)) |
|
Theorem | imainss 4998 |
An upper bound for intersection with an image. Theorem 41 of [Suppes]
p. 66. (Contributed by NM, 11-Aug-2004.)
|
⊢ ((𝑅 “ 𝐴) ∩ 𝐵) ⊆ (𝑅 “ (𝐴 ∩ (◡𝑅 “ 𝐵))) |
|
Theorem | inimass 4999 |
The image of an intersection (Contributed by Thierry Arnoux,
16-Dec-2017.)
|
⊢ ((𝐴 ∩ 𝐵) “ 𝐶) ⊆ ((𝐴 “ 𝐶) ∩ (𝐵 “ 𝐶)) |
|
Theorem | inimasn 5000 |
The intersection of the image of singleton (Contributed by Thierry
Arnoux, 16-Dec-2017.)
|
⊢ (𝐶 ∈ 𝑉 → ((𝐴 ∩ 𝐵) “ {𝐶}) = ((𝐴 “ {𝐶}) ∩ (𝐵 “ {𝐶}))) |