Theorem List for Intuitionistic Logic Explorer - 10901-11000 *Has distinct variable
group(s)
| Type | Label | Description |
| Statement |
| |
| Theorem | prhash2ex 10901 |
There is (at least) one set with two different elements: the unordered
pair containing 0 and 1.
In contrast to pr0hash2ex 10907, numbers
are used instead of sets because their representation is shorter (and more
comprehensive). (Contributed by AV, 29-Jan-2020.)
|
| ⊢ (♯‘{0, 1}) = 2 |
| |
| Theorem | hashp1i 10902 |
Size of a natural number ordinal. (Contributed by Mario Carneiro,
5-Jan-2016.)
|
| ⊢ 𝐴 ∈ ω & ⊢ 𝐵 = suc 𝐴
& ⊢ (♯‘𝐴) = 𝑀
& ⊢ (𝑀 + 1) = 𝑁 ⇒ ⊢ (♯‘𝐵) = 𝑁 |
| |
| Theorem | hash1 10903 |
Size of a natural number ordinal. (Contributed by Mario Carneiro,
5-Jan-2016.)
|
| ⊢ (♯‘1o) =
1 |
| |
| Theorem | hash2 10904 |
Size of a natural number ordinal. (Contributed by Mario Carneiro,
5-Jan-2016.)
|
| ⊢ (♯‘2o) =
2 |
| |
| Theorem | hash3 10905 |
Size of a natural number ordinal. (Contributed by Mario Carneiro,
5-Jan-2016.)
|
| ⊢ (♯‘3o) =
3 |
| |
| Theorem | hash4 10906 |
Size of a natural number ordinal. (Contributed by Mario Carneiro,
5-Jan-2016.)
|
| ⊢ (♯‘4o) =
4 |
| |
| Theorem | pr0hash2ex 10907 |
There is (at least) one set with two different elements: the unordered
pair containing the empty set and the singleton containing the empty set.
(Contributed by AV, 29-Jan-2020.)
|
| ⊢ (♯‘{∅, {∅}}) =
2 |
| |
| Theorem | fihashss 10908 |
The size of a subset is less than or equal to the size of its superset.
(Contributed by Alexander van der Vekens, 14-Jul-2018.)
|
| ⊢ ((𝐴 ∈ Fin ∧ 𝐵 ∈ Fin ∧ 𝐵 ⊆ 𝐴) → (♯‘𝐵) ≤ (♯‘𝐴)) |
| |
| Theorem | fiprsshashgt1 10909 |
The size of a superset of a proper unordered pair is greater than 1.
(Contributed by AV, 6-Feb-2021.)
|
| ⊢ (((𝐴 ∈ 𝑉 ∧ 𝐵 ∈ 𝑊 ∧ 𝐴 ≠ 𝐵) ∧ 𝐶 ∈ Fin) → ({𝐴, 𝐵} ⊆ 𝐶 → 2 ≤ (♯‘𝐶))) |
| |
| Theorem | fihashssdif 10910 |
The size of the difference of a finite set and a finite subset is the
set's size minus the subset's. (Contributed by Jim Kingdon,
31-May-2022.)
|
| ⊢ ((𝐴 ∈ Fin ∧ 𝐵 ∈ Fin ∧ 𝐵 ⊆ 𝐴) → (♯‘(𝐴 ∖ 𝐵)) = ((♯‘𝐴) − (♯‘𝐵))) |
| |
| Theorem | hashdifsn 10911 |
The size of the difference of a finite set and a singleton subset is the
set's size minus 1. (Contributed by Alexander van der Vekens,
6-Jan-2018.)
|
| ⊢ ((𝐴 ∈ Fin ∧ 𝐵 ∈ 𝐴) → (♯‘(𝐴 ∖ {𝐵})) = ((♯‘𝐴) − 1)) |
| |
| Theorem | hashdifpr 10912 |
The size of the difference of a finite set and a proper ordered pair
subset is the set's size minus 2. (Contributed by AV, 16-Dec-2020.)
|
| ⊢ ((𝐴 ∈ Fin ∧ (𝐵 ∈ 𝐴 ∧ 𝐶 ∈ 𝐴 ∧ 𝐵 ≠ 𝐶)) → (♯‘(𝐴 ∖ {𝐵, 𝐶})) = ((♯‘𝐴) − 2)) |
| |
| Theorem | hashfz 10913 |
Value of the numeric cardinality of a nonempty integer range.
(Contributed by Stefan O'Rear, 12-Sep-2014.) (Proof shortened by Mario
Carneiro, 15-Apr-2015.)
|
| ⊢ (𝐵 ∈ (ℤ≥‘𝐴) → (♯‘(𝐴...𝐵)) = ((𝐵 − 𝐴) + 1)) |
| |
| Theorem | hashfzo 10914 |
Cardinality of a half-open set of integers. (Contributed by Stefan
O'Rear, 15-Aug-2015.)
|
| ⊢ (𝐵 ∈ (ℤ≥‘𝐴) → (♯‘(𝐴..^𝐵)) = (𝐵 − 𝐴)) |
| |
| Theorem | hashfzo0 10915 |
Cardinality of a half-open set of integers based at zero. (Contributed by
Stefan O'Rear, 15-Aug-2015.)
|
| ⊢ (𝐵 ∈ ℕ0 →
(♯‘(0..^𝐵)) =
𝐵) |
| |
| Theorem | hashfzp1 10916 |
Value of the numeric cardinality of a (possibly empty) integer range.
(Contributed by AV, 19-Jun-2021.)
|
| ⊢ (𝐵 ∈ (ℤ≥‘𝐴) → (♯‘((𝐴 + 1)...𝐵)) = (𝐵 − 𝐴)) |
| |
| Theorem | hashfz0 10917 |
Value of the numeric cardinality of a nonempty range of nonnegative
integers. (Contributed by Alexander van der Vekens, 21-Jul-2018.)
|
| ⊢ (𝐵 ∈ ℕ0 →
(♯‘(0...𝐵)) =
(𝐵 + 1)) |
| |
| Theorem | hashxp 10918 |
The size of the Cartesian product of two finite sets is the product of
their sizes. (Contributed by Paul Chapman, 30-Nov-2012.)
|
| ⊢ ((𝐴 ∈ Fin ∧ 𝐵 ∈ Fin) → (♯‘(𝐴 × 𝐵)) = ((♯‘𝐴) · (♯‘𝐵))) |
| |
| Theorem | fimaxq 10919* |
A finite set of rational numbers has a maximum. (Contributed by Jim
Kingdon, 6-Sep-2022.)
|
| ⊢ ((𝐴 ⊆ ℚ ∧ 𝐴 ∈ Fin ∧ 𝐴 ≠ ∅) → ∃𝑥 ∈ 𝐴 ∀𝑦 ∈ 𝐴 𝑦 ≤ 𝑥) |
| |
| Theorem | fiubm 10920* |
Lemma for fiubz 10921 and fiubnn 10922. A general form of those theorems.
(Contributed by Jim Kingdon, 29-Oct-2024.)
|
| ⊢ (𝜑 → 𝐴 ⊆ 𝐵)
& ⊢ (𝜑 → 𝐵 ⊆ ℚ) & ⊢ (𝜑 → 𝐶 ∈ 𝐵)
& ⊢ (𝜑 → 𝐴 ∈ Fin) ⇒ ⊢ (𝜑 → ∃𝑥 ∈ 𝐵 ∀𝑦 ∈ 𝐴 𝑦 ≤ 𝑥) |
| |
| Theorem | fiubz 10921* |
A finite set of integers has an upper bound which is an integer.
(Contributed by Jim Kingdon, 29-Oct-2024.)
|
| ⊢ ((𝐴 ⊆ ℤ ∧ 𝐴 ∈ Fin) → ∃𝑥 ∈ ℤ ∀𝑦 ∈ 𝐴 𝑦 ≤ 𝑥) |
| |
| Theorem | fiubnn 10922* |
A finite set of natural numbers has an upper bound which is a a natural
number. (Contributed by Jim Kingdon, 29-Oct-2024.)
|
| ⊢ ((𝐴 ⊆ ℕ ∧ 𝐴 ∈ Fin) → ∃𝑥 ∈ ℕ ∀𝑦 ∈ 𝐴 𝑦 ≤ 𝑥) |
| |
| Theorem | resunimafz0 10923 |
The union of a restriction by an image over an open range of nonnegative
integers and a singleton of an ordered pair is a restriction by an image
over an interval of nonnegative integers. (Contributed by Mario
Carneiro, 8-Apr-2015.) (Revised by AV, 20-Feb-2021.)
|
| ⊢ (𝜑 → Fun 𝐼)
& ⊢ (𝜑 → 𝐹:(0..^(♯‘𝐹))⟶dom 𝐼)
& ⊢ (𝜑 → 𝑁 ∈ (0..^(♯‘𝐹)))
⇒ ⊢ (𝜑 → (𝐼 ↾ (𝐹 “ (0...𝑁))) = ((𝐼 ↾ (𝐹 “ (0..^𝑁))) ∪ {〈(𝐹‘𝑁), (𝐼‘(𝐹‘𝑁))〉})) |
| |
| Theorem | fnfz0hash 10924 |
The size of a function on a finite set of sequential nonnegative integers.
(Contributed by Alexander van der Vekens, 25-Jun-2018.)
|
| ⊢ ((𝑁 ∈ ℕ0 ∧ 𝐹 Fn (0...𝑁)) → (♯‘𝐹) = (𝑁 + 1)) |
| |
| Theorem | ffz0hash 10925 |
The size of a function on a finite set of sequential nonnegative integers
equals the upper bound of the sequence increased by 1. (Contributed by
Alexander van der Vekens, 15-Mar-2018.) (Proof shortened by AV,
11-Apr-2021.)
|
| ⊢ ((𝑁 ∈ ℕ0 ∧ 𝐹:(0...𝑁)⟶𝐵) → (♯‘𝐹) = (𝑁 + 1)) |
| |
| Theorem | ffzo0hash 10926 |
The size of a function on a half-open range of nonnegative integers.
(Contributed by Alexander van der Vekens, 25-Mar-2018.)
|
| ⊢ ((𝑁 ∈ ℕ0 ∧ 𝐹 Fn (0..^𝑁)) → (♯‘𝐹) = 𝑁) |
| |
| Theorem | fnfzo0hash 10927 |
The size of a function on a half-open range of nonnegative integers equals
the upper bound of this range. (Contributed by Alexander van der Vekens,
26-Jan-2018.) (Proof shortened by AV, 11-Apr-2021.)
|
| ⊢ ((𝑁 ∈ ℕ0 ∧ 𝐹:(0..^𝑁)⟶𝐵) → (♯‘𝐹) = 𝑁) |
| |
| Theorem | hashfacen 10928* |
The number of bijections between two sets is a cardinal invariant.
(Contributed by Mario Carneiro, 21-Jan-2015.)
|
| ⊢ ((𝐴 ≈ 𝐵 ∧ 𝐶 ≈ 𝐷) → {𝑓 ∣ 𝑓:𝐴–1-1-onto→𝐶} ≈ {𝑓 ∣ 𝑓:𝐵–1-1-onto→𝐷}) |
| |
| Theorem | leisorel 10929 |
Version of isorel 5855 for strictly increasing functions on the
reals.
(Contributed by Mario Carneiro, 6-Apr-2015.) (Revised by Mario Carneiro,
9-Sep-2015.)
|
| ⊢ ((𝐹 Isom < , < (𝐴, 𝐵) ∧ (𝐴 ⊆ ℝ* ∧ 𝐵 ⊆ ℝ*)
∧ (𝐶 ∈ 𝐴 ∧ 𝐷 ∈ 𝐴)) → (𝐶 ≤ 𝐷 ↔ (𝐹‘𝐶) ≤ (𝐹‘𝐷))) |
| |
| Theorem | zfz1isolemsplit 10930 |
Lemma for zfz1iso 10933. Removing one element from an integer
range.
(Contributed by Jim Kingdon, 8-Sep-2022.)
|
| ⊢ (𝜑 → 𝑋 ∈ Fin) & ⊢ (𝜑 → 𝑀 ∈ 𝑋) ⇒ ⊢ (𝜑 → (1...(♯‘𝑋)) =
((1...(♯‘(𝑋
∖ {𝑀}))) ∪
{(♯‘𝑋)})) |
| |
| Theorem | zfz1isolemiso 10931* |
Lemma for zfz1iso 10933. Adding one element to the order
isomorphism.
(Contributed by Jim Kingdon, 8-Sep-2022.)
|
| ⊢ (𝜑 → 𝑋 ∈ Fin) & ⊢ (𝜑 → 𝑋 ⊆ ℤ) & ⊢ (𝜑 → 𝑀 ∈ 𝑋)
& ⊢ (𝜑 → ∀𝑧 ∈ 𝑋 𝑧 ≤ 𝑀)
& ⊢ (𝜑 → 𝐺 Isom < , <
((1...(♯‘(𝑋
∖ {𝑀}))), (𝑋 ∖ {𝑀}))) & ⊢ (𝜑 → 𝐴 ∈ (1...(♯‘𝑋))) & ⊢ (𝜑 → 𝐵 ∈ (1...(♯‘𝑋)))
⇒ ⊢ (𝜑 → (𝐴 < 𝐵 ↔ ((𝐺 ∪ {〈(♯‘𝑋), 𝑀〉})‘𝐴) < ((𝐺 ∪ {〈(♯‘𝑋), 𝑀〉})‘𝐵))) |
| |
| Theorem | zfz1isolem1 10932* |
Lemma for zfz1iso 10933. Existence of an order isomorphism given
the
existence of shorter isomorphisms. (Contributed by Jim Kingdon,
7-Sep-2022.)
|
| ⊢ (𝜑 → 𝐾 ∈ ω) & ⊢ (𝜑 → ∀𝑦(((𝑦 ⊆ ℤ ∧ 𝑦 ∈ Fin) ∧ 𝑦 ≈ 𝐾) → ∃𝑓 𝑓 Isom < , < ((1...(♯‘𝑦)), 𝑦))) & ⊢ (𝜑 → 𝑋 ⊆ ℤ) & ⊢ (𝜑 → 𝑋 ∈ Fin) & ⊢ (𝜑 → 𝑋 ≈ suc 𝐾)
& ⊢ (𝜑 → 𝑀 ∈ 𝑋)
& ⊢ (𝜑 → ∀𝑧 ∈ 𝑋 𝑧 ≤ 𝑀) ⇒ ⊢ (𝜑 → ∃𝑓 𝑓 Isom < , < ((1...(♯‘𝑋)), 𝑋)) |
| |
| Theorem | zfz1iso 10933* |
A finite set of integers has an order isomorphism to a one-based finite
sequence. (Contributed by Jim Kingdon, 3-Sep-2022.)
|
| ⊢ ((𝐴 ⊆ ℤ ∧ 𝐴 ∈ Fin) → ∃𝑓 𝑓 Isom < , < ((1...(♯‘𝐴)), 𝐴)) |
| |
| Theorem | seq3coll 10934* |
The function 𝐹 contains a sparse set of nonzero
values to be summed.
The function 𝐺 is an order isomorphism from the set
of nonzero
values of 𝐹 to a 1-based finite sequence, and
𝐻
collects these
nonzero values together. Under these conditions, the sum over the
values in 𝐻 yields the same result as the sum
over the original set
𝐹. (Contributed by Mario Carneiro,
2-Apr-2014.) (Revised by Jim
Kingdon, 9-Apr-2023.)
|
| ⊢ ((𝜑 ∧ 𝑘 ∈ 𝑆) → (𝑍 + 𝑘) = 𝑘)
& ⊢ ((𝜑 ∧ 𝑘 ∈ 𝑆) → (𝑘 + 𝑍) = 𝑘)
& ⊢ ((𝜑 ∧ (𝑘 ∈ 𝑆 ∧ 𝑛 ∈ 𝑆)) → (𝑘 + 𝑛) ∈ 𝑆)
& ⊢ (𝜑 → 𝑍 ∈ 𝑆)
& ⊢ (𝜑 → 𝐺 Isom < , <
((1...(♯‘𝐴)),
𝐴)) & ⊢ (𝜑 → 𝑁 ∈ (1...(♯‘𝐴))) & ⊢ (𝜑 → 𝐴 ⊆
(ℤ≥‘𝑀)) & ⊢ ((𝜑 ∧ 𝑘 ∈ (ℤ≥‘𝑀)) → (𝐹‘𝑘) ∈ 𝑆)
& ⊢ ((𝜑 ∧ 𝑘 ∈ (ℤ≥‘1))
→ (𝐻‘𝑘) ∈ 𝑆)
& ⊢ ((𝜑 ∧ 𝑘 ∈ ((𝑀...(𝐺‘(♯‘𝐴))) ∖ 𝐴)) → (𝐹‘𝑘) = 𝑍)
& ⊢ ((𝜑 ∧ 𝑛 ∈ (1...(♯‘𝐴))) → (𝐻‘𝑛) = (𝐹‘(𝐺‘𝑛))) ⇒ ⊢ (𝜑 → (seq𝑀( + , 𝐹)‘(𝐺‘𝑁)) = (seq1( + , 𝐻)‘𝑁)) |
| |
| 4.7 Words over a set
This section is about words (or strings) over a set (alphabet) defined
as finite sequences of symbols (or characters) being elements of the
alphabet. Although it is often required that the underlying set/alphabet be
nonempty, finite and not a proper class, these restrictions are not made in
the current definition df-word 10936. Note that the empty word ∅ (i.e.,
the empty set) is the only word over an empty alphabet, see 0wrd0 10961.
The set Word 𝑆 of words over 𝑆 is the free monoid over 𝑆, where
the monoid law is concatenation and the monoid unit is the empty word.
Besides the definition of words themselves, several operations on words are
defined in this section:
| Name | Reference | Explanation | Example |
Remarks |
| Length (or size) of a word | df-ihash 10868: (♯‘𝑊) |
Operation which determines the number of the symbols
within the word. |
𝑊:(0..^𝑁)⟶𝑆 → (𝑊 ∈ Word 𝑆 ∧ (♯‘𝑊) = 𝑁 |
This is not a special definition for words,
but for arbitrary sets. |
| First symbol of a word | df-fv 5266: (𝑊‘0) |
Operation which extracts the first symbol of a word. The result is the
symbol at the first place in the sequence representing the word. |
𝑊:(0..^1)⟶𝑆 → (𝑊 ∈ Word 𝑆 ∧ (𝑊‘0) ∈ 𝑆 |
This is not a special definition for words,
but for arbitrary functions with a half-open range of nonnegative
integers as domain. |
Conventions:
- Words are usually represented by class variable 𝑊, or if two words
are involved, by 𝑊 and 𝑈 or by 𝐴 and 𝐵.
- The alphabets are usually represented by class variable 𝑉 (because
any arbitrary set can be an alphabet), sometimes also by 𝑆 (especially
as codomain of the function representing a word, because the alphabet is the
set of symbols).
- The symbols are usually represented by class variables 𝑆 or 𝐴,
or if two symbols are involved, by 𝑆 and 𝑇 or by 𝐴 and 𝐵.
- The indices of the sequence representing a word are usually represented
by class variable 𝐼, if two indices are involved (especially for
subwords) by 𝐼 and 𝐽, or by 𝑀 and 𝑁.
- The length of a word is usually represented by class variables 𝑁
or 𝐿.
- The number of positions by which to cyclically shift a word is usually
represented by class variables 𝑁 or 𝐿.
|
| |
| 4.7.1 Definitions and basic
theorems
|
| |
| Syntax | cword 10935 |
Syntax for the Word operator.
|
| class Word 𝑆 |
| |
| Definition | df-word 10936* |
Define the class of words over a set. A word (sometimes also called a
string) is a finite sequence of symbols from a set (alphabet)
𝑆.
Definition in Section 9.1 of [AhoHopUll] p. 318. The domain is forced
to be an initial segment of ℕ0
so that two words with the same
symbols in the same order be equal. The set Word 𝑆 is sometimes
denoted by S*, using the Kleene star, although the Kleene star, or
Kleene closure, is sometimes reserved to denote an operation on
languages. The set Word 𝑆 equipped with concatenation is the
free
monoid over 𝑆, and the monoid unit is the empty
word. (Contributed
by FL, 14-Jan-2014.) (Revised by Stefan O'Rear, 14-Aug-2015.) (Revised
by Mario Carneiro, 26-Feb-2016.)
|
| ⊢ Word 𝑆 = {𝑤 ∣ ∃𝑙 ∈ ℕ0 𝑤:(0..^𝑙)⟶𝑆} |
| |
| Theorem | iswrd 10937* |
Property of being a word over a set with an existential quantifier over
the length. (Contributed by Stefan O'Rear, 15-Aug-2015.) (Revised by
Mario Carneiro, 26-Feb-2016.) (Proof shortened by AV, 13-May-2020.)
|
| ⊢ (𝑊 ∈ Word 𝑆 ↔ ∃𝑙 ∈ ℕ0 𝑊:(0..^𝑙)⟶𝑆) |
| |
| Theorem | wrdval 10938* |
Value of the set of words over a set. (Contributed by Stefan O'Rear,
10-Aug-2015.) (Revised by Mario Carneiro, 26-Feb-2016.)
|
| ⊢ (𝑆 ∈ 𝑉 → Word 𝑆 = ∪
𝑙 ∈
ℕ0 (𝑆
↑𝑚 (0..^𝑙))) |
| |
| Theorem | lencl 10939 |
The length of a word is a nonnegative integer. This corresponds to the
definition in Section 9.1 of [AhoHopUll] p. 318. (Contributed by Stefan
O'Rear, 27-Aug-2015.)
|
| ⊢ (𝑊 ∈ Word 𝑆 → (♯‘𝑊) ∈
ℕ0) |
| |
| Theorem | iswrdinn0 10940 |
A zero-based sequence is a word. (Contributed by Stefan O'Rear,
15-Aug-2015.) (Revised by Mario Carneiro, 26-Feb-2016.) (Revised by
Jim Kingdon, 16-Aug-2025.)
|
| ⊢ ((𝑊:(0..^𝐿)⟶𝑆 ∧ 𝐿 ∈ ℕ0) → 𝑊 ∈ Word 𝑆) |
| |
| Theorem | wrdf 10941 |
A word is a zero-based sequence with a recoverable upper limit.
(Contributed by Stefan O'Rear, 15-Aug-2015.)
|
| ⊢ (𝑊 ∈ Word 𝑆 → 𝑊:(0..^(♯‘𝑊))⟶𝑆) |
| |
| Theorem | iswrdiz 10942 |
A zero-based sequence is a word. In iswrdinn0 10940 we can specify a length
as an nonnegative integer. However, it will occasionally be helpful to
allow a negative length, as well as zero, to specify an empty sequence.
(Contributed by Jim Kingdon, 18-Aug-2025.)
|
| ⊢ ((𝑊:(0..^𝐿)⟶𝑆 ∧ 𝐿 ∈ ℤ) → 𝑊 ∈ Word 𝑆) |
| |
| Theorem | wrddm 10943 |
The indices of a word (i.e. its domain regarded as function) are elements
of an open range of nonnegative integers (of length equal to the length of
the word). (Contributed by AV, 2-May-2020.)
|
| ⊢ (𝑊 ∈ Word 𝑆 → dom 𝑊 = (0..^(♯‘𝑊))) |
| |
| Theorem | sswrd 10944 |
The set of words respects ordering on the base set. (Contributed by
Stefan O'Rear, 15-Aug-2015.) (Revised by Mario Carneiro, 26-Feb-2016.)
(Proof shortened by AV, 13-May-2020.)
|
| ⊢ (𝑆 ⊆ 𝑇 → Word 𝑆 ⊆ Word 𝑇) |
| |
| Theorem | snopiswrd 10945 |
A singleton of an ordered pair (with 0 as first component) is a word.
(Contributed by AV, 23-Nov-2018.) (Proof shortened by AV,
18-Apr-2021.)
|
| ⊢ (𝑆 ∈ 𝑉 → {〈0, 𝑆〉} ∈ Word 𝑉) |
| |
| Theorem | wrdexg 10946 |
The set of words over a set is a set. (Contributed by Mario Carneiro,
26-Feb-2016.) (Proof shortened by JJ, 18-Nov-2022.)
|
| ⊢ (𝑆 ∈ 𝑉 → Word 𝑆 ∈ V) |
| |
| Theorem | wrdexb 10947 |
The set of words over a set is a set, bidirectional version.
(Contributed by Mario Carneiro, 26-Feb-2016.) (Proof shortened by AV,
23-Nov-2018.)
|
| ⊢ (𝑆 ∈ V ↔ Word 𝑆 ∈ V) |
| |
| Theorem | wrdexi 10948 |
The set of words over a set is a set, inference form. (Contributed by
AV, 23-May-2021.)
|
| ⊢ 𝑆 ∈ V ⇒ ⊢ Word 𝑆 ∈ V |
| |
| Theorem | wrdsymbcl 10949 |
A symbol within a word over an alphabet belongs to the alphabet.
(Contributed by Alexander van der Vekens, 28-Jun-2018.)
|
| ⊢ ((𝑊 ∈ Word 𝑉 ∧ 𝐼 ∈ (0..^(♯‘𝑊))) → (𝑊‘𝐼) ∈ 𝑉) |
| |
| Theorem | wrdfn 10950 |
A word is a function with a zero-based sequence of integers as domain.
(Contributed by Alexander van der Vekens, 13-Apr-2018.)
|
| ⊢ (𝑊 ∈ Word 𝑆 → 𝑊 Fn (0..^(♯‘𝑊))) |
| |
| Theorem | wrdv 10951 |
A word over an alphabet is a word over the universal class. (Contributed
by AV, 8-Feb-2021.) (Proof shortened by JJ, 18-Nov-2022.)
|
| ⊢ (𝑊 ∈ Word 𝑉 → 𝑊 ∈ Word V) |
| |
| Theorem | wrdlndm 10952 |
The length of a word is not in the domain of the word (regarded as a
function). (Contributed by AV, 3-Mar-2021.) (Proof shortened by JJ,
18-Nov-2022.)
|
| ⊢ (𝑊 ∈ Word 𝑉 → (♯‘𝑊) ∉ dom 𝑊) |
| |
| Theorem | iswrdsymb 10953* |
An arbitrary word is a word over an alphabet if all of its symbols
belong to the alphabet. (Contributed by AV, 23-Jan-2021.)
|
| ⊢ ((𝑊 ∈ Word V ∧ ∀𝑖 ∈
(0..^(♯‘𝑊))(𝑊‘𝑖) ∈ 𝑉) → 𝑊 ∈ Word 𝑉) |
| |
| Theorem | wrdfin 10954 |
A word is a finite set. (Contributed by Stefan O'Rear, 2-Nov-2015.)
(Proof shortened by AV, 18-Nov-2018.)
|
| ⊢ (𝑊 ∈ Word 𝑆 → 𝑊 ∈ Fin) |
| |
| Theorem | lennncl 10955 |
The length of a nonempty word is a positive integer. (Contributed by
Mario Carneiro, 1-Oct-2015.)
|
| ⊢ ((𝑊 ∈ Word 𝑆 ∧ 𝑊 ≠ ∅) → (♯‘𝑊) ∈
ℕ) |
| |
| Theorem | wrdffz 10956 |
A word is a function from a finite interval of integers. (Contributed by
AV, 10-Feb-2021.)
|
| ⊢ (𝑊 ∈ Word 𝑆 → 𝑊:(0...((♯‘𝑊) − 1))⟶𝑆) |
| |
| Theorem | wrdeq 10957 |
Equality theorem for the set of words. (Contributed by Mario Carneiro,
26-Feb-2016.)
|
| ⊢ (𝑆 = 𝑇 → Word 𝑆 = Word 𝑇) |
| |
| Theorem | wrdeqi 10958 |
Equality theorem for the set of words, inference form. (Contributed by
AV, 23-May-2021.)
|
| ⊢ 𝑆 = 𝑇 ⇒ ⊢ Word 𝑆 = Word 𝑇 |
| |
| Theorem | iswrddm0 10959 |
A function with empty domain is a word. (Contributed by AV,
13-Oct-2018.)
|
| ⊢ (𝑊:∅⟶𝑆 → 𝑊 ∈ Word 𝑆) |
| |
| Theorem | wrd0 10960 |
The empty set is a word (the empty word, frequently denoted ε in
this context). This corresponds to the definition in Section 9.1 of
[AhoHopUll] p. 318. (Contributed by
Stefan O'Rear, 15-Aug-2015.) (Proof
shortened by AV, 13-May-2020.)
|
| ⊢ ∅ ∈ Word 𝑆 |
| |
| Theorem | 0wrd0 10961 |
The empty word is the only word over an empty alphabet. (Contributed by
AV, 25-Oct-2018.)
|
| ⊢ (𝑊 ∈ Word ∅ ↔ 𝑊 = ∅) |
| |
| Theorem | wrdsymb 10962 |
A word is a word over the symbols it consists of. (Contributed by AV,
1-Dec-2022.)
|
| ⊢ (𝑆 ∈ Word 𝐴 → 𝑆 ∈ Word (𝑆 “ (0..^(♯‘𝑆)))) |
| |
| Theorem | nfwrd 10963 |
Hypothesis builder for Word 𝑆. (Contributed by Mario Carneiro,
26-Feb-2016.)
|
| ⊢ Ⅎ𝑥𝑆 ⇒ ⊢ Ⅎ𝑥Word 𝑆 |
| |
| Theorem | csbwrdg 10964* |
Class substitution for the symbols of a word. (Contributed by Alexander
van der Vekens, 15-Jul-2018.)
|
| ⊢ (𝑆 ∈ 𝑉 → ⦋𝑆 / 𝑥⦌Word 𝑥 = Word 𝑆) |
| |
| Theorem | wrdnval 10965* |
Words of a fixed length are mappings from a fixed half-open integer
interval. (Contributed by Alexander van der Vekens, 25-Mar-2018.)
(Proof shortened by AV, 13-May-2020.)
|
| ⊢ ((𝑉 ∈ 𝑋 ∧ 𝑁 ∈ ℕ0) → {𝑤 ∈ Word 𝑉 ∣ (♯‘𝑤) = 𝑁} = (𝑉 ↑𝑚 (0..^𝑁))) |
| |
| Theorem | wrdmap 10966 |
Words as a mapping. (Contributed by Thierry Arnoux, 4-Mar-2020.)
|
| ⊢ ((𝑉 ∈ 𝑋 ∧ 𝑁 ∈ ℕ0) → ((𝑊 ∈ Word 𝑉 ∧ (♯‘𝑊) = 𝑁) ↔ 𝑊 ∈ (𝑉 ↑𝑚 (0..^𝑁)))) |
| |
| Theorem | wrdsymb0 10967 |
A symbol at a position "outside" of a word. (Contributed by
Alexander van
der Vekens, 26-May-2018.) (Proof shortened by AV, 2-May-2020.)
|
| ⊢ ((𝑊 ∈ Word 𝑉 ∧ 𝐼 ∈ ℤ) → ((𝐼 < 0 ∨ (♯‘𝑊) ≤ 𝐼) → (𝑊‘𝐼) = ∅)) |
| |
| Theorem | wrdlenge1n0 10968 |
A word with length at least 1 is not empty. (Contributed by AV,
14-Oct-2018.)
|
| ⊢ (𝑊 ∈ Word 𝑉 → (𝑊 ≠ ∅ ↔ 1 ≤
(♯‘𝑊))) |
| |
| Theorem | len0nnbi 10969 |
The length of a word is a positive integer iff the word is not empty.
(Contributed by AV, 22-Mar-2022.)
|
| ⊢ (𝑊 ∈ Word 𝑆 → (𝑊 ≠ ∅ ↔ (♯‘𝑊) ∈
ℕ)) |
| |
| Theorem | wrdlenge2n0 10970 |
A word with length at least 2 is not empty. (Contributed by AV,
18-Jun-2018.) (Proof shortened by AV, 14-Oct-2018.)
|
| ⊢ ((𝑊 ∈ Word 𝑉 ∧ 2 ≤ (♯‘𝑊)) → 𝑊 ≠ ∅) |
| |
| Theorem | wrdsymb1 10971 |
The first symbol of a nonempty word over an alphabet belongs to the
alphabet. (Contributed by Alexander van der Vekens, 28-Jun-2018.)
|
| ⊢ ((𝑊 ∈ Word 𝑉 ∧ 1 ≤ (♯‘𝑊)) → (𝑊‘0) ∈ 𝑉) |
| |
| Theorem | wrdlen1 10972* |
A word of length 1 starts with a symbol. (Contributed by AV,
20-Jul-2018.) (Proof shortened by AV, 19-Oct-2018.)
|
| ⊢ ((𝑊 ∈ Word 𝑉 ∧ (♯‘𝑊) = 1) → ∃𝑣 ∈ 𝑉 (𝑊‘0) = 𝑣) |
| |
| Theorem | fstwrdne 10973 |
The first symbol of a nonempty word is element of the alphabet for the
word. (Contributed by AV, 28-Sep-2018.) (Proof shortened by AV,
14-Oct-2018.)
|
| ⊢ ((𝑊 ∈ Word 𝑉 ∧ 𝑊 ≠ ∅) → (𝑊‘0) ∈ 𝑉) |
| |
| Theorem | fstwrdne0 10974 |
The first symbol of a nonempty word is element of the alphabet for the
word. (Contributed by AV, 29-Sep-2018.) (Proof shortened by AV,
14-Oct-2018.)
|
| ⊢ ((𝑁 ∈ ℕ ∧ (𝑊 ∈ Word 𝑉 ∧ (♯‘𝑊) = 𝑁)) → (𝑊‘0) ∈ 𝑉) |
| |
| Theorem | eqwrd 10975* |
Two words are equal iff they have the same length and the same symbol at
each position. (Contributed by AV, 13-Apr-2018.) (Revised by JJ,
30-Dec-2023.)
|
| ⊢ ((𝑈 ∈ Word 𝑆 ∧ 𝑊 ∈ Word 𝑇) → (𝑈 = 𝑊 ↔ ((♯‘𝑈) = (♯‘𝑊) ∧ ∀𝑖 ∈ (0..^(♯‘𝑈))(𝑈‘𝑖) = (𝑊‘𝑖)))) |
| |
| Theorem | elovmpowrd 10976* |
Implications for the value of an operation defined by the maps-to
notation with a class abstraction of words as a result having an
element. Note that 𝜑 may depend on 𝑧 as well as on 𝑣 and
𝑦. (Contributed by Alexander van der
Vekens, 15-Jul-2018.)
|
| ⊢ 𝑂 = (𝑣 ∈ V, 𝑦 ∈ V ↦ {𝑧 ∈ Word 𝑣 ∣ 𝜑}) ⇒ ⊢ (𝑍 ∈ (𝑉𝑂𝑌) → (𝑉 ∈ V ∧ 𝑌 ∈ V ∧ 𝑍 ∈ Word 𝑉)) |
| |
| Theorem | wrdred1 10977 |
A word truncated by a symbol is a word. (Contributed by AV,
29-Jan-2021.)
|
| ⊢ (𝐹 ∈ Word 𝑆 → (𝐹 ↾ (0..^((♯‘𝐹) − 1))) ∈ Word
𝑆) |
| |
| Theorem | wrdred1hash 10978 |
The length of a word truncated by a symbol. (Contributed by Alexander van
der Vekens, 1-Nov-2017.) (Revised by AV, 29-Jan-2021.)
|
| ⊢ ((𝐹 ∈ Word 𝑆 ∧ 1 ≤ (♯‘𝐹)) → (♯‘(𝐹 ↾
(0..^((♯‘𝐹)
− 1)))) = ((♯‘𝐹) − 1)) |
| |
| 4.8 Elementary real and complex
functions
|
| |
| 4.8.1 The "shift" operation
|
| |
| Syntax | cshi 10979 |
Extend class notation with function shifter.
|
| class shift |
| |
| Definition | df-shft 10980* |
Define a function shifter. This operation offsets the value argument of
a function (ordinarily on a subset of ℂ)
and produces a new
function on ℂ. See shftval 10990 for its value. (Contributed by NM,
20-Jul-2005.)
|
| ⊢ shift = (𝑓 ∈ V, 𝑥 ∈ ℂ ↦ {〈𝑦, 𝑧〉 ∣ (𝑦 ∈ ℂ ∧ (𝑦 − 𝑥)𝑓𝑧)}) |
| |
| Theorem | shftlem 10981* |
Two ways to write a shifted set (𝐵 + 𝐴). (Contributed by Mario
Carneiro, 3-Nov-2013.)
|
| ⊢ ((𝐴 ∈ ℂ ∧ 𝐵 ⊆ ℂ) → {𝑥 ∈ ℂ ∣ (𝑥 − 𝐴) ∈ 𝐵} = {𝑥 ∣ ∃𝑦 ∈ 𝐵 𝑥 = (𝑦 + 𝐴)}) |
| |
| Theorem | shftuz 10982* |
A shift of the upper integers. (Contributed by Mario Carneiro,
5-Nov-2013.)
|
| ⊢ ((𝐴 ∈ ℤ ∧ 𝐵 ∈ ℤ) → {𝑥 ∈ ℂ ∣ (𝑥 − 𝐴) ∈
(ℤ≥‘𝐵)} = (ℤ≥‘(𝐵 + 𝐴))) |
| |
| Theorem | shftfvalg 10983* |
The value of the sequence shifter operation is a function on ℂ.
𝐴 is ordinarily an integer.
(Contributed by NM, 20-Jul-2005.)
(Revised by Mario Carneiro, 3-Nov-2013.)
|
| ⊢ ((𝐴 ∈ ℂ ∧ 𝐹 ∈ 𝑉) → (𝐹 shift 𝐴) = {〈𝑥, 𝑦〉 ∣ (𝑥 ∈ ℂ ∧ (𝑥 − 𝐴)𝐹𝑦)}) |
| |
| Theorem | ovshftex 10984 |
Existence of the result of applying shift. (Contributed by Jim Kingdon,
15-Aug-2021.)
|
| ⊢ ((𝐹 ∈ 𝑉 ∧ 𝐴 ∈ ℂ) → (𝐹 shift 𝐴) ∈ V) |
| |
| Theorem | shftfibg 10985 |
Value of a fiber of the relation 𝐹. (Contributed by Jim Kingdon,
15-Aug-2021.)
|
| ⊢ ((𝐹 ∈ 𝑉 ∧ 𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ) → ((𝐹 shift 𝐴) “ {𝐵}) = (𝐹 “ {(𝐵 − 𝐴)})) |
| |
| Theorem | shftfval 10986* |
The value of the sequence shifter operation is a function on ℂ.
𝐴 is ordinarily an integer.
(Contributed by NM, 20-Jul-2005.)
(Revised by Mario Carneiro, 3-Nov-2013.)
|
| ⊢ 𝐹 ∈ V ⇒ ⊢ (𝐴 ∈ ℂ → (𝐹 shift 𝐴) = {〈𝑥, 𝑦〉 ∣ (𝑥 ∈ ℂ ∧ (𝑥 − 𝐴)𝐹𝑦)}) |
| |
| Theorem | shftdm 10987* |
Domain of a relation shifted by 𝐴. The set on the right is more
commonly notated as (dom 𝐹 + 𝐴) (meaning add 𝐴 to every
element of dom 𝐹). (Contributed by Mario Carneiro,
3-Nov-2013.)
|
| ⊢ 𝐹 ∈ V ⇒ ⊢ (𝐴 ∈ ℂ → dom (𝐹 shift 𝐴) = {𝑥 ∈ ℂ ∣ (𝑥 − 𝐴) ∈ dom 𝐹}) |
| |
| Theorem | shftfib 10988 |
Value of a fiber of the relation 𝐹. (Contributed by Mario
Carneiro, 4-Nov-2013.)
|
| ⊢ 𝐹 ∈ V ⇒ ⊢ ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ) → ((𝐹 shift 𝐴) “ {𝐵}) = (𝐹 “ {(𝐵 − 𝐴)})) |
| |
| Theorem | shftfn 10989* |
Functionality and domain of a sequence shifted by 𝐴. (Contributed
by NM, 20-Jul-2005.) (Revised by Mario Carneiro, 3-Nov-2013.)
|
| ⊢ 𝐹 ∈ V ⇒ ⊢ ((𝐹 Fn 𝐵 ∧ 𝐴 ∈ ℂ) → (𝐹 shift 𝐴) Fn {𝑥 ∈ ℂ ∣ (𝑥 − 𝐴) ∈ 𝐵}) |
| |
| Theorem | shftval 10990 |
Value of a sequence shifted by 𝐴. (Contributed by NM,
20-Jul-2005.) (Revised by Mario Carneiro, 4-Nov-2013.)
|
| ⊢ 𝐹 ∈ V ⇒ ⊢ ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ) → ((𝐹 shift 𝐴)‘𝐵) = (𝐹‘(𝐵 − 𝐴))) |
| |
| Theorem | shftval2 10991 |
Value of a sequence shifted by 𝐴 − 𝐵. (Contributed by NM,
20-Jul-2005.) (Revised by Mario Carneiro, 5-Nov-2013.)
|
| ⊢ 𝐹 ∈ V ⇒ ⊢ ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ ∧ 𝐶 ∈ ℂ) → ((𝐹 shift (𝐴 − 𝐵))‘(𝐴 + 𝐶)) = (𝐹‘(𝐵 + 𝐶))) |
| |
| Theorem | shftval3 10992 |
Value of a sequence shifted by 𝐴 − 𝐵. (Contributed by NM,
20-Jul-2005.)
|
| ⊢ 𝐹 ∈ V ⇒ ⊢ ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ) → ((𝐹 shift (𝐴 − 𝐵))‘𝐴) = (𝐹‘𝐵)) |
| |
| Theorem | shftval4 10993 |
Value of a sequence shifted by -𝐴. (Contributed by NM,
18-Aug-2005.) (Revised by Mario Carneiro, 5-Nov-2013.)
|
| ⊢ 𝐹 ∈ V ⇒ ⊢ ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ) → ((𝐹 shift -𝐴)‘𝐵) = (𝐹‘(𝐴 + 𝐵))) |
| |
| Theorem | shftval5 10994 |
Value of a shifted sequence. (Contributed by NM, 19-Aug-2005.)
(Revised by Mario Carneiro, 5-Nov-2013.)
|
| ⊢ 𝐹 ∈ V ⇒ ⊢ ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ) → ((𝐹 shift 𝐴)‘(𝐵 + 𝐴)) = (𝐹‘𝐵)) |
| |
| Theorem | shftf 10995* |
Functionality of a shifted sequence. (Contributed by NM, 19-Aug-2005.)
(Revised by Mario Carneiro, 5-Nov-2013.)
|
| ⊢ 𝐹 ∈ V ⇒ ⊢ ((𝐹:𝐵⟶𝐶 ∧ 𝐴 ∈ ℂ) → (𝐹 shift 𝐴):{𝑥 ∈ ℂ ∣ (𝑥 − 𝐴) ∈ 𝐵}⟶𝐶) |
| |
| Theorem | 2shfti 10996 |
Composite shift operations. (Contributed by NM, 19-Aug-2005.) (Revised
by Mario Carneiro, 5-Nov-2013.)
|
| ⊢ 𝐹 ∈ V ⇒ ⊢ ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ) → ((𝐹 shift 𝐴) shift 𝐵) = (𝐹 shift (𝐴 + 𝐵))) |
| |
| Theorem | shftidt2 10997 |
Identity law for the shift operation. (Contributed by Mario Carneiro,
5-Nov-2013.)
|
| ⊢ 𝐹 ∈ V ⇒ ⊢ (𝐹 shift 0) = (𝐹 ↾ ℂ) |
| |
| Theorem | shftidt 10998 |
Identity law for the shift operation. (Contributed by NM, 19-Aug-2005.)
(Revised by Mario Carneiro, 5-Nov-2013.)
|
| ⊢ 𝐹 ∈ V ⇒ ⊢ (𝐴 ∈ ℂ → ((𝐹 shift 0)‘𝐴) = (𝐹‘𝐴)) |
| |
| Theorem | shftcan1 10999 |
Cancellation law for the shift operation. (Contributed by NM,
4-Aug-2005.) (Revised by Mario Carneiro, 5-Nov-2013.)
|
| ⊢ 𝐹 ∈ V ⇒ ⊢ ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ) → (((𝐹 shift 𝐴) shift -𝐴)‘𝐵) = (𝐹‘𝐵)) |
| |
| Theorem | shftcan2 11000 |
Cancellation law for the shift operation. (Contributed by NM,
4-Aug-2005.) (Revised by Mario Carneiro, 5-Nov-2013.)
|
| ⊢ 𝐹 ∈ V ⇒ ⊢ ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ) → (((𝐹 shift -𝐴) shift 𝐴)‘𝐵) = (𝐹‘𝐵)) |