Home | Metamath
Proof Explorer Theorem List (p. 147 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 | s3cl 14601 | A length 3 string is a word. (Contributed by Mario Carneiro, 26-Feb-2016.) |
⊢ ((𝐴 ∈ 𝑋 ∧ 𝐵 ∈ 𝑋 ∧ 𝐶 ∈ 𝑋) → 〈“𝐴𝐵𝐶”〉 ∈ Word 𝑋) | ||
Theorem | s2cli 14602 | A doubleton word is a word. (Contributed by Mario Carneiro, 26-Feb-2016.) |
⊢ 〈“𝐴𝐵”〉 ∈ Word V | ||
Theorem | s3cli 14603 | A length 3 string is a word. (Contributed by Mario Carneiro, 26-Feb-2016.) |
⊢ 〈“𝐴𝐵𝐶”〉 ∈ Word V | ||
Theorem | s4cli 14604 | A length 4 string is a word. (Contributed by Mario Carneiro, 26-Feb-2016.) |
⊢ 〈“𝐴𝐵𝐶𝐷”〉 ∈ Word V | ||
Theorem | s5cli 14605 | A length 5 string is a word. (Contributed by Mario Carneiro, 26-Feb-2016.) |
⊢ 〈“𝐴𝐵𝐶𝐷𝐸”〉 ∈ Word V | ||
Theorem | s6cli 14606 | A length 6 string is a word. (Contributed by Mario Carneiro, 26-Feb-2016.) |
⊢ 〈“𝐴𝐵𝐶𝐷𝐸𝐹”〉 ∈ Word V | ||
Theorem | s7cli 14607 | A length 7 string is a word. (Contributed by Mario Carneiro, 26-Feb-2016.) |
⊢ 〈“𝐴𝐵𝐶𝐷𝐸𝐹𝐺”〉 ∈ Word V | ||
Theorem | s8cli 14608 | A length 8 string is a word. (Contributed by Mario Carneiro, 26-Feb-2016.) |
⊢ 〈“𝐴𝐵𝐶𝐷𝐸𝐹𝐺𝐻”〉 ∈ Word V | ||
Theorem | s2fv0 14609 | Extract the first symbol from a doubleton word. (Contributed by Stefan O'Rear, 23-Aug-2015.) (Revised by Mario Carneiro, 26-Feb-2016.) |
⊢ (𝐴 ∈ 𝑉 → (〈“𝐴𝐵”〉‘0) = 𝐴) | ||
Theorem | s2fv1 14610 | Extract the second symbol from a doubleton word. (Contributed by Stefan O'Rear, 23-Aug-2015.) (Revised by Mario Carneiro, 26-Feb-2016.) |
⊢ (𝐵 ∈ 𝑉 → (〈“𝐴𝐵”〉‘1) = 𝐵) | ||
Theorem | s2len 14611 | The length of a doubleton word. (Contributed by Stefan O'Rear, 23-Aug-2015.) (Revised by Mario Carneiro, 26-Feb-2016.) |
⊢ (♯‘〈“𝐴𝐵”〉) = 2 | ||
Theorem | s2dm 14612 | The domain of a doubleton word is an unordered pair. (Contributed by AV, 9-Jan-2020.) |
⊢ dom 〈“𝐴𝐵”〉 = {0, 1} | ||
Theorem | s3fv0 14613 | Extract the first symbol from a length 3 string. (Contributed by Mario Carneiro, 13-Jan-2017.) |
⊢ (𝐴 ∈ 𝑉 → (〈“𝐴𝐵𝐶”〉‘0) = 𝐴) | ||
Theorem | s3fv1 14614 | Extract the second symbol from a length 3 string. (Contributed by Mario Carneiro, 13-Jan-2017.) |
⊢ (𝐵 ∈ 𝑉 → (〈“𝐴𝐵𝐶”〉‘1) = 𝐵) | ||
Theorem | s3fv2 14615 | Extract the third symbol from a length 3 string. (Contributed by Mario Carneiro, 13-Jan-2017.) |
⊢ (𝐶 ∈ 𝑉 → (〈“𝐴𝐵𝐶”〉‘2) = 𝐶) | ||
Theorem | s3len 14616 | The length of a length 3 string. (Contributed by Mario Carneiro, 26-Feb-2016.) |
⊢ (♯‘〈“𝐴𝐵𝐶”〉) = 3 | ||
Theorem | s4fv0 14617 | Extract the first symbol from a length 4 string. (Contributed by Thierry Arnoux, 8-Oct-2020.) |
⊢ (𝐴 ∈ 𝑉 → (〈“𝐴𝐵𝐶𝐷”〉‘0) = 𝐴) | ||
Theorem | s4fv1 14618 | Extract the second symbol from a length 4 string. (Contributed by Thierry Arnoux, 8-Oct-2020.) |
⊢ (𝐵 ∈ 𝑉 → (〈“𝐴𝐵𝐶𝐷”〉‘1) = 𝐵) | ||
Theorem | s4fv2 14619 | Extract the third symbol from a length 4 string. (Contributed by Thierry Arnoux, 8-Oct-2020.) |
⊢ (𝐶 ∈ 𝑉 → (〈“𝐴𝐵𝐶𝐷”〉‘2) = 𝐶) | ||
Theorem | s4fv3 14620 | Extract the fourth symbol from a length 4 string. (Contributed by Thierry Arnoux, 8-Oct-2020.) |
⊢ (𝐷 ∈ 𝑉 → (〈“𝐴𝐵𝐶𝐷”〉‘3) = 𝐷) | ||
Theorem | s4len 14621 | The length of a length 4 string. (Contributed by Mario Carneiro, 26-Feb-2016.) |
⊢ (♯‘〈“𝐴𝐵𝐶𝐷”〉) = 4 | ||
Theorem | s5len 14622 | The length of a length 5 string. (Contributed by Mario Carneiro, 26-Feb-2016.) |
⊢ (♯‘〈“𝐴𝐵𝐶𝐷𝐸”〉) = 5 | ||
Theorem | s6len 14623 | The length of a length 6 string. (Contributed by Mario Carneiro, 26-Feb-2016.) |
⊢ (♯‘〈“𝐴𝐵𝐶𝐷𝐸𝐹”〉) = 6 | ||
Theorem | s7len 14624 | The length of a length 7 string. (Contributed by Mario Carneiro, 26-Feb-2016.) |
⊢ (♯‘〈“𝐴𝐵𝐶𝐷𝐸𝐹𝐺”〉) = 7 | ||
Theorem | s8len 14625 | The length of a length 8 string. (Contributed by Mario Carneiro, 26-Feb-2016.) |
⊢ (♯‘〈“𝐴𝐵𝐶𝐷𝐸𝐹𝐺𝐻”〉) = 8 | ||
Theorem | lsws2 14626 | The last symbol of a doubleton word is its second symbol. (Contributed by AV, 8-Feb-2021.) |
⊢ (𝐵 ∈ 𝑉 → (lastS‘〈“𝐴𝐵”〉) = 𝐵) | ||
Theorem | lsws3 14627 | The last symbol of a 3 letter word is its third symbol. (Contributed by AV, 8-Feb-2021.) |
⊢ (𝐶 ∈ 𝑉 → (lastS‘〈“𝐴𝐵𝐶”〉) = 𝐶) | ||
Theorem | lsws4 14628 | The last symbol of a 4 letter word is its fourth symbol. (Contributed by AV, 8-Feb-2021.) |
⊢ (𝐷 ∈ 𝑉 → (lastS‘〈“𝐴𝐵𝐶𝐷”〉) = 𝐷) | ||
Theorem | s2prop 14629 | A length 2 word is an unordered pair of ordered pairs. (Contributed by Alexander van der Vekens, 14-Aug-2017.) |
⊢ ((𝐴 ∈ 𝑆 ∧ 𝐵 ∈ 𝑆) → 〈“𝐴𝐵”〉 = {〈0, 𝐴〉, 〈1, 𝐵〉}) | ||
Theorem | s2dmALT 14630 | Alternate version of s2dm 14612, having a shorter proof, but requiring that 𝐴 and 𝐵 are sets. (Contributed by AV, 9-Jan-2020.) (Proof modification is discouraged.) (New usage is discouraged.) |
⊢ ((𝐴 ∈ 𝑆 ∧ 𝐵 ∈ 𝑆) → dom 〈“𝐴𝐵”〉 = {0, 1}) | ||
Theorem | s3tpop 14631 | A length 3 word is an unordered triple of ordered pairs. (Contributed by AV, 23-Jan-2021.) |
⊢ ((𝐴 ∈ 𝑆 ∧ 𝐵 ∈ 𝑆 ∧ 𝐶 ∈ 𝑆) → 〈“𝐴𝐵𝐶”〉 = {〈0, 𝐴〉, 〈1, 𝐵〉, 〈2, 𝐶〉}) | ||
Theorem | s4prop 14632 | A length 4 word is a union of two unordered pairs of ordered pairs. (Contributed by Alexander van der Vekens, 14-Aug-2017.) |
⊢ (((𝐴 ∈ 𝑆 ∧ 𝐵 ∈ 𝑆) ∧ (𝐶 ∈ 𝑆 ∧ 𝐷 ∈ 𝑆)) → 〈“𝐴𝐵𝐶𝐷”〉 = ({〈0, 𝐴〉, 〈1, 𝐵〉} ∪ {〈2, 𝐶〉, 〈3, 𝐷〉})) | ||
Theorem | s3fn 14633 | A length 3 word is a function with a triple as domain. (Contributed by Alexander van der Vekens, 5-Dec-2017.) (Revised by AV, 23-Jan-2021.) |
⊢ ((𝐴 ∈ 𝑉 ∧ 𝐵 ∈ 𝑉 ∧ 𝐶 ∈ 𝑉) → 〈“𝐴𝐵𝐶”〉 Fn {0, 1, 2}) | ||
Theorem | funcnvs1 14634 | The converse of a singleton word is a function. (Contributed by AV, 22-Jan-2021.) |
⊢ Fun ◡〈“𝐴”〉 | ||
Theorem | funcnvs2 14635 | The converse of a length 2 word is a function if its symbols are different sets. (Contributed by AV, 23-Jan-2021.) |
⊢ ((𝐴 ∈ 𝑉 ∧ 𝐵 ∈ 𝑉 ∧ 𝐴 ≠ 𝐵) → Fun ◡〈“𝐴𝐵”〉) | ||
Theorem | funcnvs3 14636 | The converse of a length 3 word is a function if its symbols are different sets. (Contributed by Alexander van der Vekens, 31-Jan-2018.) (Revised by AV, 23-Jan-2021.) |
⊢ (((𝐴 ∈ 𝑉 ∧ 𝐵 ∈ 𝑉 ∧ 𝐶 ∈ 𝑉) ∧ (𝐴 ≠ 𝐵 ∧ 𝐴 ≠ 𝐶 ∧ 𝐵 ≠ 𝐶)) → Fun ◡〈“𝐴𝐵𝐶”〉) | ||
Theorem | funcnvs4 14637 | The converse of a length 4 word is a function if its symbols are different sets. (Contributed by AV, 10-Feb-2021.) |
⊢ ((((𝐴 ∈ 𝑉 ∧ 𝐵 ∈ 𝑉) ∧ (𝐶 ∈ 𝑉 ∧ 𝐷 ∈ 𝑉)) ∧ ((𝐴 ≠ 𝐵 ∧ 𝐴 ≠ 𝐶 ∧ 𝐴 ≠ 𝐷) ∧ (𝐵 ≠ 𝐶 ∧ 𝐵 ≠ 𝐷) ∧ 𝐶 ≠ 𝐷)) → Fun ◡〈“𝐴𝐵𝐶𝐷”〉) | ||
Theorem | s2f1o 14638 | A length 2 word with mutually different symbols is a one-to-one function onto the set of the symbols. (Contributed by Alexander van der Vekens, 14-Aug-2017.) |
⊢ ((𝐴 ∈ 𝑆 ∧ 𝐵 ∈ 𝑆 ∧ 𝐴 ≠ 𝐵) → (𝐸 = 〈“𝐴𝐵”〉 → 𝐸:{0, 1}–1-1-onto→{𝐴, 𝐵})) | ||
Theorem | f1oun2prg 14639 | A union of unordered pairs of ordered pairs with different elements is a one-to-one onto function. (Contributed by Alexander van der Vekens, 14-Aug-2017.) |
⊢ (((𝐴 ∈ 𝑉 ∧ 𝐵 ∈ 𝑊) ∧ (𝐶 ∈ 𝑋 ∧ 𝐷 ∈ 𝑌)) → (((𝐴 ≠ 𝐵 ∧ 𝐴 ≠ 𝐶 ∧ 𝐴 ≠ 𝐷) ∧ (𝐵 ≠ 𝐶 ∧ 𝐵 ≠ 𝐷 ∧ 𝐶 ≠ 𝐷)) → ({〈0, 𝐴〉, 〈1, 𝐵〉} ∪ {〈2, 𝐶〉, 〈3, 𝐷〉}):({0, 1} ∪ {2, 3})–1-1-onto→({𝐴, 𝐵} ∪ {𝐶, 𝐷}))) | ||
Theorem | s4f1o 14640 | A length 4 word with mutually different symbols is a one-to-one function onto the set of the symbols. (Contributed by Alexander van der Vekens, 14-Aug-2017.) |
⊢ (((𝐴 ∈ 𝑆 ∧ 𝐵 ∈ 𝑆) ∧ (𝐶 ∈ 𝑆 ∧ 𝐷 ∈ 𝑆)) → (((𝐴 ≠ 𝐵 ∧ 𝐴 ≠ 𝐶 ∧ 𝐴 ≠ 𝐷) ∧ (𝐵 ≠ 𝐶 ∧ 𝐵 ≠ 𝐷 ∧ 𝐶 ≠ 𝐷)) → (𝐸 = 〈“𝐴𝐵𝐶𝐷”〉 → 𝐸:dom 𝐸–1-1-onto→({𝐴, 𝐵} ∪ {𝐶, 𝐷})))) | ||
Theorem | s4dom 14641 | The domain of a length 4 word is the union of two (disjunct) pairs. (Contributed by Alexander van der Vekens, 15-Aug-2017.) |
⊢ (((𝐴 ∈ 𝑆 ∧ 𝐵 ∈ 𝑆) ∧ (𝐶 ∈ 𝑆 ∧ 𝐷 ∈ 𝑆)) → (𝐸 = 〈“𝐴𝐵𝐶𝐷”〉 → dom 𝐸 = ({0, 1} ∪ {2, 3}))) | ||
Theorem | s2co 14642 | Mapping a doubleton word by a function. (Contributed by Mario Carneiro, 27-Feb-2016.) |
⊢ (𝜑 → 𝐹:𝑋⟶𝑌) & ⊢ (𝜑 → 𝐴 ∈ 𝑋) & ⊢ (𝜑 → 𝐵 ∈ 𝑋) ⇒ ⊢ (𝜑 → (𝐹 ∘ 〈“𝐴𝐵”〉) = 〈“(𝐹‘𝐴)(𝐹‘𝐵)”〉) | ||
Theorem | s3co 14643 | Mapping a length 3 string by a function. (Contributed by Mario Carneiro, 27-Feb-2016.) |
⊢ (𝜑 → 𝐹:𝑋⟶𝑌) & ⊢ (𝜑 → 𝐴 ∈ 𝑋) & ⊢ (𝜑 → 𝐵 ∈ 𝑋) & ⊢ (𝜑 → 𝐶 ∈ 𝑋) ⇒ ⊢ (𝜑 → (𝐹 ∘ 〈“𝐴𝐵𝐶”〉) = 〈“(𝐹‘𝐴)(𝐹‘𝐵)(𝐹‘𝐶)”〉) | ||
Theorem | s0s1 14644 | Concatenation of fixed length strings. (This special case of ccatlid 14300 is provided to complete the pattern s0s1 14644, df-s2 14570, df-s3 14571, ...) (Contributed by Mario Carneiro, 28-Feb-2016.) |
⊢ 〈“𝐴”〉 = (∅ ++ 〈“𝐴”〉) | ||
Theorem | s1s2 14645 | Concatenation of fixed length strings. (Contributed by Mario Carneiro, 26-Feb-2016.) |
⊢ 〈“𝐴𝐵𝐶”〉 = (〈“𝐴”〉 ++ 〈“𝐵𝐶”〉) | ||
Theorem | s1s3 14646 | Concatenation of fixed length strings. (Contributed by Mario Carneiro, 26-Feb-2016.) |
⊢ 〈“𝐴𝐵𝐶𝐷”〉 = (〈“𝐴”〉 ++ 〈“𝐵𝐶𝐷”〉) | ||
Theorem | s1s4 14647 | Concatenation of fixed length strings. (Contributed by Mario Carneiro, 26-Feb-2016.) |
⊢ 〈“𝐴𝐵𝐶𝐷𝐸”〉 = (〈“𝐴”〉 ++ 〈“𝐵𝐶𝐷𝐸”〉) | ||
Theorem | s1s5 14648 | Concatenation of fixed length strings. (Contributed by Mario Carneiro, 26-Feb-2016.) |
⊢ 〈“𝐴𝐵𝐶𝐷𝐸𝐹”〉 = (〈“𝐴”〉 ++ 〈“𝐵𝐶𝐷𝐸𝐹”〉) | ||
Theorem | s1s6 14649 | Concatenation of fixed length strings. (Contributed by Mario Carneiro, 26-Feb-2016.) |
⊢ 〈“𝐴𝐵𝐶𝐷𝐸𝐹𝐺”〉 = (〈“𝐴”〉 ++ 〈“𝐵𝐶𝐷𝐸𝐹𝐺”〉) | ||
Theorem | s1s7 14650 | Concatenation of fixed length strings. (Contributed by Mario Carneiro, 26-Feb-2016.) |
⊢ 〈“𝐴𝐵𝐶𝐷𝐸𝐹𝐺𝐻”〉 = (〈“𝐴”〉 ++ 〈“𝐵𝐶𝐷𝐸𝐹𝐺𝐻”〉) | ||
Theorem | s2s2 14651 | Concatenation of fixed length strings. (Contributed by Mario Carneiro, 26-Feb-2016.) |
⊢ 〈“𝐴𝐵𝐶𝐷”〉 = (〈“𝐴𝐵”〉 ++ 〈“𝐶𝐷”〉) | ||
Theorem | s4s2 14652 | Concatenation of fixed length strings. (Contributed by Mario Carneiro, 26-Feb-2016.) |
⊢ 〈“𝐴𝐵𝐶𝐷𝐸𝐹”〉 = (〈“𝐴𝐵𝐶𝐷”〉 ++ 〈“𝐸𝐹”〉) | ||
Theorem | s4s3 14653 | Concatenation of fixed length strings. (Contributed by Mario Carneiro, 26-Feb-2016.) |
⊢ 〈“𝐴𝐵𝐶𝐷𝐸𝐹𝐺”〉 = (〈“𝐴𝐵𝐶𝐷”〉 ++ 〈“𝐸𝐹𝐺”〉) | ||
Theorem | s4s4 14654 | Concatenation of fixed length strings. (Contributed by Mario Carneiro, 26-Feb-2016.) |
⊢ 〈“𝐴𝐵𝐶𝐷𝐸𝐹𝐺𝐻”〉 = (〈“𝐴𝐵𝐶𝐷”〉 ++ 〈“𝐸𝐹𝐺𝐻”〉) | ||
Theorem | s3s4 14655 | Concatenation of fixed length strings. (Contributed by AV, 1-Mar-2021.) |
⊢ 〈“𝐴𝐵𝐶𝐷𝐸𝐹𝐺”〉 = (〈“𝐴𝐵𝐶”〉 ++ 〈“𝐷𝐸𝐹𝐺”〉) | ||
Theorem | s2s5 14656 | Concatenation of fixed length strings. (Contributed by AV, 1-Mar-2021.) |
⊢ 〈“𝐴𝐵𝐶𝐷𝐸𝐹𝐺”〉 = (〈“𝐴𝐵”〉 ++ 〈“𝐶𝐷𝐸𝐹𝐺”〉) | ||
Theorem | s5s2 14657 | Concatenation of fixed length strings. (Contributed by AV, 1-Mar-2021.) |
⊢ 〈“𝐴𝐵𝐶𝐷𝐸𝐹𝐺”〉 = (〈“𝐴𝐵𝐶𝐷𝐸”〉 ++ 〈“𝐹𝐺”〉) | ||
Theorem | s2eq2s1eq 14658 | Two length 2 words are equal iff the corresponding singleton words consisting of their symbols are equal. (Contributed by Alexander van der Vekens, 24-Sep-2018.) |
⊢ (((𝐴 ∈ 𝑉 ∧ 𝐵 ∈ 𝑉) ∧ (𝐶 ∈ 𝑉 ∧ 𝐷 ∈ 𝑉)) → (〈“𝐴𝐵”〉 = 〈“𝐶𝐷”〉 ↔ (〈“𝐴”〉 = 〈“𝐶”〉 ∧ 〈“𝐵”〉 = 〈“𝐷”〉))) | ||
Theorem | s2eq2seq 14659 | Two length 2 words are equal iff the corresponding symbols are equal. (Contributed by AV, 20-Oct-2018.) |
⊢ (((𝐴 ∈ 𝑉 ∧ 𝐵 ∈ 𝑉) ∧ (𝐶 ∈ 𝑉 ∧ 𝐷 ∈ 𝑉)) → (〈“𝐴𝐵”〉 = 〈“𝐶𝐷”〉 ↔ (𝐴 = 𝐶 ∧ 𝐵 = 𝐷))) | ||
Theorem | s3eqs2s1eq 14660 | Two length 3 words are equal iff the corresponding length 2 words and singleton words consisting of their symbols are equal. (Contributed by AV, 4-Jan-2022.) |
⊢ (((𝐴 ∈ 𝑉 ∧ 𝐵 ∈ 𝑉 ∧ 𝐶 ∈ 𝑉) ∧ (𝐷 ∈ 𝑉 ∧ 𝐸 ∈ 𝑉 ∧ 𝐹 ∈ 𝑉)) → (〈“𝐴𝐵𝐶”〉 = 〈“𝐷𝐸𝐹”〉 ↔ (〈“𝐴𝐵”〉 = 〈“𝐷𝐸”〉 ∧ 〈“𝐶”〉 = 〈“𝐹”〉))) | ||
Theorem | s3eq3seq 14661 | Two length 3 words are equal iff the corresponding symbols are equal. (Contributed by AV, 4-Jan-2022.) |
⊢ (((𝐴 ∈ 𝑉 ∧ 𝐵 ∈ 𝑉 ∧ 𝐶 ∈ 𝑉) ∧ (𝐷 ∈ 𝑉 ∧ 𝐸 ∈ 𝑉 ∧ 𝐹 ∈ 𝑉)) → (〈“𝐴𝐵𝐶”〉 = 〈“𝐷𝐸𝐹”〉 ↔ (𝐴 = 𝐷 ∧ 𝐵 = 𝐸 ∧ 𝐶 = 𝐹))) | ||
Theorem | swrds2 14662 | Extract two adjacent symbols from a word. (Contributed by Stefan O'Rear, 23-Aug-2015.) (Revised by Mario Carneiro, 26-Feb-2016.) |
⊢ ((𝑊 ∈ Word 𝐴 ∧ 𝐼 ∈ ℕ0 ∧ (𝐼 + 1) ∈ (0..^(♯‘𝑊))) → (𝑊 substr 〈𝐼, (𝐼 + 2)〉) = 〈“(𝑊‘𝐼)(𝑊‘(𝐼 + 1))”〉) | ||
Theorem | swrds2m 14663 | Extract two adjacent symbols from a word in reverse direction. (Contributed by AV, 11-May-2022.) |
⊢ ((𝑊 ∈ Word 𝑉 ∧ 𝑁 ∈ (2...(♯‘𝑊))) → (𝑊 substr 〈(𝑁 − 2), 𝑁〉) = 〈“(𝑊‘(𝑁 − 2))(𝑊‘(𝑁 − 1))”〉) | ||
Theorem | wrdlen2i 14664 | Implications of a word of length two. (Contributed by AV, 27-Jul-2018.) (Proof shortened by AV, 14-Oct-2018.) |
⊢ ((𝑆 ∈ 𝑉 ∧ 𝑇 ∈ 𝑉) → (𝑊 = {〈0, 𝑆〉, 〈1, 𝑇〉} → ((𝑊 ∈ Word 𝑉 ∧ (♯‘𝑊) = 2) ∧ ((𝑊‘0) = 𝑆 ∧ (𝑊‘1) = 𝑇)))) | ||
Theorem | wrd2pr2op 14665 | A word of length two represented as unordered pair of ordered pairs. (Contributed by AV, 20-Oct-2018.) (Proof shortened by AV, 26-Jan-2021.) |
⊢ ((𝑊 ∈ Word 𝑉 ∧ (♯‘𝑊) = 2) → 𝑊 = {〈0, (𝑊‘0)〉, 〈1, (𝑊‘1)〉}) | ||
Theorem | wrdlen2 14666 | A word of length two. (Contributed by AV, 20-Oct-2018.) |
⊢ ((𝑆 ∈ 𝑉 ∧ 𝑇 ∈ 𝑉) → (𝑊 = {〈0, 𝑆〉, 〈1, 𝑇〉} ↔ ((𝑊 ∈ Word 𝑉 ∧ (♯‘𝑊) = 2) ∧ ((𝑊‘0) = 𝑆 ∧ (𝑊‘1) = 𝑇)))) | ||
Theorem | wrdlen2s2 14667 | A word of length two as doubleton word. (Contributed by AV, 20-Oct-2018.) |
⊢ ((𝑊 ∈ Word 𝑉 ∧ (♯‘𝑊) = 2) → 𝑊 = 〈“(𝑊‘0)(𝑊‘1)”〉) | ||
Theorem | wrdl2exs2 14668* | A word of length two is a doubleton word. (Contributed by AV, 25-Jan-2021.) |
⊢ ((𝑊 ∈ Word 𝑆 ∧ (♯‘𝑊) = 2) → ∃𝑠 ∈ 𝑆 ∃𝑡 ∈ 𝑆 𝑊 = 〈“𝑠𝑡”〉) | ||
Theorem | pfx2 14669 | A prefix of length two. (Contributed by AV, 15-May-2020.) |
⊢ ((𝑊 ∈ Word 𝑉 ∧ 2 ≤ (♯‘𝑊)) → (𝑊 prefix 2) = 〈“(𝑊‘0)(𝑊‘1)”〉) | ||
Theorem | wrd3tpop 14670 | A word of length three represented as triple of ordered pairs. (Contributed by AV, 26-Jan-2021.) |
⊢ ((𝑊 ∈ Word 𝑉 ∧ (♯‘𝑊) = 3) → 𝑊 = {〈0, (𝑊‘0)〉, 〈1, (𝑊‘1)〉, 〈2, (𝑊‘2)〉}) | ||
Theorem | wrdlen3s3 14671 | A word of length three as length 3 string. (Contributed by AV, 26-Jan-2021.) |
⊢ ((𝑊 ∈ Word 𝑉 ∧ (♯‘𝑊) = 3) → 𝑊 = 〈“(𝑊‘0)(𝑊‘1)(𝑊‘2)”〉) | ||
Theorem | repsw2 14672 | The "repeated symbol word" of length two. (Contributed by AV, 6-Nov-2018.) |
⊢ (𝑆 ∈ 𝑉 → (𝑆 repeatS 2) = 〈“𝑆𝑆”〉) | ||
Theorem | repsw3 14673 | The "repeated symbol word" of length three. (Contributed by AV, 6-Nov-2018.) |
⊢ (𝑆 ∈ 𝑉 → (𝑆 repeatS 3) = 〈“𝑆𝑆𝑆”〉) | ||
Theorem | swrd2lsw 14674 | Extract the last two symbols from a word. (Contributed by Alexander van der Vekens, 23-Sep-2018.) |
⊢ ((𝑊 ∈ Word 𝑉 ∧ 1 < (♯‘𝑊)) → (𝑊 substr 〈((♯‘𝑊) − 2), (♯‘𝑊)〉) = 〈“(𝑊‘((♯‘𝑊) − 2))(lastS‘𝑊)”〉) | ||
Theorem | 2swrd2eqwrdeq 14675 | Two words of length at least two are equal if and only if they have the same prefix and the same two single symbols suffix. (Contributed by AV, 24-Sep-2018.) (Revised by AV, 12-Oct-2022.) |
⊢ ((𝑊 ∈ Word 𝑉 ∧ 𝑈 ∈ Word 𝑉 ∧ 1 < (♯‘𝑊)) → (𝑊 = 𝑈 ↔ ((♯‘𝑊) = (♯‘𝑈) ∧ ((𝑊 prefix ((♯‘𝑊) − 2)) = (𝑈 prefix ((♯‘𝑊) − 2)) ∧ (𝑊‘((♯‘𝑊) − 2)) = (𝑈‘((♯‘𝑊) − 2)) ∧ (lastS‘𝑊) = (lastS‘𝑈))))) | ||
Theorem | ccatw2s1ccatws2 14676 | The concatenation of a word with two singleton words equals the concatenation of the word with the doubleton word consisting of the symbols of the two singletons. (Contributed by Mario Carneiro/AV, 21-Oct-2018.) (Revised by AV, 29-Jan-2024.) |
⊢ (𝑊 ∈ Word 𝑉 → ((𝑊 ++ 〈“𝑋”〉) ++ 〈“𝑌”〉) = (𝑊 ++ 〈“𝑋𝑌”〉)) | ||
Theorem | ccatw2s1ccatws2OLD 14677 | Obsolete version of ccatw2s1ccatws2 14676 as of 29-Jan-2024. The concatenation of a word with two singleton words equals the concatenation of the word with the doubleton word consisting of the symbols of the two singletons. (Contributed by Mario Carneiro/AV, 21-Oct-2018.) (New usage is discouraged.) (Proof modification is discouraged.) |
⊢ ((𝑊 ∈ Word 𝑉 ∧ 𝑋 ∈ 𝑉 ∧ 𝑌 ∈ 𝑉) → ((𝑊 ++ 〈“𝑋”〉) ++ 〈“𝑌”〉) = (𝑊 ++ 〈“𝑋𝑌”〉)) | ||
Theorem | ccat2s1fvwALT 14678 | Alternate proof of ccat2s1fvw 14358 using words of length 2, see df-s2 14570. A symbol of the concatenation of a word with two single symbols corresponding to the symbol of the word. (Contributed by AV, 22-Sep-2018.) (Proof shortened by Mario Carneiro/AV, 21-Oct-2018.) (Revised by AV, 28-Jan-2024.) (New usage is discouraged.) (Proof modification is discouraged.) |
⊢ ((𝑊 ∈ Word 𝑉 ∧ 𝐼 ∈ ℕ0 ∧ 𝐼 < (♯‘𝑊)) → (((𝑊 ++ 〈“𝑋”〉) ++ 〈“𝑌”〉)‘𝐼) = (𝑊‘𝐼)) | ||
Theorem | ccat2s1fvwALTOLD 14679 | Obsolete version of ccat2s1fvwALT 14678 as of 28-Jan-2024. Alternate proof of ccat2s1fvwOLD 14359 using words of length 2, see df-s2 14570. A symbol of the concatenation of a word with two single symbols corresponding to the symbol of the word. (Contributed by AV, 22-Sep-2018.) (Proof shortened by Mario Carneiro/AV, 21-Oct-2018.) (New usage is discouraged.) (Proof modification is discouraged.) |
⊢ (((𝑊 ∈ Word 𝑉 ∧ 𝐼 ∈ ℕ0 ∧ 𝐼 < (♯‘𝑊)) ∧ (𝑋 ∈ 𝑉 ∧ 𝑌 ∈ 𝑉)) → (((𝑊 ++ 〈“𝑋”〉) ++ 〈“𝑌”〉)‘𝐼) = (𝑊‘𝐼)) | ||
Theorem | wwlktovf 14680* | Lemma 1 for wrd2f1tovbij 14684. (Contributed by Alexander van der Vekens, 27-Jul-2018.) |
⊢ 𝐷 = {𝑤 ∈ Word 𝑉 ∣ ((♯‘𝑤) = 2 ∧ (𝑤‘0) = 𝑃 ∧ {(𝑤‘0), (𝑤‘1)} ∈ 𝑋)} & ⊢ 𝑅 = {𝑛 ∈ 𝑉 ∣ {𝑃, 𝑛} ∈ 𝑋} & ⊢ 𝐹 = (𝑡 ∈ 𝐷 ↦ (𝑡‘1)) ⇒ ⊢ 𝐹:𝐷⟶𝑅 | ||
Theorem | wwlktovf1 14681* | Lemma 2 for wrd2f1tovbij 14684. (Contributed by Alexander van der Vekens, 27-Jul-2018.) |
⊢ 𝐷 = {𝑤 ∈ Word 𝑉 ∣ ((♯‘𝑤) = 2 ∧ (𝑤‘0) = 𝑃 ∧ {(𝑤‘0), (𝑤‘1)} ∈ 𝑋)} & ⊢ 𝑅 = {𝑛 ∈ 𝑉 ∣ {𝑃, 𝑛} ∈ 𝑋} & ⊢ 𝐹 = (𝑡 ∈ 𝐷 ↦ (𝑡‘1)) ⇒ ⊢ 𝐹:𝐷–1-1→𝑅 | ||
Theorem | wwlktovfo 14682* | Lemma 3 for wrd2f1tovbij 14684. (Contributed by Alexander van der Vekens, 27-Jul-2018.) |
⊢ 𝐷 = {𝑤 ∈ Word 𝑉 ∣ ((♯‘𝑤) = 2 ∧ (𝑤‘0) = 𝑃 ∧ {(𝑤‘0), (𝑤‘1)} ∈ 𝑋)} & ⊢ 𝑅 = {𝑛 ∈ 𝑉 ∣ {𝑃, 𝑛} ∈ 𝑋} & ⊢ 𝐹 = (𝑡 ∈ 𝐷 ↦ (𝑡‘1)) ⇒ ⊢ (𝑃 ∈ 𝑉 → 𝐹:𝐷–onto→𝑅) | ||
Theorem | wwlktovf1o 14683* | Lemma 4 for wrd2f1tovbij 14684. (Contributed by Alexander van der Vekens, 28-Jul-2018.) |
⊢ 𝐷 = {𝑤 ∈ Word 𝑉 ∣ ((♯‘𝑤) = 2 ∧ (𝑤‘0) = 𝑃 ∧ {(𝑤‘0), (𝑤‘1)} ∈ 𝑋)} & ⊢ 𝑅 = {𝑛 ∈ 𝑉 ∣ {𝑃, 𝑛} ∈ 𝑋} & ⊢ 𝐹 = (𝑡 ∈ 𝐷 ↦ (𝑡‘1)) ⇒ ⊢ (𝑃 ∈ 𝑉 → 𝐹:𝐷–1-1-onto→𝑅) | ||
Theorem | wrd2f1tovbij 14684* | There is a bijection between words of length two with a fixed first symbol contained in a pair and the symbols contained in a pair together with the fixed symbol. (Contributed by Alexander van der Vekens, 28-Jul-2018.) |
⊢ ((𝑉 ∈ 𝑌 ∧ 𝑃 ∈ 𝑉) → ∃𝑓 𝑓:{𝑤 ∈ Word 𝑉 ∣ ((♯‘𝑤) = 2 ∧ (𝑤‘0) = 𝑃 ∧ {(𝑤‘0), (𝑤‘1)} ∈ 𝑋)}–1-1-onto→{𝑛 ∈ 𝑉 ∣ {𝑃, 𝑛} ∈ 𝑋}) | ||
Theorem | eqwrds3 14685 | A word is equal with a length 3 string iff it has length 3 and the same symbol at each position. (Contributed by AV, 12-May-2021.) |
⊢ ((𝑊 ∈ Word 𝑉 ∧ (𝐴 ∈ 𝑉 ∧ 𝐵 ∈ 𝑉 ∧ 𝐶 ∈ 𝑉)) → (𝑊 = 〈“𝐴𝐵𝐶”〉 ↔ ((♯‘𝑊) = 3 ∧ ((𝑊‘0) = 𝐴 ∧ (𝑊‘1) = 𝐵 ∧ (𝑊‘2) = 𝐶)))) | ||
Theorem | wrdl3s3 14686* | A word of length 3 is a length 3 string. (Contributed by AV, 18-May-2021.) |
⊢ ((𝑊 ∈ Word 𝑉 ∧ (♯‘𝑊) = 3) ↔ ∃𝑎 ∈ 𝑉 ∃𝑏 ∈ 𝑉 ∃𝑐 ∈ 𝑉 𝑊 = 〈“𝑎𝑏𝑐”〉) | ||
Theorem | s3sndisj 14687* | The singletons consisting of length 3 strings which have distinct third symbols are disjunct. (Contributed by AV, 17-May-2021.) |
⊢ ((𝐴 ∈ 𝑋 ∧ 𝐵 ∈ 𝑌) → Disj 𝑐 ∈ 𝑍 {〈“𝐴𝐵𝑐”〉}) | ||
Theorem | s3iunsndisj 14688* | The union of singletons consisting of length 3 strings which have distinct first and third symbols are disjunct. (Contributed by AV, 17-May-2021.) |
⊢ (𝐵 ∈ 𝑋 → Disj 𝑎 ∈ 𝑌 ∪ 𝑐 ∈ (𝑍 ∖ {𝑎}){〈“𝑎𝐵𝑐”〉}) | ||
Theorem | ofccat 14689 | Letterwise operations on word concatenations. (Contributed by Thierry Arnoux, 28-Sep-2018.) |
⊢ (𝜑 → 𝐸 ∈ Word 𝑆) & ⊢ (𝜑 → 𝐹 ∈ Word 𝑆) & ⊢ (𝜑 → 𝐺 ∈ Word 𝑇) & ⊢ (𝜑 → 𝐻 ∈ Word 𝑇) & ⊢ (𝜑 → (♯‘𝐸) = (♯‘𝐺)) & ⊢ (𝜑 → (♯‘𝐹) = (♯‘𝐻)) ⇒ ⊢ (𝜑 → ((𝐸 ++ 𝐹) ∘f 𝑅(𝐺 ++ 𝐻)) = ((𝐸 ∘f 𝑅𝐺) ++ (𝐹 ∘f 𝑅𝐻))) | ||
Theorem | ofs1 14690 | Letterwise operations on a single letter word. (Contributed by Thierry Arnoux, 7-Oct-2018.) |
⊢ ((𝐴 ∈ 𝑆 ∧ 𝐵 ∈ 𝑇) → (〈“𝐴”〉 ∘f 𝑅〈“𝐵”〉) = 〈“(𝐴𝑅𝐵)”〉) | ||
Theorem | ofs2 14691 | Letterwise operations on a double letter word. (Contributed by Thierry Arnoux, 7-Oct-2018.) |
⊢ (((𝐴 ∈ 𝑆 ∧ 𝐵 ∈ 𝑆) ∧ (𝐶 ∈ 𝑇 ∧ 𝐷 ∈ 𝑇)) → (〈“𝐴𝐵”〉 ∘f 𝑅〈“𝐶𝐷”〉) = 〈“(𝐴𝑅𝐶)(𝐵𝑅𝐷)”〉) | ||
A relation, 𝑅, has the reflexive property if 𝐴𝑅𝐴 holds whenever 𝐴 is an element which could be related by the relation, namely, an element of its domain or range. Eliminating dummy variables, we see that a segment of the identity relation must be a subset of the relation, or ( I ↾ (ran 𝑅 ∪ dom 𝑅)) ⊆ 𝑅. See idref 7027. A relation, 𝑅, has the transitive property if 𝐴𝑅𝐶 holds whenever there exists an intermediate value 𝐵 such that both 𝐴𝑅𝐵 and 𝐵𝑅𝐶 hold. This can be expressed without dummy variables as (𝑅 ∘ 𝑅) ⊆ 𝑅. See cotr 6022. The transitive closure of a relation, (t+‘𝑅), is the smallest superset of the relation which has the transitive property. Likewise, the reflexive-transitive closure, (t*‘𝑅), is the smallest superset which has both the reflexive and transitive properties. Not to be confused with the transitive closure of a set, trcl 9495, which is a closure relative to a different transitive property, df-tr 5193. | ||
Theorem | coss12d 14692 | Subset deduction for composition of two classes. (Contributed by RP, 24-Dec-2019.) |
⊢ (𝜑 → 𝐴 ⊆ 𝐵) & ⊢ (𝜑 → 𝐶 ⊆ 𝐷) ⇒ ⊢ (𝜑 → (𝐴 ∘ 𝐶) ⊆ (𝐵 ∘ 𝐷)) | ||
Theorem | trrelssd 14693 | The composition of subclasses of a transitive relation is a subclass of that relation. (Contributed by RP, 24-Dec-2019.) |
⊢ (𝜑 → (𝑅 ∘ 𝑅) ⊆ 𝑅) & ⊢ (𝜑 → 𝑆 ⊆ 𝑅) & ⊢ (𝜑 → 𝑇 ⊆ 𝑅) ⇒ ⊢ (𝜑 → (𝑆 ∘ 𝑇) ⊆ 𝑅) | ||
Theorem | xpcogend 14694 | The most interesting case of the composition of two Cartesian products. (Contributed by RP, 24-Dec-2019.) |
⊢ (𝜑 → (𝐵 ∩ 𝐶) ≠ ∅) ⇒ ⊢ (𝜑 → ((𝐶 × 𝐷) ∘ (𝐴 × 𝐵)) = (𝐴 × 𝐷)) | ||
Theorem | xpcoidgend 14695 | If two classes are not disjoint, then the composition of their Cartesian product with itself is idempotent. (Contributed by RP, 24-Dec-2019.) |
⊢ (𝜑 → (𝐴 ∩ 𝐵) ≠ ∅) ⇒ ⊢ (𝜑 → ((𝐴 × 𝐵) ∘ (𝐴 × 𝐵)) = (𝐴 × 𝐵)) | ||
Theorem | cotr2g 14696* | Two ways of saying that the composition of two relations is included in a third relation. See its special instance cotr2 14697 for the main application. (Contributed by RP, 22-Mar-2020.) |
⊢ dom 𝐵 ⊆ 𝐷 & ⊢ (ran 𝐵 ∩ dom 𝐴) ⊆ 𝐸 & ⊢ ran 𝐴 ⊆ 𝐹 ⇒ ⊢ ((𝐴 ∘ 𝐵) ⊆ 𝐶 ↔ ∀𝑥 ∈ 𝐷 ∀𝑦 ∈ 𝐸 ∀𝑧 ∈ 𝐹 ((𝑥𝐵𝑦 ∧ 𝑦𝐴𝑧) → 𝑥𝐶𝑧)) | ||
Theorem | cotr2 14697* | Two ways of saying a relation is transitive. Special instance of cotr2g 14696. (Contributed by RP, 22-Mar-2020.) |
⊢ dom 𝑅 ⊆ 𝐴 & ⊢ (dom 𝑅 ∩ ran 𝑅) ⊆ 𝐵 & ⊢ ran 𝑅 ⊆ 𝐶 ⇒ ⊢ ((𝑅 ∘ 𝑅) ⊆ 𝑅 ↔ ∀𝑥 ∈ 𝐴 ∀𝑦 ∈ 𝐵 ∀𝑧 ∈ 𝐶 ((𝑥𝑅𝑦 ∧ 𝑦𝑅𝑧) → 𝑥𝑅𝑧)) | ||
Theorem | cotr3 14698* | Two ways of saying a relation is transitive. (Contributed by RP, 22-Mar-2020.) |
⊢ 𝐴 = dom 𝑅 & ⊢ 𝐵 = (𝐴 ∩ 𝐶) & ⊢ 𝐶 = ran 𝑅 ⇒ ⊢ ((𝑅 ∘ 𝑅) ⊆ 𝑅 ↔ ∀𝑥 ∈ 𝐴 ∀𝑦 ∈ 𝐵 ∀𝑧 ∈ 𝐶 ((𝑥𝑅𝑦 ∧ 𝑦𝑅𝑧) → 𝑥𝑅𝑧)) | ||
Theorem | coemptyd 14699 | Deduction about composition of classes with no relational content in common. (Contributed by RP, 24-Dec-2019.) |
⊢ (𝜑 → (dom 𝐴 ∩ ran 𝐵) = ∅) ⇒ ⊢ (𝜑 → (𝐴 ∘ 𝐵) = ∅) | ||
Theorem | xptrrel 14700 | The cross product is always a transitive relation. (Contributed by RP, 24-Dec-2019.) |
⊢ ((𝐴 × 𝐵) ∘ (𝐴 × 𝐵)) ⊆ (𝐴 × 𝐵) |
< Previous Next > |
Copyright terms: Public domain | < Previous Next > |