Home | Metamath
Proof Explorer Theorem List (p. 135 of 466) | < Previous Next > |
Bad symbols? Try the
GIF version. |
||
Mirrors > Metamath Home Page > MPE Home Page > Theorem List Contents > Recent Proofs This page: Page List |
Color key: | Metamath Proof Explorer
(1-29289) |
Hilbert Space Explorer
(29290-30812) |
Users' Mathboxes
(30813-46532) |
Type | Label | Description |
---|---|---|
Statement | ||
Theorem | nelfzo 13401 | An integer not being a member of a half-open finite set of integers. (Contributed by AV, 29-Apr-2020.) |
⊢ ((𝐾 ∈ ℤ ∧ 𝑀 ∈ ℤ ∧ 𝑁 ∈ ℤ) → (𝐾 ∉ (𝑀..^𝑁) ↔ (𝐾 < 𝑀 ∨ 𝑁 ≤ 𝐾))) | ||
Theorem | fzolb 13402 | The left endpoint of a half-open integer interval is in the set iff the two arguments are integers with 𝑀 < 𝑁. This provides an alternative notation for the "strict upper integer" predicate by analogy to the "weak upper integer" predicate 𝑀 ∈ (ℤ≥‘𝑁). (Contributed by Mario Carneiro, 29-Sep-2015.) |
⊢ (𝑀 ∈ (𝑀..^𝑁) ↔ (𝑀 ∈ ℤ ∧ 𝑁 ∈ ℤ ∧ 𝑀 < 𝑁)) | ||
Theorem | fzolb2 13403 | The left endpoint of a half-open integer interval is in the set iff the two arguments are integers with 𝑀 < 𝑁. This provides an alternative notation for the "strict upper integer" predicate by analogy to the "weak upper integer" predicate 𝑀 ∈ (ℤ≥‘𝑁). (Contributed by Mario Carneiro, 29-Sep-2015.) |
⊢ ((𝑀 ∈ ℤ ∧ 𝑁 ∈ ℤ) → (𝑀 ∈ (𝑀..^𝑁) ↔ 𝑀 < 𝑁)) | ||
Theorem | elfzole1 13404 | A member in a half-open integer interval is greater than or equal to the lower bound. (Contributed by Stefan O'Rear, 15-Aug-2015.) |
⊢ (𝐾 ∈ (𝑀..^𝑁) → 𝑀 ≤ 𝐾) | ||
Theorem | elfzolt2 13405 | A member in a half-open integer interval is less than the upper bound. (Contributed by Stefan O'Rear, 15-Aug-2015.) |
⊢ (𝐾 ∈ (𝑀..^𝑁) → 𝐾 < 𝑁) | ||
Theorem | elfzolt3 13406 | Membership in a half-open integer interval implies that the bounds are unequal. (Contributed by Stefan O'Rear, 15-Aug-2015.) |
⊢ (𝐾 ∈ (𝑀..^𝑁) → 𝑀 < 𝑁) | ||
Theorem | elfzolt2b 13407 | A member in a half-open integer interval is less than the upper bound. (Contributed by Mario Carneiro, 29-Sep-2015.) |
⊢ (𝐾 ∈ (𝑀..^𝑁) → 𝐾 ∈ (𝐾..^𝑁)) | ||
Theorem | elfzolt3b 13408 | Membership in a half-open integer interval implies that the bounds are unequal. (Contributed by Mario Carneiro, 29-Sep-2015.) |
⊢ (𝐾 ∈ (𝑀..^𝑁) → 𝑀 ∈ (𝑀..^𝑁)) | ||
Theorem | elfzop1le2 13409 | A member in a half-open integer interval plus 1 is less than or equal to the upper bound. (Contributed by Glauco Siliprandi, 11-Dec-2019.) |
⊢ (𝐾 ∈ (𝑀..^𝑁) → (𝐾 + 1) ≤ 𝑁) | ||
Theorem | fzonel 13410 | A half-open range does not contain its right endpoint. (Contributed by Stefan O'Rear, 25-Aug-2015.) |
⊢ ¬ 𝐵 ∈ (𝐴..^𝐵) | ||
Theorem | elfzouz2 13411 | The upper bound of a half-open range is greater than or equal to an element of the range. (Contributed by Mario Carneiro, 29-Sep-2015.) |
⊢ (𝐾 ∈ (𝑀..^𝑁) → 𝑁 ∈ (ℤ≥‘𝐾)) | ||
Theorem | elfzofz 13412 | A half-open range is contained in the corresponding closed range. (Contributed by Stefan O'Rear, 23-Aug-2015.) |
⊢ (𝐾 ∈ (𝑀..^𝑁) → 𝐾 ∈ (𝑀...𝑁)) | ||
Theorem | elfzo3 13413 | Express membership in a half-open integer interval in terms of the "less than or equal to" and "less than" predicates on integers, resp. 𝐾 ∈ (ℤ≥‘𝑀) ↔ 𝑀 ≤ 𝐾, 𝐾 ∈ (𝐾..^𝑁) ↔ 𝐾 < 𝑁. (Contributed by Mario Carneiro, 29-Sep-2015.) |
⊢ (𝐾 ∈ (𝑀..^𝑁) ↔ (𝐾 ∈ (ℤ≥‘𝑀) ∧ 𝐾 ∈ (𝐾..^𝑁))) | ||
Theorem | fzon0 13414 | A half-open integer interval is nonempty iff it contains its left endpoint. (Contributed by Mario Carneiro, 29-Sep-2015.) |
⊢ ((𝑀..^𝑁) ≠ ∅ ↔ 𝑀 ∈ (𝑀..^𝑁)) | ||
Theorem | fzossfz 13415 | A half-open range is contained in the corresponding closed range. (Contributed by Stefan O'Rear, 23-Aug-2015.) (Revised by Mario Carneiro, 29-Sep-2015.) |
⊢ (𝐴..^𝐵) ⊆ (𝐴...𝐵) | ||
Theorem | fzossz 13416 | A half-open integer interval is a set of integers. (Contributed by Glauco Siliprandi, 8-Apr-2021.) |
⊢ (𝑀..^𝑁) ⊆ ℤ | ||
Theorem | fzon 13417 | A half-open set of sequential integers is empty if the bounds are equal or reversed. (Contributed by Alexander van der Vekens, 30-Oct-2017.) |
⊢ ((𝑀 ∈ ℤ ∧ 𝑁 ∈ ℤ) → (𝑁 ≤ 𝑀 ↔ (𝑀..^𝑁) = ∅)) | ||
Theorem | fzo0n 13418 | A half-open range of nonnegative integers is empty iff the upper bound is not positive. (Contributed by AV, 2-May-2020.) |
⊢ ((𝑀 ∈ ℤ ∧ 𝑁 ∈ ℤ) → (𝑁 ≤ 𝑀 ↔ (0..^(𝑁 − 𝑀)) = ∅)) | ||
Theorem | fzonlt0 13419 | A half-open integer range is empty if the bounds are equal or reversed. (Contributed by AV, 20-Oct-2018.) |
⊢ ((𝑀 ∈ ℤ ∧ 𝑁 ∈ ℤ) → (¬ 𝑀 < 𝑁 ↔ (𝑀..^𝑁) = ∅)) | ||
Theorem | fzo0 13420 | Half-open sets with equal endpoints are empty. (Contributed by Stefan O'Rear, 15-Aug-2015.) (Revised by Mario Carneiro, 29-Sep-2015.) |
⊢ (𝐴..^𝐴) = ∅ | ||
Theorem | fzonnsub 13421 | If 𝐾 < 𝑁 then 𝑁 − 𝐾 is a positive integer. (Contributed by Mario Carneiro, 29-Sep-2015.) (Revised by Mario Carneiro, 1-Jan-2017.) |
⊢ (𝐾 ∈ (𝑀..^𝑁) → (𝑁 − 𝐾) ∈ ℕ) | ||
Theorem | fzonnsub2 13422 | If 𝑀 < 𝑁 then 𝑁 − 𝑀 is a positive integer. (Contributed by Mario Carneiro, 1-Jan-2017.) |
⊢ (𝐾 ∈ (𝑀..^𝑁) → (𝑁 − 𝑀) ∈ ℕ) | ||
Theorem | fzoss1 13423 | Subset relationship for half-open sequences of integers. (Contributed by Stefan O'Rear, 15-Aug-2015.) (Revised by Mario Carneiro, 29-Sep-2015.) |
⊢ (𝐾 ∈ (ℤ≥‘𝑀) → (𝐾..^𝑁) ⊆ (𝑀..^𝑁)) | ||
Theorem | fzoss2 13424 | Subset relationship for half-open sequences of integers. (Contributed by Stefan O'Rear, 15-Aug-2015.) (Revised by Mario Carneiro, 29-Sep-2015.) |
⊢ (𝑁 ∈ (ℤ≥‘𝐾) → (𝑀..^𝐾) ⊆ (𝑀..^𝑁)) | ||
Theorem | fzossrbm1 13425 | Subset of a half-open range. (Contributed by Alexander van der Vekens, 1-Nov-2017.) |
⊢ (𝑁 ∈ ℤ → (0..^(𝑁 − 1)) ⊆ (0..^𝑁)) | ||
Theorem | fzo0ss1 13426 | Subset relationship for half-open integer ranges with lower bounds 0 and 1. (Contributed by Alexander van der Vekens, 18-Mar-2018.) |
⊢ (1..^𝑁) ⊆ (0..^𝑁) | ||
Theorem | fzossnn0 13427 | A half-open integer range starting at a nonnegative integer is a subset of the nonnegative integers. (Contributed by Alexander van der Vekens, 13-May-2018.) |
⊢ (𝑀 ∈ ℕ0 → (𝑀..^𝑁) ⊆ ℕ0) | ||
Theorem | fzospliti 13428 | One direction of splitting a half-open integer range in half. (Contributed by Stefan O'Rear, 14-Aug-2015.) |
⊢ ((𝐴 ∈ (𝐵..^𝐶) ∧ 𝐷 ∈ ℤ) → (𝐴 ∈ (𝐵..^𝐷) ∨ 𝐴 ∈ (𝐷..^𝐶))) | ||
Theorem | fzosplit 13429 | Split a half-open integer range in half. (Contributed by Stefan O'Rear, 14-Aug-2015.) |
⊢ (𝐷 ∈ (𝐵...𝐶) → (𝐵..^𝐶) = ((𝐵..^𝐷) ∪ (𝐷..^𝐶))) | ||
Theorem | fzodisj 13430 | Abutting half-open integer ranges are disjoint. (Contributed by Stefan O'Rear, 14-Aug-2015.) |
⊢ ((𝐴..^𝐵) ∩ (𝐵..^𝐶)) = ∅ | ||
Theorem | fzouzsplit 13431 | Split an upper integer set into a half-open integer range and another upper integer set. (Contributed by Mario Carneiro, 21-Sep-2016.) |
⊢ (𝐵 ∈ (ℤ≥‘𝐴) → (ℤ≥‘𝐴) = ((𝐴..^𝐵) ∪ (ℤ≥‘𝐵))) | ||
Theorem | fzouzdisj 13432 | A half-open integer range does not overlap the upper integer range starting at the endpoint of the first range. (Contributed by Mario Carneiro, 21-Sep-2016.) |
⊢ ((𝐴..^𝐵) ∩ (ℤ≥‘𝐵)) = ∅ | ||
Theorem | fzoun 13433 | A half-open integer range as union of two half-open integer ranges. (Contributed by AV, 23-Apr-2022.) |
⊢ ((𝐵 ∈ (ℤ≥‘𝐴) ∧ 𝐶 ∈ ℕ0) → (𝐴..^(𝐵 + 𝐶)) = ((𝐴..^𝐵) ∪ (𝐵..^(𝐵 + 𝐶)))) | ||
Theorem | fzodisjsn 13434 | A half-open integer range and the singleton of its upper bound are disjoint. (Contributed by AV, 7-Mar-2021.) |
⊢ ((𝐴..^𝐵) ∩ {𝐵}) = ∅ | ||
Theorem | prinfzo0 13435 | The intersection of a half-open integer range and the pair of its outer left borders is empty. (Contributed by AV, 9-Jan-2021.) |
⊢ (𝑀 ∈ ℤ → ({𝑀, 𝑁} ∩ ((𝑀 + 1)..^𝑁)) = ∅) | ||
Theorem | lbfzo0 13436 | An integer is strictly greater than zero iff it is a member of ℕ. (Contributed by Mario Carneiro, 29-Sep-2015.) |
⊢ (0 ∈ (0..^𝐴) ↔ 𝐴 ∈ ℕ) | ||
Theorem | elfzo0 13437 | Membership in a half-open integer range based at 0. (Contributed by Stefan O'Rear, 15-Aug-2015.) (Revised by Mario Carneiro, 29-Sep-2015.) |
⊢ (𝐴 ∈ (0..^𝐵) ↔ (𝐴 ∈ ℕ0 ∧ 𝐵 ∈ ℕ ∧ 𝐴 < 𝐵)) | ||
Theorem | elfzo0z 13438 | Membership in a half-open range of nonnegative integers, generalization of elfzo0 13437 requiring the upper bound to be an integer only. (Contributed by Alexander van der Vekens, 23-Sep-2018.) |
⊢ (𝐴 ∈ (0..^𝐵) ↔ (𝐴 ∈ ℕ0 ∧ 𝐵 ∈ ℤ ∧ 𝐴 < 𝐵)) | ||
Theorem | nn0p1elfzo 13439 | A nonnegative integer increased by 1 which is less than or equal to another integer is an element of a half-open range of integers. (Contributed by AV, 27-Feb-2021.) |
⊢ ((𝐾 ∈ ℕ0 ∧ 𝑁 ∈ ℕ0 ∧ (𝐾 + 1) ≤ 𝑁) → 𝐾 ∈ (0..^𝑁)) | ||
Theorem | elfzo0le 13440 | A member in a half-open range of nonnegative integers is less than or equal to the upper bound of the range. (Contributed by Alexander van der Vekens, 23-Sep-2018.) |
⊢ (𝐴 ∈ (0..^𝐵) → 𝐴 ≤ 𝐵) | ||
Theorem | elfzonn0 13441 | A member of a half-open range of nonnegative integers is a nonnegative integer. (Contributed by Alexander van der Vekens, 21-May-2018.) |
⊢ (𝐾 ∈ (0..^𝑁) → 𝐾 ∈ ℕ0) | ||
Theorem | fzonmapblen 13442 | The result of subtracting a nonnegative integer from a positive integer and adding another nonnegative integer which is less than the first one is less than the positive integer. (Contributed by Alexander van der Vekens, 19-May-2018.) |
⊢ ((𝐴 ∈ (0..^𝑁) ∧ 𝐵 ∈ (0..^𝑁) ∧ 𝐵 < 𝐴) → (𝐵 + (𝑁 − 𝐴)) < 𝑁) | ||
Theorem | fzofzim 13443 | If a nonnegative integer in a finite interval of integers is not the upper bound of the interval, it is contained in the corresponding half-open integer range. (Contributed by Alexander van der Vekens, 15-Jun-2018.) |
⊢ ((𝐾 ≠ 𝑀 ∧ 𝐾 ∈ (0...𝑀)) → 𝐾 ∈ (0..^𝑀)) | ||
Theorem | fz1fzo0m1 13444 | Translation of one between closed and open integer ranges. (Contributed by Thierry Arnoux, 28-Jul-2020.) |
⊢ (𝑀 ∈ (1...𝑁) → (𝑀 − 1) ∈ (0..^𝑁)) | ||
Theorem | fzossnn 13445 | Half-open integer ranges starting with 1 are subsets of ℕ. (Contributed by Thierry Arnoux, 28-Dec-2016.) |
⊢ (1..^𝑁) ⊆ ℕ | ||
Theorem | elfzo1 13446 | Membership in a half-open integer range based at 1. (Contributed by Thierry Arnoux, 14-Feb-2017.) |
⊢ (𝑁 ∈ (1..^𝑀) ↔ (𝑁 ∈ ℕ ∧ 𝑀 ∈ ℕ ∧ 𝑁 < 𝑀)) | ||
Theorem | fzo1fzo0n0 13447 | An integer between 1 and an upper bound of a half-open integer range is not 0 and between 0 and the upper bound of the half-open integer range. (Contributed by Alexander van der Vekens, 21-Mar-2018.) |
⊢ (𝐾 ∈ (1..^𝑁) ↔ (𝐾 ∈ (0..^𝑁) ∧ 𝐾 ≠ 0)) | ||
Theorem | fzo0n0 13448 | A half-open integer range based at 0 is nonempty precisely if the upper bound is a positive integer. (Contributed by Stefan O'Rear, 15-Aug-2015.) (Revised by Mario Carneiro, 29-Sep-2015.) |
⊢ ((0..^𝐴) ≠ ∅ ↔ 𝐴 ∈ ℕ) | ||
Theorem | fzoaddel 13449 | Translate membership in a half-open integer range. (Contributed by Stefan O'Rear, 15-Aug-2015.) |
⊢ ((𝐴 ∈ (𝐵..^𝐶) ∧ 𝐷 ∈ ℤ) → (𝐴 + 𝐷) ∈ ((𝐵 + 𝐷)..^(𝐶 + 𝐷))) | ||
Theorem | fzo0addel 13450 | Translate membership in a 0-based half-open integer range. (Contributed by AV, 30-Apr-2020.) |
⊢ ((𝐴 ∈ (0..^𝐶) ∧ 𝐷 ∈ ℤ) → (𝐴 + 𝐷) ∈ (𝐷..^(𝐶 + 𝐷))) | ||
Theorem | fzo0addelr 13451 | Translate membership in a 0-based half-open integer range. (Contributed by AV, 30-Apr-2020.) |
⊢ ((𝐴 ∈ (0..^𝐶) ∧ 𝐷 ∈ ℤ) → (𝐴 + 𝐷) ∈ (𝐷..^(𝐷 + 𝐶))) | ||
Theorem | fzoaddel2 13452 | Translate membership in a shifted-down half-open integer range. (Contributed by Stefan O'Rear, 15-Aug-2015.) |
⊢ ((𝐴 ∈ (0..^(𝐵 − 𝐶)) ∧ 𝐵 ∈ ℤ ∧ 𝐶 ∈ ℤ) → (𝐴 + 𝐶) ∈ (𝐶..^𝐵)) | ||
Theorem | elfzoext 13453 | Membership of an integer in an extended open range of integers. (Contributed by AV, 30-Apr-2020.) |
⊢ ((𝑍 ∈ (𝑀..^𝑁) ∧ 𝐼 ∈ ℕ0) → 𝑍 ∈ (𝑀..^(𝑁 + 𝐼))) | ||
Theorem | elincfzoext 13454 | Membership of an increased integer in a correspondingly extended half-open range of integers. (Contributed by AV, 30-Apr-2020.) |
⊢ ((𝑍 ∈ (𝑀..^𝑁) ∧ 𝐼 ∈ ℕ0) → (𝑍 + 𝐼) ∈ (𝑀..^(𝑁 + 𝐼))) | ||
Theorem | fzosubel 13455 | Translate membership in a half-open integer range. (Contributed by Stefan O'Rear, 15-Aug-2015.) |
⊢ ((𝐴 ∈ (𝐵..^𝐶) ∧ 𝐷 ∈ ℤ) → (𝐴 − 𝐷) ∈ ((𝐵 − 𝐷)..^(𝐶 − 𝐷))) | ||
Theorem | fzosubel2 13456 | Membership in a translated half-open integer range implies translated membership in the original range. (Contributed by Stefan O'Rear, 15-Aug-2015.) |
⊢ ((𝐴 ∈ ((𝐵 + 𝐶)..^(𝐵 + 𝐷)) ∧ (𝐵 ∈ ℤ ∧ 𝐶 ∈ ℤ ∧ 𝐷 ∈ ℤ)) → (𝐴 − 𝐵) ∈ (𝐶..^𝐷)) | ||
Theorem | fzosubel3 13457 | Membership in a translated half-open integer range when the original range is zero-based. (Contributed by Stefan O'Rear, 15-Aug-2015.) |
⊢ ((𝐴 ∈ (𝐵..^(𝐵 + 𝐷)) ∧ 𝐷 ∈ ℤ) → (𝐴 − 𝐵) ∈ (0..^𝐷)) | ||
Theorem | eluzgtdifelfzo 13458 | Membership of the difference of integers in a half-open range of nonnegative integers. (Contributed by Alexander van der Vekens, 17-Sep-2018.) |
⊢ ((𝐴 ∈ ℤ ∧ 𝐵 ∈ ℤ) → ((𝑁 ∈ (ℤ≥‘𝐴) ∧ 𝐵 < 𝐴) → (𝑁 − 𝐴) ∈ (0..^(𝑁 − 𝐵)))) | ||
Theorem | ige2m2fzo 13459 | Membership of an integer greater than 1 decreased by 2 in a half-open range of nonnegative integers. (Contributed by Alexander van der Vekens, 3-Oct-2018.) |
⊢ (𝑁 ∈ (ℤ≥‘2) → (𝑁 − 2) ∈ (0..^(𝑁 − 1))) | ||
Theorem | fzocatel 13460 | Translate membership in a half-open integer range. (Contributed by Thierry Arnoux, 28-Sep-2018.) |
⊢ (((𝐴 ∈ (0..^(𝐵 + 𝐶)) ∧ ¬ 𝐴 ∈ (0..^𝐵)) ∧ (𝐵 ∈ ℤ ∧ 𝐶 ∈ ℤ)) → (𝐴 − 𝐵) ∈ (0..^𝐶)) | ||
Theorem | ubmelfzo 13461 | If an integer in a 1-based finite set of sequential integers is subtracted from the upper bound of this finite set of sequential integers, the result is contained in a half-open range of nonnegative integers with the same upper bound. (Contributed by AV, 18-Mar-2018.) (Revised by AV, 30-Oct-2018.) |
⊢ (𝐾 ∈ (1...𝑁) → (𝑁 − 𝐾) ∈ (0..^𝑁)) | ||
Theorem | elfzodifsumelfzo 13462 | If an integer is in a half-open range of nonnegative integers with a difference as upper bound, the sum of the integer with the subtrahend of the difference is in a half-open range of nonnegative integers containing the minuend of the difference. (Contributed by AV, 13-Nov-2018.) |
⊢ ((𝑀 ∈ (0...𝑁) ∧ 𝑁 ∈ (0...𝑃)) → (𝐼 ∈ (0..^(𝑁 − 𝑀)) → (𝐼 + 𝑀) ∈ (0..^𝑃))) | ||
Theorem | elfzom1elp1fzo 13463 | Membership of an integer incremented by one in a half-open range of nonnegative integers. (Contributed by Alexander van der Vekens, 24-Jun-2018.) (Proof shortened by AV, 5-Jan-2020.) |
⊢ ((𝑁 ∈ ℤ ∧ 𝐼 ∈ (0..^(𝑁 − 1))) → (𝐼 + 1) ∈ (0..^𝑁)) | ||
Theorem | elfzom1elfzo 13464 | Membership in a half-open range of nonnegative integers. (Contributed by Alexander van der Vekens, 18-Jun-2018.) |
⊢ ((𝑁 ∈ ℤ ∧ 𝐼 ∈ (0..^(𝑁 − 1))) → 𝐼 ∈ (0..^𝑁)) | ||
Theorem | fzval3 13465 | Expressing a closed integer range as a half-open integer range. (Contributed by Stefan O'Rear, 15-Aug-2015.) |
⊢ (𝑁 ∈ ℤ → (𝑀...𝑁) = (𝑀..^(𝑁 + 1))) | ||
Theorem | fz0add1fz1 13466 | Translate membership in a 0-based half-open integer range into membership in a 1-based finite sequence of integers. (Contributed by Alexander van der Vekens, 23-Nov-2017.) |
⊢ ((𝑁 ∈ ℕ0 ∧ 𝑋 ∈ (0..^𝑁)) → (𝑋 + 1) ∈ (1...𝑁)) | ||
Theorem | fzosn 13467 | Expressing a singleton as a half-open range. (Contributed by Stefan O'Rear, 23-Aug-2015.) |
⊢ (𝐴 ∈ ℤ → (𝐴..^(𝐴 + 1)) = {𝐴}) | ||
Theorem | elfzomin 13468 | Membership of an integer in the smallest open range of integers. (Contributed by Alexander van der Vekens, 22-Sep-2018.) |
⊢ (𝑍 ∈ ℤ → 𝑍 ∈ (𝑍..^(𝑍 + 1))) | ||
Theorem | zpnn0elfzo 13469 | Membership of an integer increased by a nonnegative integer in a half- open integer range. (Contributed by Alexander van der Vekens, 22-Sep-2018.) |
⊢ ((𝑍 ∈ ℤ ∧ 𝑁 ∈ ℕ0) → (𝑍 + 𝑁) ∈ (𝑍..^((𝑍 + 𝑁) + 1))) | ||
Theorem | zpnn0elfzo1 13470 | Membership of an integer increased by a nonnegative integer in a half- open integer range. (Contributed by Alexander van der Vekens, 22-Sep-2018.) |
⊢ ((𝑍 ∈ ℤ ∧ 𝑁 ∈ ℕ0) → (𝑍 + 𝑁) ∈ (𝑍..^(𝑍 + (𝑁 + 1)))) | ||
Theorem | fzosplitsnm1 13471 | Removing a singleton from a half-open integer range at the end. (Contributed by Alexander van der Vekens, 23-Mar-2018.) |
⊢ ((𝐴 ∈ ℤ ∧ 𝐵 ∈ (ℤ≥‘(𝐴 + 1))) → (𝐴..^𝐵) = ((𝐴..^(𝐵 − 1)) ∪ {(𝐵 − 1)})) | ||
Theorem | elfzonlteqm1 13472 | If an element of a half-open integer range is not less than the upper bound of the range decreased by 1, it must be equal to the upper bound of the range decreased by 1. (Contributed by AV, 3-Nov-2018.) |
⊢ ((𝐴 ∈ (0..^𝐵) ∧ ¬ 𝐴 < (𝐵 − 1)) → 𝐴 = (𝐵 − 1)) | ||
Theorem | fzonn0p1 13473 | A nonnegative integer is element of the half-open range of nonnegative integers with the element increased by one as an upper bound. (Contributed by Alexander van der Vekens, 5-Aug-2018.) |
⊢ (𝑁 ∈ ℕ0 → 𝑁 ∈ (0..^(𝑁 + 1))) | ||
Theorem | fzossfzop1 13474 | A half-open range of nonnegative integers is a subset of a half-open range of nonnegative integers with the upper bound increased by one. (Contributed by Alexander van der Vekens, 5-Aug-2018.) |
⊢ (𝑁 ∈ ℕ0 → (0..^𝑁) ⊆ (0..^(𝑁 + 1))) | ||
Theorem | fzonn0p1p1 13475 | If a nonnegative integer is element of a half-open range of nonnegative integers, increasing this integer by one results in an element of a half- open range of nonnegative integers with the upper bound increased by one. (Contributed by Alexander van der Vekens, 5-Aug-2018.) |
⊢ (𝐼 ∈ (0..^𝑁) → (𝐼 + 1) ∈ (0..^(𝑁 + 1))) | ||
Theorem | elfzom1p1elfzo 13476 | Increasing an element of a half-open range of nonnegative integers by 1 results in an element of the half-open range of nonnegative integers with an upper bound increased by 1. (Contributed by Alexander van der Vekens, 1-Aug-2018.) (Proof shortened by Thierry Arnoux, 14-Dec-2023.) |
⊢ ((𝑁 ∈ ℕ ∧ 𝑋 ∈ (0..^(𝑁 − 1))) → (𝑋 + 1) ∈ (0..^𝑁)) | ||
Theorem | fzo0ssnn0 13477 | Half-open integer ranges starting with 0 are subsets of NN0. (Contributed by Thierry Arnoux, 8-Oct-2018.) (Proof shortened by JJ, 1-Jun-2021.) |
⊢ (0..^𝑁) ⊆ ℕ0 | ||
Theorem | fzo01 13478 | Expressing the singleton of 0 as a half-open integer range. (Contributed by Stefan O'Rear, 15-Aug-2015.) |
⊢ (0..^1) = {0} | ||
Theorem | fzo12sn 13479 | A 1-based half-open integer interval up to, but not including, 2 is a singleton. (Contributed by Alexander van der Vekens, 31-Jan-2018.) |
⊢ (1..^2) = {1} | ||
Theorem | fzo13pr 13480 | A 1-based half-open integer interval up to, but not including, 3 is a pair. (Contributed by Thierry Arnoux, 11-Jul-2020.) |
⊢ (1..^3) = {1, 2} | ||
Theorem | fzo0to2pr 13481 | A half-open integer range from 0 to 2 is an unordered pair. (Contributed by Alexander van der Vekens, 4-Dec-2017.) |
⊢ (0..^2) = {0, 1} | ||
Theorem | fzo0to3tp 13482 | A half-open integer range from 0 to 3 is an unordered triple. (Contributed by Alexander van der Vekens, 9-Nov-2017.) |
⊢ (0..^3) = {0, 1, 2} | ||
Theorem | fzo0to42pr 13483 | A half-open integer range from 0 to 4 is a union of two unordered pairs. (Contributed by Alexander van der Vekens, 17-Nov-2017.) |
⊢ (0..^4) = ({0, 1} ∪ {2, 3}) | ||
Theorem | fzo1to4tp 13484 | A half-open integer range from 1 to 4 is an unordered triple. (Contributed by AV, 28-Jul-2021.) |
⊢ (1..^4) = {1, 2, 3} | ||
Theorem | fzo0sn0fzo1 13485 | A half-open range of nonnegative integers is the union of the singleton set containing 0 and a half-open range of positive integers. (Contributed by Alexander van der Vekens, 18-May-2018.) |
⊢ (𝑁 ∈ ℕ → (0..^𝑁) = ({0} ∪ (1..^𝑁))) | ||
Theorem | elfzo0l 13486 | A member of a half-open range of nonnegative integers is either 0 or a member of the corresponding half-open range of positive integers. (Contributed by AV, 5-Feb-2021.) |
⊢ (𝐾 ∈ (0..^𝑁) → (𝐾 = 0 ∨ 𝐾 ∈ (1..^𝑁))) | ||
Theorem | fzoend 13487 | The endpoint of a half-open integer range. (Contributed by Mario Carneiro, 29-Sep-2015.) |
⊢ (𝐴 ∈ (𝐴..^𝐵) → (𝐵 − 1) ∈ (𝐴..^𝐵)) | ||
Theorem | fzo0end 13488 | The endpoint of a zero-based half-open range. (Contributed by Stefan O'Rear, 27-Aug-2015.) (Revised by Mario Carneiro, 29-Sep-2015.) |
⊢ (𝐵 ∈ ℕ → (𝐵 − 1) ∈ (0..^𝐵)) | ||
Theorem | ssfzo12 13489 | Subset relationship for half-open integer ranges. (Contributed by Alexander van der Vekens, 16-Mar-2018.) |
⊢ ((𝐾 ∈ ℤ ∧ 𝐿 ∈ ℤ ∧ 𝐾 < 𝐿) → ((𝐾..^𝐿) ⊆ (𝑀..^𝑁) → (𝑀 ≤ 𝐾 ∧ 𝐿 ≤ 𝑁))) | ||
Theorem | ssfzoulel 13490 | If a half-open integer range is a subset of a half-open range of nonnegative integers, but its lower bound is greater than or equal to the upper bound of the containing range, or its upper bound is less than or equal to 0, then its upper bound is less than or equal to its lower bound (and therefore it is actually empty). (Contributed by Alexander van der Vekens, 24-May-2018.) |
⊢ ((𝑁 ∈ ℕ0 ∧ 𝐴 ∈ ℤ ∧ 𝐵 ∈ ℤ) → ((𝑁 ≤ 𝐴 ∨ 𝐵 ≤ 0) → ((𝐴..^𝐵) ⊆ (0..^𝑁) → 𝐵 ≤ 𝐴))) | ||
Theorem | ssfzo12bi 13491 | Subset relationship for half-open integer ranges. (Contributed by Alexander van der Vekens, 5-Nov-2018.) |
⊢ (((𝐾 ∈ ℤ ∧ 𝐿 ∈ ℤ) ∧ (𝑀 ∈ ℤ ∧ 𝑁 ∈ ℤ) ∧ 𝐾 < 𝐿) → ((𝐾..^𝐿) ⊆ (𝑀..^𝑁) ↔ (𝑀 ≤ 𝐾 ∧ 𝐿 ≤ 𝑁))) | ||
Theorem | ubmelm1fzo 13492 | The result of subtracting 1 and an integer of a half-open range of nonnegative integers from the upper bound of this range is contained in this range. (Contributed by AV, 23-Mar-2018.) (Revised by AV, 30-Oct-2018.) |
⊢ (𝐾 ∈ (0..^𝑁) → ((𝑁 − 𝐾) − 1) ∈ (0..^𝑁)) | ||
Theorem | fzofzp1 13493 | If a point is in a half-open range, the next point is in the closed range. (Contributed by Stefan O'Rear, 23-Aug-2015.) |
⊢ (𝐶 ∈ (𝐴..^𝐵) → (𝐶 + 1) ∈ (𝐴...𝐵)) | ||
Theorem | fzofzp1b 13494 | If a point is in a half-open range, the next point is in the closed range. (Contributed by Mario Carneiro, 27-Sep-2015.) |
⊢ (𝐶 ∈ (ℤ≥‘𝐴) → (𝐶 ∈ (𝐴..^𝐵) ↔ (𝐶 + 1) ∈ (𝐴...𝐵))) | ||
Theorem | elfzom1b 13495 | An integer is a member of a 1-based finite set of sequential integers iff its predecessor is a member of the corresponding 0-based set. (Contributed by Mario Carneiro, 27-Sep-2015.) |
⊢ ((𝐾 ∈ ℤ ∧ 𝑁 ∈ ℤ) → (𝐾 ∈ (1..^𝑁) ↔ (𝐾 − 1) ∈ (0..^(𝑁 − 1)))) | ||
Theorem | elfzom1elp1fzo1 13496 | Membership of a nonnegative integer incremented by one in a half-open range of positive integers. (Contributed by AV, 20-Mar-2021.) |
⊢ ((𝑁 ∈ ℤ ∧ 𝐼 ∈ (0..^(𝑁 − 1))) → (𝐼 + 1) ∈ (1..^𝑁)) | ||
Theorem | elfzo1elm1fzo0 13497 | Membership of a positive integer decremented by one in a half-open range of nonnegative integers. (Contributed by AV, 20-Mar-2021.) |
⊢ (𝐼 ∈ (1..^𝑁) → (𝐼 − 1) ∈ (0..^(𝑁 − 1))) | ||
Theorem | elfzonelfzo 13498 | If an element of a half-open integer range is not contained in the lower subrange, it must be in the upper subrange. (Contributed by Alexander van der Vekens, 30-Mar-2018.) |
⊢ (𝑁 ∈ ℤ → ((𝐾 ∈ (𝑀..^𝑅) ∧ ¬ 𝐾 ∈ (𝑀..^𝑁)) → 𝐾 ∈ (𝑁..^𝑅))) | ||
Theorem | fzonfzoufzol 13499 | If an element of a half-open integer range is not in the upper part of the range, it is in the lower part of the range. (Contributed by Alexander van der Vekens, 29-Oct-2018.) |
⊢ ((𝑀 ∈ ℤ ∧ 𝑀 < 𝑁 ∧ 𝐼 ∈ (0..^𝑁)) → (¬ 𝐼 ∈ ((𝑁 − 𝑀)..^𝑁) → 𝐼 ∈ (0..^(𝑁 − 𝑀)))) | ||
Theorem | elfzomelpfzo 13500 | An integer increased by another integer is an element of a half-open integer range if and only if the integer is contained in the half-open integer range with bounds decreased by the other integer. (Contributed by Alexander van der Vekens, 30-Mar-2018.) |
⊢ (((𝑀 ∈ ℤ ∧ 𝑁 ∈ ℤ) ∧ (𝐾 ∈ ℤ ∧ 𝐿 ∈ ℤ)) → (𝐾 ∈ ((𝑀 − 𝐿)..^(𝑁 − 𝐿)) ↔ (𝐾 + 𝐿) ∈ (𝑀..^𝑁))) |
< Previous Next > |
Copyright terms: Public domain | < Previous Next > |