Theorem List for Intuitionistic Logic Explorer - 9801-9900 *Has distinct variable
group(s)
Type | Label | Description |
Statement |
|
Theorem | rexneg 9801 |
Minus a real number. Remark [BourbakiTop1] p. IV.15. (Contributed by
FL, 26-Dec-2011.) (Proof shortened by Mario Carneiro, 20-Aug-2015.)
|
⊢ (𝐴 ∈ ℝ →
-𝑒𝐴 =
-𝐴) |
|
Theorem | xneg0 9802 |
The negative of zero. (Contributed by Mario Carneiro, 20-Aug-2015.)
|
⊢ -𝑒0 = 0 |
|
Theorem | xnegcl 9803 |
Closure of extended real negative. (Contributed by Mario Carneiro,
20-Aug-2015.)
|
⊢ (𝐴 ∈ ℝ* →
-𝑒𝐴
∈ ℝ*) |
|
Theorem | xnegneg 9804 |
Extended real version of negneg 8181. (Contributed by Mario Carneiro,
20-Aug-2015.)
|
⊢ (𝐴 ∈ ℝ* →
-𝑒-𝑒𝐴 = 𝐴) |
|
Theorem | xneg11 9805 |
Extended real version of neg11 8182. (Contributed by Mario Carneiro,
20-Aug-2015.)
|
⊢ ((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*)
→ (-𝑒𝐴 = -𝑒𝐵 ↔ 𝐴 = 𝐵)) |
|
Theorem | xltnegi 9806 |
Forward direction of xltneg 9807. (Contributed by Mario Carneiro,
20-Aug-2015.)
|
⊢ ((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*
∧ 𝐴 < 𝐵) →
-𝑒𝐵
< -𝑒𝐴) |
|
Theorem | xltneg 9807 |
Extended real version of ltneg 8393. (Contributed by Mario Carneiro,
20-Aug-2015.)
|
⊢ ((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*)
→ (𝐴 < 𝐵 ↔
-𝑒𝐵
< -𝑒𝐴)) |
|
Theorem | xleneg 9808 |
Extended real version of leneg 8396. (Contributed by Mario Carneiro,
20-Aug-2015.)
|
⊢ ((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*)
→ (𝐴 ≤ 𝐵 ↔
-𝑒𝐵
≤ -𝑒𝐴)) |
|
Theorem | xlt0neg1 9809 |
Extended real version of lt0neg1 8399. (Contributed by Mario Carneiro,
20-Aug-2015.)
|
⊢ (𝐴 ∈ ℝ* → (𝐴 < 0 ↔ 0 <
-𝑒𝐴)) |
|
Theorem | xlt0neg2 9810 |
Extended real version of lt0neg2 8400. (Contributed by Mario Carneiro,
20-Aug-2015.)
|
⊢ (𝐴 ∈ ℝ* → (0 <
𝐴 ↔
-𝑒𝐴
< 0)) |
|
Theorem | xle0neg1 9811 |
Extended real version of le0neg1 8401. (Contributed by Mario Carneiro,
9-Sep-2015.)
|
⊢ (𝐴 ∈ ℝ* → (𝐴 ≤ 0 ↔ 0 ≤
-𝑒𝐴)) |
|
Theorem | xle0neg2 9812 |
Extended real version of le0neg2 8402. (Contributed by Mario Carneiro,
9-Sep-2015.)
|
⊢ (𝐴 ∈ ℝ* → (0 ≤
𝐴 ↔
-𝑒𝐴
≤ 0)) |
|
Theorem | xrpnfdc 9813 |
An extended real is or is not plus infinity. (Contributed by Jim Kingdon,
13-Apr-2023.)
|
⊢ (𝐴 ∈ ℝ* →
DECID 𝐴 =
+∞) |
|
Theorem | xrmnfdc 9814 |
An extended real is or is not minus infinity. (Contributed by Jim
Kingdon, 13-Apr-2023.)
|
⊢ (𝐴 ∈ ℝ* →
DECID 𝐴 =
-∞) |
|
Theorem | xaddf 9815 |
The extended real addition operation is closed in extended reals.
(Contributed by Mario Carneiro, 21-Aug-2015.)
|
⊢ +𝑒 :(ℝ*
× ℝ*)⟶ℝ* |
|
Theorem | xaddval 9816 |
Value of the extended real addition operation. (Contributed by Mario
Carneiro, 20-Aug-2015.)
|
⊢ ((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*)
→ (𝐴
+𝑒 𝐵) =
if(𝐴 = +∞, if(𝐵 = -∞, 0, +∞),
if(𝐴 = -∞, if(𝐵 = +∞, 0, -∞),
if(𝐵 = +∞, +∞,
if(𝐵 = -∞, -∞,
(𝐴 + 𝐵)))))) |
|
Theorem | xaddpnf1 9817 |
Addition of positive infinity on the right. (Contributed by Mario
Carneiro, 20-Aug-2015.)
|
⊢ ((𝐴 ∈ ℝ* ∧ 𝐴 ≠ -∞) → (𝐴 +𝑒
+∞) = +∞) |
|
Theorem | xaddpnf2 9818 |
Addition of positive infinity on the left. (Contributed by Mario
Carneiro, 20-Aug-2015.)
|
⊢ ((𝐴 ∈ ℝ* ∧ 𝐴 ≠ -∞) →
(+∞ +𝑒 𝐴) = +∞) |
|
Theorem | xaddmnf1 9819 |
Addition of negative infinity on the right. (Contributed by Mario
Carneiro, 20-Aug-2015.)
|
⊢ ((𝐴 ∈ ℝ* ∧ 𝐴 ≠ +∞) → (𝐴 +𝑒
-∞) = -∞) |
|
Theorem | xaddmnf2 9820 |
Addition of negative infinity on the left. (Contributed by Mario
Carneiro, 20-Aug-2015.)
|
⊢ ((𝐴 ∈ ℝ* ∧ 𝐴 ≠ +∞) →
(-∞ +𝑒 𝐴) = -∞) |
|
Theorem | pnfaddmnf 9821 |
Addition of positive and negative infinity. This is often taken to be a
"null" value or out of the domain, but we define it (somewhat
arbitrarily)
to be zero so that the resulting function is total, which simplifies
proofs. (Contributed by Mario Carneiro, 20-Aug-2015.)
|
⊢ (+∞ +𝑒 -∞) =
0 |
|
Theorem | mnfaddpnf 9822 |
Addition of negative and positive infinity. This is often taken to be a
"null" value or out of the domain, but we define it (somewhat
arbitrarily)
to be zero so that the resulting function is total, which simplifies
proofs. (Contributed by Mario Carneiro, 20-Aug-2015.)
|
⊢ (-∞ +𝑒 +∞) =
0 |
|
Theorem | rexadd 9823 |
The extended real addition operation when both arguments are real.
(Contributed by Mario Carneiro, 20-Aug-2015.)
|
⊢ ((𝐴 ∈ ℝ ∧ 𝐵 ∈ ℝ) → (𝐴 +𝑒 𝐵) = (𝐴 + 𝐵)) |
|
Theorem | rexsub 9824 |
Extended real subtraction when both arguments are real. (Contributed by
Mario Carneiro, 23-Aug-2015.)
|
⊢ ((𝐴 ∈ ℝ ∧ 𝐵 ∈ ℝ) → (𝐴 +𝑒
-𝑒𝐵) =
(𝐴 − 𝐵)) |
|
Theorem | rexaddd 9825 |
The extended real addition operation when both arguments are real.
Deduction version of rexadd 9823. (Contributed by Glauco Siliprandi,
24-Dec-2020.)
|
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ)
⇒ ⊢ (𝜑 → (𝐴 +𝑒 𝐵) = (𝐴 + 𝐵)) |
|
Theorem | xnegcld 9826 |
Closure of extended real negative. (Contributed by Mario Carneiro,
28-May-2016.)
|
⊢ (𝜑 → 𝐴 ∈
ℝ*) ⇒ ⊢ (𝜑 → -𝑒𝐴 ∈
ℝ*) |
|
Theorem | xrex 9827 |
The set of extended reals exists. (Contributed by NM, 24-Dec-2006.)
|
⊢ ℝ* ∈
V |
|
Theorem | xaddnemnf 9828 |
Closure of extended real addition in the subset ℝ* / {-∞}.
(Contributed by Mario Carneiro, 20-Aug-2015.)
|
⊢ (((𝐴 ∈ ℝ* ∧ 𝐴 ≠ -∞) ∧ (𝐵 ∈ ℝ*
∧ 𝐵 ≠ -∞))
→ (𝐴
+𝑒 𝐵)
≠ -∞) |
|
Theorem | xaddnepnf 9829 |
Closure of extended real addition in the subset ℝ* / {+∞}.
(Contributed by Mario Carneiro, 20-Aug-2015.)
|
⊢ (((𝐴 ∈ ℝ* ∧ 𝐴 ≠ +∞) ∧ (𝐵 ∈ ℝ*
∧ 𝐵 ≠ +∞))
→ (𝐴
+𝑒 𝐵)
≠ +∞) |
|
Theorem | xnegid 9830 |
Extended real version of negid 8178. (Contributed by Mario Carneiro,
20-Aug-2015.)
|
⊢ (𝐴 ∈ ℝ* → (𝐴 +𝑒
-𝑒𝐴) =
0) |
|
Theorem | xaddcl 9831 |
The extended real addition operation is closed in extended reals.
(Contributed by Mario Carneiro, 20-Aug-2015.)
|
⊢ ((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*)
→ (𝐴
+𝑒 𝐵)
∈ ℝ*) |
|
Theorem | xaddcom 9832 |
The extended real addition operation is commutative. (Contributed by NM,
26-Dec-2011.)
|
⊢ ((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*)
→ (𝐴
+𝑒 𝐵) =
(𝐵 +𝑒
𝐴)) |
|
Theorem | xaddid1 9833 |
Extended real version of addid1 8069. (Contributed by Mario Carneiro,
20-Aug-2015.)
|
⊢ (𝐴 ∈ ℝ* → (𝐴 +𝑒 0) =
𝐴) |
|
Theorem | xaddid2 9834 |
Extended real version of addid2 8070. (Contributed by Mario Carneiro,
20-Aug-2015.)
|
⊢ (𝐴 ∈ ℝ* → (0
+𝑒 𝐴) =
𝐴) |
|
Theorem | xaddid1d 9835 |
0 is a right identity for extended real addition.
(Contributed by
Glauco Siliprandi, 17-Aug-2020.)
|
⊢ (𝜑 → 𝐴 ∈
ℝ*) ⇒ ⊢ (𝜑 → (𝐴 +𝑒 0) = 𝐴) |
|
Theorem | xnn0lenn0nn0 9836 |
An extended nonnegative integer which is less than or equal to a
nonnegative integer is a nonnegative integer. (Contributed by AV,
24-Nov-2021.)
|
⊢ ((𝑀 ∈ ℕ0*
∧ 𝑁 ∈
ℕ0 ∧ 𝑀 ≤ 𝑁) → 𝑀 ∈
ℕ0) |
|
Theorem | xnn0le2is012 9837 |
An extended nonnegative integer which is less than or equal to 2 is either
0 or 1 or 2. (Contributed by AV, 24-Nov-2021.)
|
⊢ ((𝑁 ∈ ℕ0*
∧ 𝑁 ≤ 2) →
(𝑁 = 0 ∨ 𝑁 = 1 ∨ 𝑁 = 2)) |
|
Theorem | xnn0xadd0 9838 |
The sum of two extended nonnegative integers is 0 iff
each of the two
extended nonnegative integers is 0. (Contributed
by AV,
14-Dec-2020.)
|
⊢ ((𝐴 ∈ ℕ0*
∧ 𝐵 ∈
ℕ0*) → ((𝐴 +𝑒 𝐵) = 0 ↔ (𝐴 = 0 ∧ 𝐵 = 0))) |
|
Theorem | xnegdi 9839 |
Extended real version of negdi 8188. (Contributed by Mario Carneiro,
20-Aug-2015.)
|
⊢ ((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*)
→ -𝑒(𝐴 +𝑒 𝐵) = (-𝑒𝐴 +𝑒
-𝑒𝐵)) |
|
Theorem | xaddass 9840 |
Associativity of extended real addition. The correct condition here is
"it is not the case that both +∞ and
-∞ appear as one of
𝐴,
𝐵, 𝐶, i.e. ¬
{+∞, -∞} ⊆ {𝐴, 𝐵, 𝐶}", but this
condition is difficult to work with, so we break the theorem into two
parts: this one, where -∞ is not present in
𝐴, 𝐵, 𝐶, and
xaddass2 9841, where +∞ is
not present. (Contributed by Mario
Carneiro, 20-Aug-2015.)
|
⊢ (((𝐴 ∈ ℝ* ∧ 𝐴 ≠ -∞) ∧ (𝐵 ∈ ℝ*
∧ 𝐵 ≠ -∞)
∧ (𝐶 ∈
ℝ* ∧ 𝐶 ≠ -∞)) → ((𝐴 +𝑒 𝐵) +𝑒 𝐶) = (𝐴 +𝑒 (𝐵 +𝑒 𝐶))) |
|
Theorem | xaddass2 9841 |
Associativity of extended real addition. See xaddass 9840 for notes on the
hypotheses. (Contributed by Mario Carneiro, 20-Aug-2015.)
|
⊢ (((𝐴 ∈ ℝ* ∧ 𝐴 ≠ +∞) ∧ (𝐵 ∈ ℝ*
∧ 𝐵 ≠ +∞)
∧ (𝐶 ∈
ℝ* ∧ 𝐶 ≠ +∞)) → ((𝐴 +𝑒 𝐵) +𝑒 𝐶) = (𝐴 +𝑒 (𝐵 +𝑒 𝐶))) |
|
Theorem | xpncan 9842 |
Extended real version of pncan 8137. (Contributed by Mario Carneiro,
20-Aug-2015.)
|
⊢ ((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ) → ((𝐴 +𝑒 𝐵) +𝑒
-𝑒𝐵) =
𝐴) |
|
Theorem | xnpcan 9843 |
Extended real version of npcan 8140. (Contributed by Mario Carneiro,
20-Aug-2015.)
|
⊢ ((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ) → ((𝐴 +𝑒
-𝑒𝐵)
+𝑒 𝐵) =
𝐴) |
|
Theorem | xleadd1a 9844 |
Extended real version of leadd1 8361; note that the converse implication is
not true, unlike the real version (for example 0 <
1 but
(1 +𝑒 +∞) ≤ (0
+𝑒 +∞)). (Contributed by Mario Carneiro,
20-Aug-2015.)
|
⊢ (((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*
∧ 𝐶 ∈
ℝ*) ∧ 𝐴 ≤ 𝐵) → (𝐴 +𝑒 𝐶) ≤ (𝐵 +𝑒 𝐶)) |
|
Theorem | xleadd2a 9845 |
Commuted form of xleadd1a 9844. (Contributed by Mario Carneiro,
20-Aug-2015.)
|
⊢ (((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*
∧ 𝐶 ∈
ℝ*) ∧ 𝐴 ≤ 𝐵) → (𝐶 +𝑒 𝐴) ≤ (𝐶 +𝑒 𝐵)) |
|
Theorem | xleadd1 9846 |
Weakened version of xleadd1a 9844 under which the reverse implication is
true. (Contributed by Mario Carneiro, 20-Aug-2015.)
|
⊢ ((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*
∧ 𝐶 ∈ ℝ)
→ (𝐴 ≤ 𝐵 ↔ (𝐴 +𝑒 𝐶) ≤ (𝐵 +𝑒 𝐶))) |
|
Theorem | xltadd1 9847 |
Extended real version of ltadd1 8360. (Contributed by Mario Carneiro,
23-Aug-2015.) (Revised by Jim Kingdon, 16-Apr-2023.)
|
⊢ ((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*
∧ 𝐶 ∈ ℝ)
→ (𝐴 < 𝐵 ↔ (𝐴 +𝑒 𝐶) < (𝐵 +𝑒 𝐶))) |
|
Theorem | xltadd2 9848 |
Extended real version of ltadd2 8350. (Contributed by Mario Carneiro,
23-Aug-2015.)
|
⊢ ((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*
∧ 𝐶 ∈ ℝ)
→ (𝐴 < 𝐵 ↔ (𝐶 +𝑒 𝐴) < (𝐶 +𝑒 𝐵))) |
|
Theorem | xaddge0 9849 |
The sum of nonnegative extended reals is nonnegative. (Contributed by
Mario Carneiro, 21-Aug-2015.)
|
⊢ (((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*)
∧ (0 ≤ 𝐴 ∧ 0
≤ 𝐵)) → 0 ≤
(𝐴 +𝑒
𝐵)) |
|
Theorem | xle2add 9850 |
Extended real version of le2add 8375. (Contributed by Mario Carneiro,
23-Aug-2015.)
|
⊢ (((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*)
∧ (𝐶 ∈
ℝ* ∧ 𝐷 ∈ ℝ*)) →
((𝐴 ≤ 𝐶 ∧ 𝐵 ≤ 𝐷) → (𝐴 +𝑒 𝐵) ≤ (𝐶 +𝑒 𝐷))) |
|
Theorem | xlt2add 9851 |
Extended real version of lt2add 8376. Note that ltleadd 8377, which has
weaker assumptions, is not true for the extended reals (since
0 + +∞ < 1 + +∞ fails).
(Contributed by Mario Carneiro,
23-Aug-2015.)
|
⊢ (((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*)
∧ (𝐶 ∈
ℝ* ∧ 𝐷 ∈ ℝ*)) →
((𝐴 < 𝐶 ∧ 𝐵 < 𝐷) → (𝐴 +𝑒 𝐵) < (𝐶 +𝑒 𝐷))) |
|
Theorem | xsubge0 9852 |
Extended real version of subge0 8406. (Contributed by Mario Carneiro,
24-Aug-2015.)
|
⊢ ((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*)
→ (0 ≤ (𝐴
+𝑒 -𝑒𝐵) ↔ 𝐵 ≤ 𝐴)) |
|
Theorem | xposdif 9853 |
Extended real version of posdif 8386. (Contributed by Mario Carneiro,
24-Aug-2015.) (Revised by Jim Kingdon, 17-Apr-2023.)
|
⊢ ((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*)
→ (𝐴 < 𝐵 ↔ 0 < (𝐵 +𝑒
-𝑒𝐴))) |
|
Theorem | xlesubadd 9854 |
Under certain conditions, the conclusion of lesubadd 8365 is true even in the
extended reals. (Contributed by Mario Carneiro, 4-Sep-2015.)
|
⊢ (((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*
∧ 𝐶 ∈
ℝ*) ∧ (0 ≤ 𝐴 ∧ 𝐵 ≠ -∞ ∧ 0 ≤ 𝐶)) → ((𝐴 +𝑒
-𝑒𝐵)
≤ 𝐶 ↔ 𝐴 ≤ (𝐶 +𝑒 𝐵))) |
|
Theorem | xaddcld 9855 |
The extended real addition operation is closed in extended reals.
(Contributed by Mario Carneiro, 28-May-2016.)
|
⊢ (𝜑 → 𝐴 ∈ ℝ*) & ⊢ (𝜑 → 𝐵 ∈
ℝ*) ⇒ ⊢ (𝜑 → (𝐴 +𝑒 𝐵) ∈
ℝ*) |
|
Theorem | xadd4d 9856 |
Rearrangement of 4 terms in a sum for extended addition, analogous to
add4d 8100. (Contributed by Alexander van der Vekens,
21-Dec-2017.)
|
⊢ (𝜑 → (𝐴 ∈ ℝ* ∧ 𝐴 ≠ -∞)) & ⊢ (𝜑 → (𝐵 ∈ ℝ* ∧ 𝐵 ≠ -∞)) & ⊢ (𝜑 → (𝐶 ∈ ℝ* ∧ 𝐶 ≠ -∞)) & ⊢ (𝜑 → (𝐷 ∈ ℝ* ∧ 𝐷 ≠
-∞)) ⇒ ⊢ (𝜑 → ((𝐴 +𝑒 𝐵) +𝑒 (𝐶 +𝑒 𝐷)) = ((𝐴 +𝑒 𝐶) +𝑒 (𝐵 +𝑒 𝐷))) |
|
Theorem | xnn0add4d 9857 |
Rearrangement of 4 terms in a sum for extended addition of extended
nonnegative integers, analogous to xadd4d 9856. (Contributed by AV,
12-Dec-2020.)
|
⊢ (𝜑 → 𝐴 ∈
ℕ0*)
& ⊢ (𝜑 → 𝐵 ∈
ℕ0*)
& ⊢ (𝜑 → 𝐶 ∈
ℕ0*)
& ⊢ (𝜑 → 𝐷 ∈
ℕ0*) ⇒ ⊢ (𝜑 → ((𝐴 +𝑒 𝐵) +𝑒 (𝐶 +𝑒 𝐷)) = ((𝐴 +𝑒 𝐶) +𝑒 (𝐵 +𝑒 𝐷))) |
|
Theorem | xleaddadd 9858 |
Cancelling a factor of two in ≤ (expressed as
addition rather than
as a factor to avoid extended real multiplication). (Contributed by Jim
Kingdon, 18-Apr-2023.)
|
⊢ ((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*)
→ (𝐴 ≤ 𝐵 ↔ (𝐴 +𝑒 𝐴) ≤ (𝐵 +𝑒 𝐵))) |
|
4.5.3 Real number intervals
|
|
Syntax | cioo 9859 |
Extend class notation with the set of open intervals of extended reals.
|
class (,) |
|
Syntax | cioc 9860 |
Extend class notation with the set of open-below, closed-above intervals
of extended reals.
|
class (,] |
|
Syntax | cico 9861 |
Extend class notation with the set of closed-below, open-above intervals
of extended reals.
|
class [,) |
|
Syntax | cicc 9862 |
Extend class notation with the set of closed intervals of extended
reals.
|
class [,] |
|
Definition | df-ioo 9863* |
Define the set of open intervals of extended reals. (Contributed by NM,
24-Dec-2006.)
|
⊢ (,) = (𝑥 ∈ ℝ*, 𝑦 ∈ ℝ*
↦ {𝑧 ∈
ℝ* ∣ (𝑥 < 𝑧 ∧ 𝑧 < 𝑦)}) |
|
Definition | df-ioc 9864* |
Define the set of open-below, closed-above intervals of extended reals.
(Contributed by NM, 24-Dec-2006.)
|
⊢ (,] = (𝑥 ∈ ℝ*, 𝑦 ∈ ℝ*
↦ {𝑧 ∈
ℝ* ∣ (𝑥 < 𝑧 ∧ 𝑧 ≤ 𝑦)}) |
|
Definition | df-ico 9865* |
Define the set of closed-below, open-above intervals of extended reals.
(Contributed by NM, 24-Dec-2006.)
|
⊢ [,) = (𝑥 ∈ ℝ*, 𝑦 ∈ ℝ*
↦ {𝑧 ∈
ℝ* ∣ (𝑥 ≤ 𝑧 ∧ 𝑧 < 𝑦)}) |
|
Definition | df-icc 9866* |
Define the set of closed intervals of extended reals. (Contributed by
NM, 24-Dec-2006.)
|
⊢ [,] = (𝑥 ∈ ℝ*, 𝑦 ∈ ℝ*
↦ {𝑧 ∈
ℝ* ∣ (𝑥 ≤ 𝑧 ∧ 𝑧 ≤ 𝑦)}) |
|
Theorem | ixxval 9867* |
Value of the interval function. (Contributed by Mario Carneiro,
3-Nov-2013.)
|
⊢ 𝑂 = (𝑥 ∈ ℝ*, 𝑦 ∈ ℝ*
↦ {𝑧 ∈
ℝ* ∣ (𝑥𝑅𝑧 ∧ 𝑧𝑆𝑦)}) ⇒ ⊢ ((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*)
→ (𝐴𝑂𝐵) = {𝑧 ∈ ℝ* ∣ (𝐴𝑅𝑧 ∧ 𝑧𝑆𝐵)}) |
|
Theorem | elixx1 9868* |
Membership in an interval of extended reals. (Contributed by Mario
Carneiro, 3-Nov-2013.)
|
⊢ 𝑂 = (𝑥 ∈ ℝ*, 𝑦 ∈ ℝ*
↦ {𝑧 ∈
ℝ* ∣ (𝑥𝑅𝑧 ∧ 𝑧𝑆𝑦)}) ⇒ ⊢ ((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*)
→ (𝐶 ∈ (𝐴𝑂𝐵) ↔ (𝐶 ∈ ℝ* ∧ 𝐴𝑅𝐶 ∧ 𝐶𝑆𝐵))) |
|
Theorem | ixxf 9869* |
The set of intervals of extended reals maps to subsets of extended
reals. (Contributed by FL, 14-Jun-2007.) (Revised by Mario Carneiro,
16-Nov-2013.)
|
⊢ 𝑂 = (𝑥 ∈ ℝ*, 𝑦 ∈ ℝ*
↦ {𝑧 ∈
ℝ* ∣ (𝑥𝑅𝑧 ∧ 𝑧𝑆𝑦)}) ⇒ ⊢ 𝑂:(ℝ* ×
ℝ*)⟶𝒫 ℝ* |
|
Theorem | ixxex 9870* |
The set of intervals of extended reals exists. (Contributed by Mario
Carneiro, 3-Nov-2013.) (Revised by Mario Carneiro, 17-Nov-2014.)
|
⊢ 𝑂 = (𝑥 ∈ ℝ*, 𝑦 ∈ ℝ*
↦ {𝑧 ∈
ℝ* ∣ (𝑥𝑅𝑧 ∧ 𝑧𝑆𝑦)}) ⇒ ⊢ 𝑂 ∈ V |
|
Theorem | ixxssxr 9871* |
The set of intervals of extended reals maps to subsets of extended
reals. (Contributed by Mario Carneiro, 4-Jul-2014.)
|
⊢ 𝑂 = (𝑥 ∈ ℝ*, 𝑦 ∈ ℝ*
↦ {𝑧 ∈
ℝ* ∣ (𝑥𝑅𝑧 ∧ 𝑧𝑆𝑦)}) ⇒ ⊢ (𝐴𝑂𝐵) ⊆
ℝ* |
|
Theorem | elixx3g 9872* |
Membership in a set of open intervals of extended reals. We use the
fact that an operation's value is empty outside of its domain to show
𝐴
∈ ℝ* and 𝐵 ∈ ℝ*.
(Contributed by Mario Carneiro,
3-Nov-2013.)
|
⊢ 𝑂 = (𝑥 ∈ ℝ*, 𝑦 ∈ ℝ*
↦ {𝑧 ∈
ℝ* ∣ (𝑥𝑅𝑧 ∧ 𝑧𝑆𝑦)}) ⇒ ⊢ (𝐶 ∈ (𝐴𝑂𝐵) ↔ ((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*
∧ 𝐶 ∈
ℝ*) ∧ (𝐴𝑅𝐶 ∧ 𝐶𝑆𝐵))) |
|
Theorem | ixxssixx 9873* |
An interval is a subset of its closure. (Contributed by Paul Chapman,
18-Oct-2007.) (Revised by Mario Carneiro, 3-Nov-2013.)
|
⊢ 𝑂 = (𝑥 ∈ ℝ*, 𝑦 ∈ ℝ*
↦ {𝑧 ∈
ℝ* ∣ (𝑥𝑅𝑧 ∧ 𝑧𝑆𝑦)}) & ⊢ 𝑃 = (𝑥 ∈ ℝ*, 𝑦 ∈ ℝ*
↦ {𝑧 ∈
ℝ* ∣ (𝑥𝑇𝑧 ∧ 𝑧𝑈𝑦)}) & ⊢ ((𝐴 ∈ ℝ*
∧ 𝑤 ∈
ℝ*) → (𝐴𝑅𝑤 → 𝐴𝑇𝑤))
& ⊢ ((𝑤 ∈ ℝ* ∧ 𝐵 ∈ ℝ*)
→ (𝑤𝑆𝐵 → 𝑤𝑈𝐵)) ⇒ ⊢ (𝐴𝑂𝐵) ⊆ (𝐴𝑃𝐵) |
|
Theorem | ixxdisj 9874* |
Split an interval into disjoint pieces. (Contributed by Mario
Carneiro, 16-Jun-2014.)
|
⊢ 𝑂 = (𝑥 ∈ ℝ*, 𝑦 ∈ ℝ*
↦ {𝑧 ∈
ℝ* ∣ (𝑥𝑅𝑧 ∧ 𝑧𝑆𝑦)}) & ⊢ 𝑃 = (𝑥 ∈ ℝ*, 𝑦 ∈ ℝ*
↦ {𝑧 ∈
ℝ* ∣ (𝑥𝑇𝑧 ∧ 𝑧𝑈𝑦)}) & ⊢ ((𝐵 ∈ ℝ*
∧ 𝑤 ∈
ℝ*) → (𝐵𝑇𝑤 ↔ ¬ 𝑤𝑆𝐵)) ⇒ ⊢ ((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*
∧ 𝐶 ∈
ℝ*) → ((𝐴𝑂𝐵) ∩ (𝐵𝑃𝐶)) = ∅) |
|
Theorem | ixxss1 9875* |
Subset relationship for intervals of extended reals. (Contributed by
Mario Carneiro, 3-Nov-2013.) (Revised by Mario Carneiro,
28-Apr-2015.)
|
⊢ 𝑂 = (𝑥 ∈ ℝ*, 𝑦 ∈ ℝ*
↦ {𝑧 ∈
ℝ* ∣ (𝑥𝑅𝑧 ∧ 𝑧𝑆𝑦)}) & ⊢ 𝑃 = (𝑥 ∈ ℝ*, 𝑦 ∈ ℝ*
↦ {𝑧 ∈
ℝ* ∣ (𝑥𝑇𝑧 ∧ 𝑧𝑆𝑦)}) & ⊢ ((𝐴 ∈ ℝ*
∧ 𝐵 ∈
ℝ* ∧ 𝑤 ∈ ℝ*) → ((𝐴𝑊𝐵 ∧ 𝐵𝑇𝑤) → 𝐴𝑅𝑤)) ⇒ ⊢ ((𝐴 ∈ ℝ* ∧ 𝐴𝑊𝐵) → (𝐵𝑃𝐶) ⊆ (𝐴𝑂𝐶)) |
|
Theorem | ixxss2 9876* |
Subset relationship for intervals of extended reals. (Contributed by
Mario Carneiro, 3-Nov-2013.) (Revised by Mario Carneiro,
28-Apr-2015.)
|
⊢ 𝑂 = (𝑥 ∈ ℝ*, 𝑦 ∈ ℝ*
↦ {𝑧 ∈
ℝ* ∣ (𝑥𝑅𝑧 ∧ 𝑧𝑆𝑦)}) & ⊢ 𝑃 = (𝑥 ∈ ℝ*, 𝑦 ∈ ℝ*
↦ {𝑧 ∈
ℝ* ∣ (𝑥𝑅𝑧 ∧ 𝑧𝑇𝑦)}) & ⊢ ((𝑤 ∈ ℝ*
∧ 𝐵 ∈
ℝ* ∧ 𝐶 ∈ ℝ*) → ((𝑤𝑇𝐵 ∧ 𝐵𝑊𝐶) → 𝑤𝑆𝐶)) ⇒ ⊢ ((𝐶 ∈ ℝ* ∧ 𝐵𝑊𝐶) → (𝐴𝑃𝐵) ⊆ (𝐴𝑂𝐶)) |
|
Theorem | ixxss12 9877* |
Subset relationship for intervals of extended reals. (Contributed by
Mario Carneiro, 20-Feb-2015.) (Revised by Mario Carneiro,
28-Apr-2015.)
|
⊢ 𝑂 = (𝑥 ∈ ℝ*, 𝑦 ∈ ℝ*
↦ {𝑧 ∈
ℝ* ∣ (𝑥𝑅𝑧 ∧ 𝑧𝑆𝑦)}) & ⊢ 𝑃 = (𝑥 ∈ ℝ*, 𝑦 ∈ ℝ*
↦ {𝑧 ∈
ℝ* ∣ (𝑥𝑇𝑧 ∧ 𝑧𝑈𝑦)}) & ⊢ ((𝐴 ∈ ℝ*
∧ 𝐶 ∈
ℝ* ∧ 𝑤 ∈ ℝ*) → ((𝐴𝑊𝐶 ∧ 𝐶𝑇𝑤) → 𝐴𝑅𝑤))
& ⊢ ((𝑤 ∈ ℝ* ∧ 𝐷 ∈ ℝ*
∧ 𝐵 ∈
ℝ*) → ((𝑤𝑈𝐷 ∧ 𝐷𝑋𝐵) → 𝑤𝑆𝐵)) ⇒ ⊢ (((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*)
∧ (𝐴𝑊𝐶 ∧ 𝐷𝑋𝐵)) → (𝐶𝑃𝐷) ⊆ (𝐴𝑂𝐵)) |
|
Theorem | iooex 9878 |
The set of open intervals of extended reals exists. (Contributed by NM,
6-Feb-2007.) (Revised by Mario Carneiro, 3-Nov-2013.)
|
⊢ (,) ∈ V |
|
Theorem | iooval 9879* |
Value of the open interval function. (Contributed by NM, 24-Dec-2006.)
(Revised by Mario Carneiro, 3-Nov-2013.)
|
⊢ ((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*)
→ (𝐴(,)𝐵) = {𝑥 ∈ ℝ* ∣ (𝐴 < 𝑥 ∧ 𝑥 < 𝐵)}) |
|
Theorem | iooidg 9880 |
An open interval with identical lower and upper bounds is empty.
(Contributed by Jim Kingdon, 29-Mar-2020.)
|
⊢ (𝐴 ∈ ℝ* → (𝐴(,)𝐴) = ∅) |
|
Theorem | elioo3g 9881 |
Membership in a set of open intervals of extended reals. We use the
fact that an operation's value is empty outside of its domain to show
𝐴
∈ ℝ* and 𝐵 ∈ ℝ*.
(Contributed by NM, 24-Dec-2006.)
(Revised by Mario Carneiro, 3-Nov-2013.)
|
⊢ (𝐶 ∈ (𝐴(,)𝐵) ↔ ((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*
∧ 𝐶 ∈
ℝ*) ∧ (𝐴 < 𝐶 ∧ 𝐶 < 𝐵))) |
|
Theorem | elioo1 9882 |
Membership in an open interval of extended reals. (Contributed by NM,
24-Dec-2006.) (Revised by Mario Carneiro, 3-Nov-2013.)
|
⊢ ((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*)
→ (𝐶 ∈ (𝐴(,)𝐵) ↔ (𝐶 ∈ ℝ* ∧ 𝐴 < 𝐶 ∧ 𝐶 < 𝐵))) |
|
Theorem | elioore 9883 |
A member of an open interval of reals is a real. (Contributed by NM,
17-Aug-2008.) (Revised by Mario Carneiro, 3-Nov-2013.)
|
⊢ (𝐴 ∈ (𝐵(,)𝐶) → 𝐴 ∈ ℝ) |
|
Theorem | lbioog 9884 |
An open interval does not contain its left endpoint. (Contributed by
Jim Kingdon, 30-Mar-2020.)
|
⊢ ((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*)
→ ¬ 𝐴 ∈
(𝐴(,)𝐵)) |
|
Theorem | ubioog 9885 |
An open interval does not contain its right endpoint. (Contributed by
Jim Kingdon, 30-Mar-2020.)
|
⊢ ((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*)
→ ¬ 𝐵 ∈
(𝐴(,)𝐵)) |
|
Theorem | iooval2 9886* |
Value of the open interval function. (Contributed by NM, 6-Feb-2007.)
(Revised by Mario Carneiro, 3-Nov-2013.)
|
⊢ ((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*)
→ (𝐴(,)𝐵) = {𝑥 ∈ ℝ ∣ (𝐴 < 𝑥 ∧ 𝑥 < 𝐵)}) |
|
Theorem | iooss1 9887 |
Subset relationship for open intervals of extended reals. (Contributed
by NM, 7-Feb-2007.) (Revised by Mario Carneiro, 20-Feb-2015.)
|
⊢ ((𝐴 ∈ ℝ* ∧ 𝐴 ≤ 𝐵) → (𝐵(,)𝐶) ⊆ (𝐴(,)𝐶)) |
|
Theorem | iooss2 9888 |
Subset relationship for open intervals of extended reals. (Contributed
by NM, 7-Feb-2007.) (Revised by Mario Carneiro, 3-Nov-2013.)
|
⊢ ((𝐶 ∈ ℝ* ∧ 𝐵 ≤ 𝐶) → (𝐴(,)𝐵) ⊆ (𝐴(,)𝐶)) |
|
Theorem | iocval 9889* |
Value of the open-below, closed-above interval function. (Contributed
by NM, 24-Dec-2006.) (Revised by Mario Carneiro, 3-Nov-2013.)
|
⊢ ((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*)
→ (𝐴(,]𝐵) = {𝑥 ∈ ℝ* ∣ (𝐴 < 𝑥 ∧ 𝑥 ≤ 𝐵)}) |
|
Theorem | icoval 9890* |
Value of the closed-below, open-above interval function. (Contributed
by NM, 24-Dec-2006.) (Revised by Mario Carneiro, 3-Nov-2013.)
|
⊢ ((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*)
→ (𝐴[,)𝐵) = {𝑥 ∈ ℝ* ∣ (𝐴 ≤ 𝑥 ∧ 𝑥 < 𝐵)}) |
|
Theorem | iccval 9891* |
Value of the closed interval function. (Contributed by NM,
24-Dec-2006.) (Revised by Mario Carneiro, 3-Nov-2013.)
|
⊢ ((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*)
→ (𝐴[,]𝐵) = {𝑥 ∈ ℝ* ∣ (𝐴 ≤ 𝑥 ∧ 𝑥 ≤ 𝐵)}) |
|
Theorem | elioo2 9892 |
Membership in an open interval of extended reals. (Contributed by NM,
6-Feb-2007.)
|
⊢ ((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*)
→ (𝐶 ∈ (𝐴(,)𝐵) ↔ (𝐶 ∈ ℝ ∧ 𝐴 < 𝐶 ∧ 𝐶 < 𝐵))) |
|
Theorem | elioc1 9893 |
Membership in an open-below, closed-above interval of extended reals.
(Contributed by NM, 24-Dec-2006.) (Revised by Mario Carneiro,
3-Nov-2013.)
|
⊢ ((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*)
→ (𝐶 ∈ (𝐴(,]𝐵) ↔ (𝐶 ∈ ℝ* ∧ 𝐴 < 𝐶 ∧ 𝐶 ≤ 𝐵))) |
|
Theorem | elico1 9894 |
Membership in a closed-below, open-above interval of extended reals.
(Contributed by NM, 24-Dec-2006.) (Revised by Mario Carneiro,
3-Nov-2013.)
|
⊢ ((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*)
→ (𝐶 ∈ (𝐴[,)𝐵) ↔ (𝐶 ∈ ℝ* ∧ 𝐴 ≤ 𝐶 ∧ 𝐶 < 𝐵))) |
|
Theorem | elicc1 9895 |
Membership in a closed interval of extended reals. (Contributed by NM,
24-Dec-2006.) (Revised by Mario Carneiro, 3-Nov-2013.)
|
⊢ ((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*)
→ (𝐶 ∈ (𝐴[,]𝐵) ↔ (𝐶 ∈ ℝ* ∧ 𝐴 ≤ 𝐶 ∧ 𝐶 ≤ 𝐵))) |
|
Theorem | iccid 9896 |
A closed interval with identical lower and upper bounds is a singleton.
(Contributed by Jeff Hankins, 13-Jul-2009.)
|
⊢ (𝐴 ∈ ℝ* → (𝐴[,]𝐴) = {𝐴}) |
|
Theorem | icc0r 9897 |
An empty closed interval of extended reals. (Contributed by Jim
Kingdon, 30-Mar-2020.)
|
⊢ ((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*)
→ (𝐵 < 𝐴 → (𝐴[,]𝐵) = ∅)) |
|
Theorem | eliooxr 9898 |
An inhabited open interval spans an interval of extended reals.
(Contributed by NM, 17-Aug-2008.)
|
⊢ (𝐴 ∈ (𝐵(,)𝐶) → (𝐵 ∈ ℝ* ∧ 𝐶 ∈
ℝ*)) |
|
Theorem | eliooord 9899 |
Ordering implied by a member of an open interval of reals. (Contributed
by NM, 17-Aug-2008.) (Revised by Mario Carneiro, 9-May-2014.)
|
⊢ (𝐴 ∈ (𝐵(,)𝐶) → (𝐵 < 𝐴 ∧ 𝐴 < 𝐶)) |
|
Theorem | ubioc1 9900 |
The upper bound belongs to an open-below, closed-above interval. See
ubicc2 9956. (Contributed by FL, 29-May-2014.)
|
⊢ ((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*
∧ 𝐴 < 𝐵) → 𝐵 ∈ (𝐴(,]𝐵)) |