Home | Metamath
Proof Explorer Theorem List (p. 147 of 465) | < 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-29268) |
Hilbert Space Explorer
(29269-30791) |
Users' Mathboxes
(30792-46474) |
Type | Label | Description |
---|---|---|
Statement | ||
Theorem | s4fv3 14601 | Extract the fourth symbol from a length 4 string. (Contributed by Thierry Arnoux, 8-Oct-2020.) |
⊢ (𝐷 ∈ 𝑉 → (〈“𝐴𝐵𝐶𝐷”〉‘3) = 𝐷) | ||
Theorem | s4len 14602 | The length of a length 4 string. (Contributed by Mario Carneiro, 26-Feb-2016.) |
⊢ (♯‘〈“𝐴𝐵𝐶𝐷”〉) = 4 | ||
Theorem | s5len 14603 | The length of a length 5 string. (Contributed by Mario Carneiro, 26-Feb-2016.) |
⊢ (♯‘〈“𝐴𝐵𝐶𝐷𝐸”〉) = 5 | ||
Theorem | s6len 14604 | The length of a length 6 string. (Contributed by Mario Carneiro, 26-Feb-2016.) |
⊢ (♯‘〈“𝐴𝐵𝐶𝐷𝐸𝐹”〉) = 6 | ||
Theorem | s7len 14605 | The length of a length 7 string. (Contributed by Mario Carneiro, 26-Feb-2016.) |
⊢ (♯‘〈“𝐴𝐵𝐶𝐷𝐸𝐹𝐺”〉) = 7 | ||
Theorem | s8len 14606 | The length of a length 8 string. (Contributed by Mario Carneiro, 26-Feb-2016.) |
⊢ (♯‘〈“𝐴𝐵𝐶𝐷𝐸𝐹𝐺𝐻”〉) = 8 | ||
Theorem | lsws2 14607 | The last symbol of a doubleton word is its second symbol. (Contributed by AV, 8-Feb-2021.) |
⊢ (𝐵 ∈ 𝑉 → (lastS‘〈“𝐴𝐵”〉) = 𝐵) | ||
Theorem | lsws3 14608 | The last symbol of a 3 letter word is its third symbol. (Contributed by AV, 8-Feb-2021.) |
⊢ (𝐶 ∈ 𝑉 → (lastS‘〈“𝐴𝐵𝐶”〉) = 𝐶) | ||
Theorem | lsws4 14609 | The last symbol of a 4 letter word is its fourth symbol. (Contributed by AV, 8-Feb-2021.) |
⊢ (𝐷 ∈ 𝑉 → (lastS‘〈“𝐴𝐵𝐶𝐷”〉) = 𝐷) | ||
Theorem | s2prop 14610 | A length 2 word is an unordered pair of ordered pairs. (Contributed by Alexander van der Vekens, 14-Aug-2017.) |
⊢ ((𝐴 ∈ 𝑆 ∧ 𝐵 ∈ 𝑆) → 〈“𝐴𝐵”〉 = {〈0, 𝐴〉, 〈1, 𝐵〉}) | ||
Theorem | s2dmALT 14611 | Alternate version of s2dm 14593, 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 14612 | A length 3 word is an unordered triple of ordered pairs. (Contributed by AV, 23-Jan-2021.) |
⊢ ((𝐴 ∈ 𝑆 ∧ 𝐵 ∈ 𝑆 ∧ 𝐶 ∈ 𝑆) → 〈“𝐴𝐵𝐶”〉 = {〈0, 𝐴〉, 〈1, 𝐵〉, 〈2, 𝐶〉}) | ||
Theorem | s4prop 14613 | 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 14614 | 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 14615 | The converse of a singleton word is a function. (Contributed by AV, 22-Jan-2021.) |
⊢ Fun ◡〈“𝐴”〉 | ||
Theorem | funcnvs2 14616 | 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 14617 | 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 14618 | 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 14619 | 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 14620 | 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 14621 | 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 14622 | 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 14623 | Mapping a doubleton word by a function. (Contributed by Mario Carneiro, 27-Feb-2016.) |
⊢ (𝜑 → 𝐹:𝑋⟶𝑌) & ⊢ (𝜑 → 𝐴 ∈ 𝑋) & ⊢ (𝜑 → 𝐵 ∈ 𝑋) ⇒ ⊢ (𝜑 → (𝐹 ∘ 〈“𝐴𝐵”〉) = 〈“(𝐹‘𝐴)(𝐹‘𝐵)”〉) | ||
Theorem | s3co 14624 | Mapping a length 3 string by a function. (Contributed by Mario Carneiro, 27-Feb-2016.) |
⊢ (𝜑 → 𝐹:𝑋⟶𝑌) & ⊢ (𝜑 → 𝐴 ∈ 𝑋) & ⊢ (𝜑 → 𝐵 ∈ 𝑋) & ⊢ (𝜑 → 𝐶 ∈ 𝑋) ⇒ ⊢ (𝜑 → (𝐹 ∘ 〈“𝐴𝐵𝐶”〉) = 〈“(𝐹‘𝐴)(𝐹‘𝐵)(𝐹‘𝐶)”〉) | ||
Theorem | s0s1 14625 | Concatenation of fixed length strings. (This special case of ccatlid 14281 is provided to complete the pattern s0s1 14625, df-s2 14551, df-s3 14552, ...) (Contributed by Mario Carneiro, 28-Feb-2016.) |
⊢ 〈“𝐴”〉 = (∅ ++ 〈“𝐴”〉) | ||
Theorem | s1s2 14626 | Concatenation of fixed length strings. (Contributed by Mario Carneiro, 26-Feb-2016.) |
⊢ 〈“𝐴𝐵𝐶”〉 = (〈“𝐴”〉 ++ 〈“𝐵𝐶”〉) | ||
Theorem | s1s3 14627 | Concatenation of fixed length strings. (Contributed by Mario Carneiro, 26-Feb-2016.) |
⊢ 〈“𝐴𝐵𝐶𝐷”〉 = (〈“𝐴”〉 ++ 〈“𝐵𝐶𝐷”〉) | ||
Theorem | s1s4 14628 | Concatenation of fixed length strings. (Contributed by Mario Carneiro, 26-Feb-2016.) |
⊢ 〈“𝐴𝐵𝐶𝐷𝐸”〉 = (〈“𝐴”〉 ++ 〈“𝐵𝐶𝐷𝐸”〉) | ||
Theorem | s1s5 14629 | Concatenation of fixed length strings. (Contributed by Mario Carneiro, 26-Feb-2016.) |
⊢ 〈“𝐴𝐵𝐶𝐷𝐸𝐹”〉 = (〈“𝐴”〉 ++ 〈“𝐵𝐶𝐷𝐸𝐹”〉) | ||
Theorem | s1s6 14630 | Concatenation of fixed length strings. (Contributed by Mario Carneiro, 26-Feb-2016.) |
⊢ 〈“𝐴𝐵𝐶𝐷𝐸𝐹𝐺”〉 = (〈“𝐴”〉 ++ 〈“𝐵𝐶𝐷𝐸𝐹𝐺”〉) | ||
Theorem | s1s7 14631 | Concatenation of fixed length strings. (Contributed by Mario Carneiro, 26-Feb-2016.) |
⊢ 〈“𝐴𝐵𝐶𝐷𝐸𝐹𝐺𝐻”〉 = (〈“𝐴”〉 ++ 〈“𝐵𝐶𝐷𝐸𝐹𝐺𝐻”〉) | ||
Theorem | s2s2 14632 | Concatenation of fixed length strings. (Contributed by Mario Carneiro, 26-Feb-2016.) |
⊢ 〈“𝐴𝐵𝐶𝐷”〉 = (〈“𝐴𝐵”〉 ++ 〈“𝐶𝐷”〉) | ||
Theorem | s4s2 14633 | Concatenation of fixed length strings. (Contributed by Mario Carneiro, 26-Feb-2016.) |
⊢ 〈“𝐴𝐵𝐶𝐷𝐸𝐹”〉 = (〈“𝐴𝐵𝐶𝐷”〉 ++ 〈“𝐸𝐹”〉) | ||
Theorem | s4s3 14634 | Concatenation of fixed length strings. (Contributed by Mario Carneiro, 26-Feb-2016.) |
⊢ 〈“𝐴𝐵𝐶𝐷𝐸𝐹𝐺”〉 = (〈“𝐴𝐵𝐶𝐷”〉 ++ 〈“𝐸𝐹𝐺”〉) | ||
Theorem | s4s4 14635 | Concatenation of fixed length strings. (Contributed by Mario Carneiro, 26-Feb-2016.) |
⊢ 〈“𝐴𝐵𝐶𝐷𝐸𝐹𝐺𝐻”〉 = (〈“𝐴𝐵𝐶𝐷”〉 ++ 〈“𝐸𝐹𝐺𝐻”〉) | ||
Theorem | s3s4 14636 | Concatenation of fixed length strings. (Contributed by AV, 1-Mar-2021.) |
⊢ 〈“𝐴𝐵𝐶𝐷𝐸𝐹𝐺”〉 = (〈“𝐴𝐵𝐶”〉 ++ 〈“𝐷𝐸𝐹𝐺”〉) | ||
Theorem | s2s5 14637 | Concatenation of fixed length strings. (Contributed by AV, 1-Mar-2021.) |
⊢ 〈“𝐴𝐵𝐶𝐷𝐸𝐹𝐺”〉 = (〈“𝐴𝐵”〉 ++ 〈“𝐶𝐷𝐸𝐹𝐺”〉) | ||
Theorem | s5s2 14638 | Concatenation of fixed length strings. (Contributed by AV, 1-Mar-2021.) |
⊢ 〈“𝐴𝐵𝐶𝐷𝐸𝐹𝐺”〉 = (〈“𝐴𝐵𝐶𝐷𝐸”〉 ++ 〈“𝐹𝐺”〉) | ||
Theorem | s2eq2s1eq 14639 | 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 14640 | Two length 2 words are equal iff the corresponding symbols are equal. (Contributed by AV, 20-Oct-2018.) |
⊢ (((𝐴 ∈ 𝑉 ∧ 𝐵 ∈ 𝑉) ∧ (𝐶 ∈ 𝑉 ∧ 𝐷 ∈ 𝑉)) → (〈“𝐴𝐵”〉 = 〈“𝐶𝐷”〉 ↔ (𝐴 = 𝐶 ∧ 𝐵 = 𝐷))) | ||
Theorem | s3eqs2s1eq 14641 | 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 14642 | Two length 3 words are equal iff the corresponding symbols are equal. (Contributed by AV, 4-Jan-2022.) |
⊢ (((𝐴 ∈ 𝑉 ∧ 𝐵 ∈ 𝑉 ∧ 𝐶 ∈ 𝑉) ∧ (𝐷 ∈ 𝑉 ∧ 𝐸 ∈ 𝑉 ∧ 𝐹 ∈ 𝑉)) → (〈“𝐴𝐵𝐶”〉 = 〈“𝐷𝐸𝐹”〉 ↔ (𝐴 = 𝐷 ∧ 𝐵 = 𝐸 ∧ 𝐶 = 𝐹))) | ||
Theorem | swrds2 14643 | 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 14644 | Extract two adjacent symbols from a word in reverse direction. (Contributed by AV, 11-May-2022.) |
⊢ ((𝑊 ∈ Word 𝑉 ∧ 𝑁 ∈ (2...(♯‘𝑊))) → (𝑊 substr 〈(𝑁 − 2), 𝑁〉) = 〈“(𝑊‘(𝑁 − 2))(𝑊‘(𝑁 − 1))”〉) | ||
Theorem | wrdlen2i 14645 | 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 14646 | 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 14647 | A word of length two. (Contributed by AV, 20-Oct-2018.) |
⊢ ((𝑆 ∈ 𝑉 ∧ 𝑇 ∈ 𝑉) → (𝑊 = {〈0, 𝑆〉, 〈1, 𝑇〉} ↔ ((𝑊 ∈ Word 𝑉 ∧ (♯‘𝑊) = 2) ∧ ((𝑊‘0) = 𝑆 ∧ (𝑊‘1) = 𝑇)))) | ||
Theorem | wrdlen2s2 14648 | A word of length two as doubleton word. (Contributed by AV, 20-Oct-2018.) |
⊢ ((𝑊 ∈ Word 𝑉 ∧ (♯‘𝑊) = 2) → 𝑊 = 〈“(𝑊‘0)(𝑊‘1)”〉) | ||
Theorem | wrdl2exs2 14649* | A word of length two is a doubleton word. (Contributed by AV, 25-Jan-2021.) |
⊢ ((𝑊 ∈ Word 𝑆 ∧ (♯‘𝑊) = 2) → ∃𝑠 ∈ 𝑆 ∃𝑡 ∈ 𝑆 𝑊 = 〈“𝑠𝑡”〉) | ||
Theorem | pfx2 14650 | A prefix of length two. (Contributed by AV, 15-May-2020.) |
⊢ ((𝑊 ∈ Word 𝑉 ∧ 2 ≤ (♯‘𝑊)) → (𝑊 prefix 2) = 〈“(𝑊‘0)(𝑊‘1)”〉) | ||
Theorem | wrd3tpop 14651 | 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 14652 | A word of length three as length 3 string. (Contributed by AV, 26-Jan-2021.) |
⊢ ((𝑊 ∈ Word 𝑉 ∧ (♯‘𝑊) = 3) → 𝑊 = 〈“(𝑊‘0)(𝑊‘1)(𝑊‘2)”〉) | ||
Theorem | repsw2 14653 | The "repeated symbol word" of length two. (Contributed by AV, 6-Nov-2018.) |
⊢ (𝑆 ∈ 𝑉 → (𝑆 repeatS 2) = 〈“𝑆𝑆”〉) | ||
Theorem | repsw3 14654 | The "repeated symbol word" of length three. (Contributed by AV, 6-Nov-2018.) |
⊢ (𝑆 ∈ 𝑉 → (𝑆 repeatS 3) = 〈“𝑆𝑆𝑆”〉) | ||
Theorem | swrd2lsw 14655 | 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 14656 | 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 14657 | 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 14658 | Obsolete version of ccatw2s1ccatws2 14657 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 14659 | Alternate proof of ccat2s1fvw 14339 using words of length 2, see df-s2 14551. 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 14660 | Obsolete version of ccat2s1fvwALT 14659 as of 28-Jan-2024. Alternate proof of ccat2s1fvwOLD 14340 using words of length 2, see df-s2 14551. 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 14661* | Lemma 1 for wrd2f1tovbij 14665. (Contributed by Alexander van der Vekens, 27-Jul-2018.) |
⊢ 𝐷 = {𝑤 ∈ Word 𝑉 ∣ ((♯‘𝑤) = 2 ∧ (𝑤‘0) = 𝑃 ∧ {(𝑤‘0), (𝑤‘1)} ∈ 𝑋)} & ⊢ 𝑅 = {𝑛 ∈ 𝑉 ∣ {𝑃, 𝑛} ∈ 𝑋} & ⊢ 𝐹 = (𝑡 ∈ 𝐷 ↦ (𝑡‘1)) ⇒ ⊢ 𝐹:𝐷⟶𝑅 | ||
Theorem | wwlktovf1 14662* | Lemma 2 for wrd2f1tovbij 14665. (Contributed by Alexander van der Vekens, 27-Jul-2018.) |
⊢ 𝐷 = {𝑤 ∈ Word 𝑉 ∣ ((♯‘𝑤) = 2 ∧ (𝑤‘0) = 𝑃 ∧ {(𝑤‘0), (𝑤‘1)} ∈ 𝑋)} & ⊢ 𝑅 = {𝑛 ∈ 𝑉 ∣ {𝑃, 𝑛} ∈ 𝑋} & ⊢ 𝐹 = (𝑡 ∈ 𝐷 ↦ (𝑡‘1)) ⇒ ⊢ 𝐹:𝐷–1-1→𝑅 | ||
Theorem | wwlktovfo 14663* | Lemma 3 for wrd2f1tovbij 14665. (Contributed by Alexander van der Vekens, 27-Jul-2018.) |
⊢ 𝐷 = {𝑤 ∈ Word 𝑉 ∣ ((♯‘𝑤) = 2 ∧ (𝑤‘0) = 𝑃 ∧ {(𝑤‘0), (𝑤‘1)} ∈ 𝑋)} & ⊢ 𝑅 = {𝑛 ∈ 𝑉 ∣ {𝑃, 𝑛} ∈ 𝑋} & ⊢ 𝐹 = (𝑡 ∈ 𝐷 ↦ (𝑡‘1)) ⇒ ⊢ (𝑃 ∈ 𝑉 → 𝐹:𝐷–onto→𝑅) | ||
Theorem | wwlktovf1o 14664* | Lemma 4 for wrd2f1tovbij 14665. (Contributed by Alexander van der Vekens, 28-Jul-2018.) |
⊢ 𝐷 = {𝑤 ∈ Word 𝑉 ∣ ((♯‘𝑤) = 2 ∧ (𝑤‘0) = 𝑃 ∧ {(𝑤‘0), (𝑤‘1)} ∈ 𝑋)} & ⊢ 𝑅 = {𝑛 ∈ 𝑉 ∣ {𝑃, 𝑛} ∈ 𝑋} & ⊢ 𝐹 = (𝑡 ∈ 𝐷 ↦ (𝑡‘1)) ⇒ ⊢ (𝑃 ∈ 𝑉 → 𝐹:𝐷–1-1-onto→𝑅) | ||
Theorem | wrd2f1tovbij 14665* | 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 14666 | 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 14667* | A word of length 3 is a length 3 string. (Contributed by AV, 18-May-2021.) |
⊢ ((𝑊 ∈ Word 𝑉 ∧ (♯‘𝑊) = 3) ↔ ∃𝑎 ∈ 𝑉 ∃𝑏 ∈ 𝑉 ∃𝑐 ∈ 𝑉 𝑊 = 〈“𝑎𝑏𝑐”〉) | ||
Theorem | s3sndisj 14668* | The singletons consisting of length 3 strings which have distinct third symbols are disjunct. (Contributed by AV, 17-May-2021.) |
⊢ ((𝐴 ∈ 𝑋 ∧ 𝐵 ∈ 𝑌) → Disj 𝑐 ∈ 𝑍 {〈“𝐴𝐵𝑐”〉}) | ||
Theorem | s3iunsndisj 14669* | 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 14670 | Letterwise operations on word concatenations. (Contributed by Thierry Arnoux, 28-Sep-2018.) |
⊢ (𝜑 → 𝐸 ∈ Word 𝑆) & ⊢ (𝜑 → 𝐹 ∈ Word 𝑆) & ⊢ (𝜑 → 𝐺 ∈ Word 𝑇) & ⊢ (𝜑 → 𝐻 ∈ Word 𝑇) & ⊢ (𝜑 → (♯‘𝐸) = (♯‘𝐺)) & ⊢ (𝜑 → (♯‘𝐹) = (♯‘𝐻)) ⇒ ⊢ (𝜑 → ((𝐸 ++ 𝐹) ∘f 𝑅(𝐺 ++ 𝐻)) = ((𝐸 ∘f 𝑅𝐺) ++ (𝐹 ∘f 𝑅𝐻))) | ||
Theorem | ofs1 14671 | Letterwise operations on a single letter word. (Contributed by Thierry Arnoux, 7-Oct-2018.) |
⊢ ((𝐴 ∈ 𝑆 ∧ 𝐵 ∈ 𝑇) → (〈“𝐴”〉 ∘f 𝑅〈“𝐵”〉) = 〈“(𝐴𝑅𝐵)”〉) | ||
Theorem | ofs2 14672 | 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 7013. 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 6015. 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 9478, which is a closure relative to a different transitive property, df-tr 5197. | ||
Theorem | coss12d 14673 | Subset deduction for composition of two classes. (Contributed by RP, 24-Dec-2019.) |
⊢ (𝜑 → 𝐴 ⊆ 𝐵) & ⊢ (𝜑 → 𝐶 ⊆ 𝐷) ⇒ ⊢ (𝜑 → (𝐴 ∘ 𝐶) ⊆ (𝐵 ∘ 𝐷)) | ||
Theorem | trrelssd 14674 | The composition of subclasses of a transitive relation is a subclass of that relation. (Contributed by RP, 24-Dec-2019.) |
⊢ (𝜑 → (𝑅 ∘ 𝑅) ⊆ 𝑅) & ⊢ (𝜑 → 𝑆 ⊆ 𝑅) & ⊢ (𝜑 → 𝑇 ⊆ 𝑅) ⇒ ⊢ (𝜑 → (𝑆 ∘ 𝑇) ⊆ 𝑅) | ||
Theorem | xpcogend 14675 | The most interesting case of the composition of two Cartesian products. (Contributed by RP, 24-Dec-2019.) |
⊢ (𝜑 → (𝐵 ∩ 𝐶) ≠ ∅) ⇒ ⊢ (𝜑 → ((𝐶 × 𝐷) ∘ (𝐴 × 𝐵)) = (𝐴 × 𝐷)) | ||
Theorem | xpcoidgend 14676 | 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 14677* | Two ways of saying that the composition of two relations is included in a third relation. See its special instance cotr2 14678 for the main application. (Contributed by RP, 22-Mar-2020.) |
⊢ dom 𝐵 ⊆ 𝐷 & ⊢ (ran 𝐵 ∩ dom 𝐴) ⊆ 𝐸 & ⊢ ran 𝐴 ⊆ 𝐹 ⇒ ⊢ ((𝐴 ∘ 𝐵) ⊆ 𝐶 ↔ ∀𝑥 ∈ 𝐷 ∀𝑦 ∈ 𝐸 ∀𝑧 ∈ 𝐹 ((𝑥𝐵𝑦 ∧ 𝑦𝐴𝑧) → 𝑥𝐶𝑧)) | ||
Theorem | cotr2 14678* | Two ways of saying a relation is transitive. Special instance of cotr2g 14677. (Contributed by RP, 22-Mar-2020.) |
⊢ dom 𝑅 ⊆ 𝐴 & ⊢ (dom 𝑅 ∩ ran 𝑅) ⊆ 𝐵 & ⊢ ran 𝑅 ⊆ 𝐶 ⇒ ⊢ ((𝑅 ∘ 𝑅) ⊆ 𝑅 ↔ ∀𝑥 ∈ 𝐴 ∀𝑦 ∈ 𝐵 ∀𝑧 ∈ 𝐶 ((𝑥𝑅𝑦 ∧ 𝑦𝑅𝑧) → 𝑥𝑅𝑧)) | ||
Theorem | cotr3 14679* | Two ways of saying a relation is transitive. (Contributed by RP, 22-Mar-2020.) |
⊢ 𝐴 = dom 𝑅 & ⊢ 𝐵 = (𝐴 ∩ 𝐶) & ⊢ 𝐶 = ran 𝑅 ⇒ ⊢ ((𝑅 ∘ 𝑅) ⊆ 𝑅 ↔ ∀𝑥 ∈ 𝐴 ∀𝑦 ∈ 𝐵 ∀𝑧 ∈ 𝐶 ((𝑥𝑅𝑦 ∧ 𝑦𝑅𝑧) → 𝑥𝑅𝑧)) | ||
Theorem | coemptyd 14680 | Deduction about composition of classes with no relational content in common. (Contributed by RP, 24-Dec-2019.) |
⊢ (𝜑 → (dom 𝐴 ∩ ran 𝐵) = ∅) ⇒ ⊢ (𝜑 → (𝐴 ∘ 𝐵) = ∅) | ||
Theorem | xptrrel 14681 | The cross product is always a transitive relation. (Contributed by RP, 24-Dec-2019.) |
⊢ ((𝐴 × 𝐵) ∘ (𝐴 × 𝐵)) ⊆ (𝐴 × 𝐵) | ||
Theorem | 0trrel 14682 | The empty class is a transitive relation. (Contributed by RP, 24-Dec-2019.) |
⊢ (∅ ∘ ∅) ⊆ ∅ | ||
Theorem | cleq1lem 14683 | Equality implies bijection. (Contributed by RP, 9-May-2020.) |
⊢ (𝐴 = 𝐵 → ((𝐴 ⊆ 𝐶 ∧ 𝜑) ↔ (𝐵 ⊆ 𝐶 ∧ 𝜑))) | ||
Theorem | cleq1 14684* | Equality of relations implies equality of closures. (Contributed by RP, 9-May-2020.) |
⊢ (𝑅 = 𝑆 → ∩ {𝑟 ∣ (𝑅 ⊆ 𝑟 ∧ 𝜑)} = ∩ {𝑟 ∣ (𝑆 ⊆ 𝑟 ∧ 𝜑)}) | ||
Theorem | clsslem 14685* | The closure of a subclass is a subclass of the closure. (Contributed by RP, 16-May-2020.) |
⊢ (𝑅 ⊆ 𝑆 → ∩ {𝑟 ∣ (𝑅 ⊆ 𝑟 ∧ 𝜑)} ⊆ ∩ {𝑟 ∣ (𝑆 ⊆ 𝑟 ∧ 𝜑)}) | ||
Syntax | ctcl 14686 | Extend class notation to include the transitive closure symbol. |
class t+ | ||
Syntax | crtcl 14687 | Extend class notation with reflexive-transitive closure. |
class t* | ||
Definition | df-trcl 14688* | Transitive closure of a relation. This is the smallest superset which has the transitive property. (Contributed by FL, 27-Jun-2011.) |
⊢ t+ = (𝑥 ∈ V ↦ ∩ {𝑧 ∣ (𝑥 ⊆ 𝑧 ∧ (𝑧 ∘ 𝑧) ⊆ 𝑧)}) | ||
Definition | df-rtrcl 14689* | Reflexive-transitive closure of a relation. This is the smallest superset which is reflexive property over all elements of its domain and range and has the transitive property. (Contributed by FL, 27-Jun-2011.) |
⊢ t* = (𝑥 ∈ V ↦ ∩ {𝑧 ∣ (( I ↾ (dom 𝑥 ∪ ran 𝑥)) ⊆ 𝑧 ∧ 𝑥 ⊆ 𝑧 ∧ (𝑧 ∘ 𝑧) ⊆ 𝑧)}) | ||
Theorem | trcleq1 14690* | Equality of relations implies equality of transitive closures. (Contributed by RP, 9-May-2020.) |
⊢ (𝑅 = 𝑆 → ∩ {𝑟 ∣ (𝑅 ⊆ 𝑟 ∧ (𝑟 ∘ 𝑟) ⊆ 𝑟)} = ∩ {𝑟 ∣ (𝑆 ⊆ 𝑟 ∧ (𝑟 ∘ 𝑟) ⊆ 𝑟)}) | ||
Theorem | trclsslem 14691* | The transitive closure (as a relation) of a subclass is a subclass of the transitive closure. (Contributed by RP, 3-May-2020.) |
⊢ (𝑅 ⊆ 𝑆 → ∩ {𝑟 ∣ (𝑅 ⊆ 𝑟 ∧ (𝑟 ∘ 𝑟) ⊆ 𝑟)} ⊆ ∩ {𝑟 ∣ (𝑆 ⊆ 𝑟 ∧ (𝑟 ∘ 𝑟) ⊆ 𝑟)}) | ||
Theorem | trcleq2lem 14692 | Equality implies bijection. (Contributed by RP, 5-May-2020.) |
⊢ (𝐴 = 𝐵 → ((𝑅 ⊆ 𝐴 ∧ (𝐴 ∘ 𝐴) ⊆ 𝐴) ↔ (𝑅 ⊆ 𝐵 ∧ (𝐵 ∘ 𝐵) ⊆ 𝐵))) | ||
Theorem | cvbtrcl 14693* | Change of bound variable in class of all transitive relations which are supersets of a relation. (Contributed by RP, 5-May-2020.) |
⊢ {𝑥 ∣ (𝑅 ⊆ 𝑥 ∧ (𝑥 ∘ 𝑥) ⊆ 𝑥)} = {𝑦 ∣ (𝑅 ⊆ 𝑦 ∧ (𝑦 ∘ 𝑦) ⊆ 𝑦)} | ||
Theorem | trcleq12lem 14694 | Equality implies bijection. (Contributed by RP, 9-May-2020.) |
⊢ ((𝑅 = 𝑆 ∧ 𝐴 = 𝐵) → ((𝑅 ⊆ 𝐴 ∧ (𝐴 ∘ 𝐴) ⊆ 𝐴) ↔ (𝑆 ⊆ 𝐵 ∧ (𝐵 ∘ 𝐵) ⊆ 𝐵))) | ||
Theorem | trclexlem 14695 | Existence of relation implies existence of union with Cartesian product of domain and range. (Contributed by RP, 5-May-2020.) |
⊢ (𝑅 ∈ 𝑉 → (𝑅 ∪ (dom 𝑅 × ran 𝑅)) ∈ V) | ||
Theorem | trclublem 14696* | If a relation exists then the class of transitive relations which are supersets of that relation is not empty. (Contributed by RP, 28-Apr-2020.) |
⊢ (𝑅 ∈ 𝑉 → (𝑅 ∪ (dom 𝑅 × ran 𝑅)) ∈ {𝑥 ∣ (𝑅 ⊆ 𝑥 ∧ (𝑥 ∘ 𝑥) ⊆ 𝑥)}) | ||
Theorem | trclubi 14697* | The Cartesian product of the domain and range of a relation is an upper bound for its transitive closure. (Contributed by RP, 2-Jan-2020.) (Revised by RP, 28-Apr-2020.) (Revised by AV, 26-Mar-2021.) |
⊢ Rel 𝑅 & ⊢ 𝑅 ∈ V ⇒ ⊢ ∩ {𝑠 ∣ (𝑅 ⊆ 𝑠 ∧ (𝑠 ∘ 𝑠) ⊆ 𝑠)} ⊆ (dom 𝑅 × ran 𝑅) | ||
Theorem | trclubgi 14698* | The union with the Cartesian product of its domain and range is an upper bound for a set's transitive closure. (Contributed by RP, 3-Jan-2020.) (Revised by RP, 28-Apr-2020.) (Revised by AV, 26-Mar-2021.) |
⊢ 𝑅 ∈ V ⇒ ⊢ ∩ {𝑠 ∣ (𝑅 ⊆ 𝑠 ∧ (𝑠 ∘ 𝑠) ⊆ 𝑠)} ⊆ (𝑅 ∪ (dom 𝑅 × ran 𝑅)) | ||
Theorem | trclub 14699* | The Cartesian product of the domain and range of a relation is an upper bound for its transitive closure. (Contributed by RP, 17-May-2020.) |
⊢ ((𝑅 ∈ 𝑉 ∧ Rel 𝑅) → ∩ {𝑟 ∣ (𝑅 ⊆ 𝑟 ∧ (𝑟 ∘ 𝑟) ⊆ 𝑟)} ⊆ (dom 𝑅 × ran 𝑅)) | ||
Theorem | trclubg 14700* | The union with the Cartesian product of its domain and range is an upper bound for a set's transitive closure (as a relation). (Contributed by RP, 17-May-2020.) |
⊢ (𝑅 ∈ 𝑉 → ∩ {𝑟 ∣ (𝑅 ⊆ 𝑟 ∧ (𝑟 ∘ 𝑟) ⊆ 𝑟)} ⊆ (𝑅 ∪ (dom 𝑅 × ran 𝑅))) |
< Previous Next > |
Copyright terms: Public domain | < Previous Next > |