| Metamath
Proof Explorer Theorem List (p. 331 of 497) | < 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: | (1-30845) |
(30846-32368) |
(32369-49617) |
| Type | Label | Description |
|---|---|---|
| Statement | ||
| Theorem | gsumhashmul 33001* | Express a group sum by grouping by nonzero values. (Contributed by Thierry Arnoux, 22-Jun-2024.) |
| ⊢ 𝐵 = (Base‘𝐺) & ⊢ 0 = (0g‘𝐺) & ⊢ · = (.g‘𝐺) & ⊢ (𝜑 → 𝐺 ∈ CMnd) & ⊢ (𝜑 → 𝐹:𝐴⟶𝐵) & ⊢ (𝜑 → 𝐹 finSupp 0 ) ⇒ ⊢ (𝜑 → (𝐺 Σg 𝐹) = (𝐺 Σg (𝑥 ∈ (ran 𝐹 ∖ { 0 }) ↦ ((♯‘(◡𝐹 “ {𝑥})) · 𝑥)))) | ||
| Theorem | xrge0tsmsd 33002* | Any finite or infinite sum in the nonnegative extended reals is uniquely convergent to the supremum of all finite sums. (Contributed by Mario Carneiro, 13-Sep-2015.) (Revised by Thierry Arnoux, 30-Jan-2017.) |
| ⊢ 𝐺 = (ℝ*𝑠 ↾s (0[,]+∞)) & ⊢ (𝜑 → 𝐴 ∈ 𝑉) & ⊢ (𝜑 → 𝐹:𝐴⟶(0[,]+∞)) & ⊢ (𝜑 → 𝑆 = sup(ran (𝑠 ∈ (𝒫 𝐴 ∩ Fin) ↦ (𝐺 Σg (𝐹 ↾ 𝑠))), ℝ*, < )) ⇒ ⊢ (𝜑 → (𝐺 tsums 𝐹) = {𝑆}) | ||
| Theorem | xrge0tsmsbi 33003 | Any limit of a finite or infinite sum in the nonnegative extended reals is the union of the sets limits, since this set is a singleton. (Contributed by Thierry Arnoux, 23-Jun-2017.) |
| ⊢ 𝐺 = (ℝ*𝑠 ↾s (0[,]+∞)) & ⊢ (𝜑 → 𝐴 ∈ 𝑉) & ⊢ (𝜑 → 𝐹:𝐴⟶(0[,]+∞)) ⇒ ⊢ (𝜑 → (𝐶 ∈ (𝐺 tsums 𝐹) ↔ 𝐶 = ∪ (𝐺 tsums 𝐹))) | ||
| Theorem | xrge0tsmseq 33004 | Any limit of a finite or infinite sum in the nonnegative extended reals is the union of the sets limits, since this set is a singleton. (Contributed by Thierry Arnoux, 24-Mar-2017.) |
| ⊢ 𝐺 = (ℝ*𝑠 ↾s (0[,]+∞)) & ⊢ (𝜑 → 𝐴 ∈ 𝑉) & ⊢ (𝜑 → 𝐹:𝐴⟶(0[,]+∞)) & ⊢ (𝜑 → 𝐶 ∈ (𝐺 tsums 𝐹)) ⇒ ⊢ (𝜑 → 𝐶 = ∪ (𝐺 tsums 𝐹)) | ||
| Theorem | gsumwun 33005* | In a commutative ring, a group sum of a word 𝑊 of characters taken from two submonoids 𝐸 and 𝐹 can be written as a simple sum. (Contributed by Thierry Arnoux, 6-Oct-2025.) |
| ⊢ + = (+g‘𝑀) & ⊢ (𝜑 → 𝑀 ∈ CMnd) & ⊢ (𝜑 → 𝐸 ∈ (SubMnd‘𝑀)) & ⊢ (𝜑 → 𝐹 ∈ (SubMnd‘𝑀)) & ⊢ (𝜑 → 𝑊 ∈ Word (𝐸 ∪ 𝐹)) ⇒ ⊢ (𝜑 → ∃𝑒 ∈ 𝐸 ∃𝑓 ∈ 𝐹 (𝑀 Σg 𝑊) = (𝑒 + 𝑓)) | ||
| Theorem | gsumwrd2dccatlem 33006* | Lemma for gsumwrd2dccat 33007. Expose a bijection 𝐹 between (ordered) pairs of words and words with a length of a subword. (Contributed by Thierry Arnoux, 5-Oct-2025.) |
| ⊢ 𝑈 = ∪ 𝑤 ∈ Word 𝐴({𝑤} × (0...(♯‘𝑤))) & ⊢ 𝐹 = (𝑎 ∈ (Word 𝐴 × Word 𝐴) ↦ 〈((1st ‘𝑎) ++ (2nd ‘𝑎)), (♯‘(1st ‘𝑎))〉) & ⊢ 𝐺 = (𝑏 ∈ 𝑈 ↦ 〈((1st ‘𝑏) prefix (2nd ‘𝑏)), ((1st ‘𝑏) substr 〈(2nd ‘𝑏), (♯‘(1st ‘𝑏))〉)〉) & ⊢ (𝜑 → 𝐴 ∈ 𝑉) ⇒ ⊢ (𝜑 → (𝐹:(Word 𝐴 × Word 𝐴)–1-1-onto→𝑈 ∧ ◡𝐹 = 𝐺)) | ||
| Theorem | gsumwrd2dccat 33007* | Rewrite a sum ranging over pairs of words as a sum of sums over concatenated subwords. (Contributed by Thierry Arnoux, 5-Oct-2025.) |
| ⊢ 𝐵 = (Base‘𝑀) & ⊢ 𝑍 = (0g‘𝑀) & ⊢ (𝜑 → 𝐹:(Word 𝐴 × Word 𝐴)⟶𝐵) & ⊢ (𝜑 → 𝐹 finSupp 𝑍) & ⊢ (𝜑 → 𝑀 ∈ CMnd) & ⊢ (𝜑 → 𝐴 ⊆ 𝐵) ⇒ ⊢ (𝜑 → (𝑀 Σg 𝐹) = (𝑀 Σg (𝑤 ∈ Word 𝐴 ↦ (𝑀 Σg (𝑗 ∈ (0...(♯‘𝑤)) ↦ (𝐹‘〈(𝑤 prefix 𝑗), (𝑤 substr 〈𝑗, (♯‘𝑤)〉)〉)))))) | ||
| Theorem | cntzun 33008 | The centralizer of a union is the intersection of the centralizers. (Contributed by Thierry Arnoux, 27-Nov-2023.) |
| ⊢ 𝐵 = (Base‘𝑀) & ⊢ 𝑍 = (Cntz‘𝑀) ⇒ ⊢ ((𝑋 ⊆ 𝐵 ∧ 𝑌 ⊆ 𝐵) → (𝑍‘(𝑋 ∪ 𝑌)) = ((𝑍‘𝑋) ∩ (𝑍‘𝑌))) | ||
| Theorem | cntzsnid 33009 | The centralizer of the identity element is the whole base set. (Contributed by Thierry Arnoux, 27-Nov-2023.) |
| ⊢ 𝐵 = (Base‘𝑀) & ⊢ 𝑍 = (Cntz‘𝑀) & ⊢ 0 = (0g‘𝑀) ⇒ ⊢ (𝑀 ∈ Mnd → (𝑍‘{ 0 }) = 𝐵) | ||
| Theorem | cntrcrng 33010 | The center of a ring is a commutative ring. (Contributed by Thierry Arnoux, 21-Aug-2023.) |
| ⊢ 𝑍 = (𝑅 ↾s (Cntr‘(mulGrp‘𝑅))) ⇒ ⊢ (𝑅 ∈ Ring → 𝑍 ∈ CRing) | ||
| Syntax | comnd 33011 | Extend class notation with the class of all right ordered monoids. |
| class oMnd | ||
| Syntax | cogrp 33012 | Extend class notation with the class of all right ordered groups. |
| class oGrp | ||
| Definition | df-omnd 33013* | Define class of all right ordered monoids. An ordered monoid is a monoid with a total ordering compatible with its operation. It is possible to use this definition also for left ordered monoids, by applying it to (oppg‘𝑀). (Contributed by Thierry Arnoux, 13-Mar-2018.) |
| ⊢ oMnd = {𝑔 ∈ Mnd ∣ [(Base‘𝑔) / 𝑣][(+g‘𝑔) / 𝑝][(le‘𝑔) / 𝑙](𝑔 ∈ Toset ∧ ∀𝑎 ∈ 𝑣 ∀𝑏 ∈ 𝑣 ∀𝑐 ∈ 𝑣 (𝑎𝑙𝑏 → (𝑎𝑝𝑐)𝑙(𝑏𝑝𝑐)))} | ||
| Definition | df-ogrp 33014 | Define class of all ordered groups. An ordered group is a group with a total ordering compatible with its operation. (Contributed by Thierry Arnoux, 13-Mar-2018.) |
| ⊢ oGrp = (Grp ∩ oMnd) | ||
| Theorem | isomnd 33015* | A (left) ordered monoid is a monoid with a total ordering compatible with its operation. (Contributed by Thierry Arnoux, 30-Jan-2018.) |
| ⊢ 𝐵 = (Base‘𝑀) & ⊢ + = (+g‘𝑀) & ⊢ ≤ = (le‘𝑀) ⇒ ⊢ (𝑀 ∈ oMnd ↔ (𝑀 ∈ Mnd ∧ 𝑀 ∈ Toset ∧ ∀𝑎 ∈ 𝐵 ∀𝑏 ∈ 𝐵 ∀𝑐 ∈ 𝐵 (𝑎 ≤ 𝑏 → (𝑎 + 𝑐) ≤ (𝑏 + 𝑐)))) | ||
| Theorem | isogrp 33016 | A (left-)ordered group is a group with a total ordering compatible with its operations. (Contributed by Thierry Arnoux, 23-Mar-2018.) |
| ⊢ (𝐺 ∈ oGrp ↔ (𝐺 ∈ Grp ∧ 𝐺 ∈ oMnd)) | ||
| Theorem | ogrpgrp 33017 | A left-ordered group is a group. (Contributed by Thierry Arnoux, 9-Jul-2018.) |
| ⊢ (𝐺 ∈ oGrp → 𝐺 ∈ Grp) | ||
| Theorem | omndmnd 33018 | A left-ordered monoid is a monoid. (Contributed by Thierry Arnoux, 13-Mar-2018.) |
| ⊢ (𝑀 ∈ oMnd → 𝑀 ∈ Mnd) | ||
| Theorem | omndtos 33019 | A left-ordered monoid is a totally ordered set. (Contributed by Thierry Arnoux, 13-Mar-2018.) |
| ⊢ (𝑀 ∈ oMnd → 𝑀 ∈ Toset) | ||
| Theorem | omndadd 33020 | In an ordered monoid, the ordering is compatible with group addition. (Contributed by Thierry Arnoux, 30-Jan-2018.) |
| ⊢ 𝐵 = (Base‘𝑀) & ⊢ ≤ = (le‘𝑀) & ⊢ + = (+g‘𝑀) ⇒ ⊢ ((𝑀 ∈ oMnd ∧ (𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵 ∧ 𝑍 ∈ 𝐵) ∧ 𝑋 ≤ 𝑌) → (𝑋 + 𝑍) ≤ (𝑌 + 𝑍)) | ||
| Theorem | omndaddr 33021 | In a right ordered monoid, the ordering is compatible with group addition. (Contributed by Thierry Arnoux, 30-Jan-2018.) |
| ⊢ 𝐵 = (Base‘𝑀) & ⊢ ≤ = (le‘𝑀) & ⊢ + = (+g‘𝑀) ⇒ ⊢ (((oppg‘𝑀) ∈ oMnd ∧ (𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵 ∧ 𝑍 ∈ 𝐵) ∧ 𝑋 ≤ 𝑌) → (𝑍 + 𝑋) ≤ (𝑍 + 𝑌)) | ||
| Theorem | omndadd2d 33022 | In a commutative left ordered monoid, the ordering is compatible with monoid addition. Double addition version. (Contributed by Thierry Arnoux, 30-Jan-2018.) |
| ⊢ 𝐵 = (Base‘𝑀) & ⊢ ≤ = (le‘𝑀) & ⊢ + = (+g‘𝑀) & ⊢ (𝜑 → 𝑀 ∈ oMnd) & ⊢ (𝜑 → 𝑊 ∈ 𝐵) & ⊢ (𝜑 → 𝑋 ∈ 𝐵) & ⊢ (𝜑 → 𝑌 ∈ 𝐵) & ⊢ (𝜑 → 𝑍 ∈ 𝐵) & ⊢ (𝜑 → 𝑋 ≤ 𝑍) & ⊢ (𝜑 → 𝑌 ≤ 𝑊) & ⊢ (𝜑 → 𝑀 ∈ CMnd) ⇒ ⊢ (𝜑 → (𝑋 + 𝑌) ≤ (𝑍 + 𝑊)) | ||
| Theorem | omndadd2rd 33023 | In a left- and right- ordered monoid, the ordering is compatible with monoid addition. Double addition version. (Contributed by Thierry Arnoux, 2-May-2018.) |
| ⊢ 𝐵 = (Base‘𝑀) & ⊢ ≤ = (le‘𝑀) & ⊢ + = (+g‘𝑀) & ⊢ (𝜑 → 𝑀 ∈ oMnd) & ⊢ (𝜑 → 𝑊 ∈ 𝐵) & ⊢ (𝜑 → 𝑋 ∈ 𝐵) & ⊢ (𝜑 → 𝑌 ∈ 𝐵) & ⊢ (𝜑 → 𝑍 ∈ 𝐵) & ⊢ (𝜑 → 𝑋 ≤ 𝑍) & ⊢ (𝜑 → 𝑌 ≤ 𝑊) & ⊢ (𝜑 → (oppg‘𝑀) ∈ oMnd) ⇒ ⊢ (𝜑 → (𝑋 + 𝑌) ≤ (𝑍 + 𝑊)) | ||
| Theorem | submomnd 33024 | A submonoid of an ordered monoid is also ordered. (Contributed by Thierry Arnoux, 23-Mar-2018.) |
| ⊢ ((𝑀 ∈ oMnd ∧ (𝑀 ↾s 𝐴) ∈ Mnd) → (𝑀 ↾s 𝐴) ∈ oMnd) | ||
| Theorem | xrge0omnd 33025 | The nonnegative extended real numbers form an ordered monoid. (Contributed by Thierry Arnoux, 22-Mar-2018.) |
| ⊢ (ℝ*𝑠 ↾s (0[,]+∞)) ∈ oMnd | ||
| Theorem | omndmul2 33026 | In an ordered monoid, the ordering is compatible with group power. This version does not require the monoid to be commutative. (Contributed by Thierry Arnoux, 23-Mar-2018.) |
| ⊢ 𝐵 = (Base‘𝑀) & ⊢ ≤ = (le‘𝑀) & ⊢ · = (.g‘𝑀) & ⊢ 0 = (0g‘𝑀) ⇒ ⊢ ((𝑀 ∈ oMnd ∧ (𝑋 ∈ 𝐵 ∧ 𝑁 ∈ ℕ0) ∧ 0 ≤ 𝑋) → 0 ≤ (𝑁 · 𝑋)) | ||
| Theorem | omndmul3 33027 | In an ordered monoid, the ordering is compatible with group power. This version does not require the monoid to be commutative. (Contributed by Thierry Arnoux, 23-Mar-2018.) |
| ⊢ 𝐵 = (Base‘𝑀) & ⊢ ≤ = (le‘𝑀) & ⊢ · = (.g‘𝑀) & ⊢ 0 = (0g‘𝑀) & ⊢ (𝜑 → 𝑀 ∈ oMnd) & ⊢ (𝜑 → 𝑁 ∈ ℕ0) & ⊢ (𝜑 → 𝑃 ∈ ℕ0) & ⊢ (𝜑 → 𝑁 ≤ 𝑃) & ⊢ (𝜑 → 𝑋 ∈ 𝐵) & ⊢ (𝜑 → 0 ≤ 𝑋) ⇒ ⊢ (𝜑 → (𝑁 · 𝑋) ≤ (𝑃 · 𝑋)) | ||
| Theorem | omndmul 33028 | In a commutative ordered monoid, the ordering is compatible with group power. (Contributed by Thierry Arnoux, 30-Jan-2018.) |
| ⊢ 𝐵 = (Base‘𝑀) & ⊢ ≤ = (le‘𝑀) & ⊢ · = (.g‘𝑀) & ⊢ (𝜑 → 𝑀 ∈ oMnd) & ⊢ (𝜑 → 𝑀 ∈ CMnd) & ⊢ (𝜑 → 𝑋 ∈ 𝐵) & ⊢ (𝜑 → 𝑌 ∈ 𝐵) & ⊢ (𝜑 → 𝑁 ∈ ℕ0) & ⊢ (𝜑 → 𝑋 ≤ 𝑌) ⇒ ⊢ (𝜑 → (𝑁 · 𝑋) ≤ (𝑁 · 𝑌)) | ||
| Theorem | ogrpinv0le 33029 | In an ordered group, the ordering is compatible with group inverse. (Contributed by Thierry Arnoux, 3-Sep-2018.) |
| ⊢ 𝐵 = (Base‘𝐺) & ⊢ ≤ = (le‘𝐺) & ⊢ 𝐼 = (invg‘𝐺) & ⊢ 0 = (0g‘𝐺) ⇒ ⊢ ((𝐺 ∈ oGrp ∧ 𝑋 ∈ 𝐵) → ( 0 ≤ 𝑋 ↔ (𝐼‘𝑋) ≤ 0 )) | ||
| Theorem | ogrpsub 33030 | In an ordered group, the ordering is compatible with group subtraction. (Contributed by Thierry Arnoux, 30-Jan-2018.) |
| ⊢ 𝐵 = (Base‘𝐺) & ⊢ ≤ = (le‘𝐺) & ⊢ − = (-g‘𝐺) ⇒ ⊢ ((𝐺 ∈ oGrp ∧ (𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵 ∧ 𝑍 ∈ 𝐵) ∧ 𝑋 ≤ 𝑌) → (𝑋 − 𝑍) ≤ (𝑌 − 𝑍)) | ||
| Theorem | ogrpaddlt 33031 | In an ordered group, strict ordering is compatible with group addition. (Contributed by Thierry Arnoux, 20-Jan-2018.) |
| ⊢ 𝐵 = (Base‘𝐺) & ⊢ < = (lt‘𝐺) & ⊢ + = (+g‘𝐺) ⇒ ⊢ ((𝐺 ∈ oGrp ∧ (𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵 ∧ 𝑍 ∈ 𝐵) ∧ 𝑋 < 𝑌) → (𝑋 + 𝑍) < (𝑌 + 𝑍)) | ||
| Theorem | ogrpaddltbi 33032 | In a right ordered group, strict ordering is compatible with group addition. (Contributed by Thierry Arnoux, 3-Sep-2018.) |
| ⊢ 𝐵 = (Base‘𝐺) & ⊢ < = (lt‘𝐺) & ⊢ + = (+g‘𝐺) ⇒ ⊢ ((𝐺 ∈ oGrp ∧ (𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵 ∧ 𝑍 ∈ 𝐵)) → (𝑋 < 𝑌 ↔ (𝑋 + 𝑍) < (𝑌 + 𝑍))) | ||
| Theorem | ogrpaddltrd 33033 | In a right ordered group, strict ordering is compatible with group addition. (Contributed by Thierry Arnoux, 3-Sep-2018.) |
| ⊢ 𝐵 = (Base‘𝐺) & ⊢ < = (lt‘𝐺) & ⊢ + = (+g‘𝐺) & ⊢ (𝜑 → 𝐺 ∈ 𝑉) & ⊢ (𝜑 → (oppg‘𝐺) ∈ oGrp) & ⊢ (𝜑 → 𝑋 ∈ 𝐵) & ⊢ (𝜑 → 𝑌 ∈ 𝐵) & ⊢ (𝜑 → 𝑍 ∈ 𝐵) & ⊢ (𝜑 → 𝑋 < 𝑌) ⇒ ⊢ (𝜑 → (𝑍 + 𝑋) < (𝑍 + 𝑌)) | ||
| Theorem | ogrpaddltrbid 33034 | In a right ordered group, strict ordering is compatible with group addition. (Contributed by Thierry Arnoux, 4-Sep-2018.) |
| ⊢ 𝐵 = (Base‘𝐺) & ⊢ < = (lt‘𝐺) & ⊢ + = (+g‘𝐺) & ⊢ (𝜑 → 𝐺 ∈ 𝑉) & ⊢ (𝜑 → (oppg‘𝐺) ∈ oGrp) & ⊢ (𝜑 → 𝑋 ∈ 𝐵) & ⊢ (𝜑 → 𝑌 ∈ 𝐵) & ⊢ (𝜑 → 𝑍 ∈ 𝐵) ⇒ ⊢ (𝜑 → (𝑋 < 𝑌 ↔ (𝑍 + 𝑋) < (𝑍 + 𝑌))) | ||
| Theorem | ogrpsublt 33035 | In an ordered group, strict ordering is compatible with group addition. (Contributed by Thierry Arnoux, 3-Sep-2018.) |
| ⊢ 𝐵 = (Base‘𝐺) & ⊢ < = (lt‘𝐺) & ⊢ − = (-g‘𝐺) ⇒ ⊢ ((𝐺 ∈ oGrp ∧ (𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵 ∧ 𝑍 ∈ 𝐵) ∧ 𝑋 < 𝑌) → (𝑋 − 𝑍) < (𝑌 − 𝑍)) | ||
| Theorem | ogrpinv0lt 33036 | In an ordered group, the ordering is compatible with group inverse. (Contributed by Thierry Arnoux, 3-Sep-2018.) |
| ⊢ 𝐵 = (Base‘𝐺) & ⊢ < = (lt‘𝐺) & ⊢ 𝐼 = (invg‘𝐺) & ⊢ 0 = (0g‘𝐺) ⇒ ⊢ ((𝐺 ∈ oGrp ∧ 𝑋 ∈ 𝐵) → ( 0 < 𝑋 ↔ (𝐼‘𝑋) < 0 )) | ||
| Theorem | ogrpinvlt 33037 | In an ordered group, the ordering is compatible with group inverse. (Contributed by Thierry Arnoux, 3-Sep-2018.) |
| ⊢ 𝐵 = (Base‘𝐺) & ⊢ < = (lt‘𝐺) & ⊢ 𝐼 = (invg‘𝐺) ⇒ ⊢ (((𝐺 ∈ oGrp ∧ (oppg‘𝐺) ∈ oGrp) ∧ 𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵) → (𝑋 < 𝑌 ↔ (𝐼‘𝑌) < (𝐼‘𝑋))) | ||
| Theorem | gsumle 33038 | A finite sum in an ordered monoid is monotonic. This proof would be much easier in an ordered group, where an inverse element would be available. (Contributed by Thierry Arnoux, 13-Mar-2018.) |
| ⊢ 𝐵 = (Base‘𝑀) & ⊢ ≤ = (le‘𝑀) & ⊢ (𝜑 → 𝑀 ∈ oMnd) & ⊢ (𝜑 → 𝑀 ∈ CMnd) & ⊢ (𝜑 → 𝐴 ∈ Fin) & ⊢ (𝜑 → 𝐹:𝐴⟶𝐵) & ⊢ (𝜑 → 𝐺:𝐴⟶𝐵) & ⊢ (𝜑 → 𝐹 ∘r ≤ 𝐺) ⇒ ⊢ (𝜑 → (𝑀 Σg 𝐹) ≤ (𝑀 Σg 𝐺)) | ||
| Theorem | symgfcoeu 33039* | Uniqueness property of permutations. (Contributed by Thierry Arnoux, 22-Aug-2020.) |
| ⊢ 𝐺 = (Base‘(SymGrp‘𝐷)) ⇒ ⊢ ((𝐷 ∈ 𝑉 ∧ 𝑃 ∈ 𝐺 ∧ 𝑄 ∈ 𝐺) → ∃!𝑝 ∈ 𝐺 𝑄 = (𝑃 ∘ 𝑝)) | ||
| Theorem | symgcom 33040 | Two permutations 𝑋 and 𝑌 commute if their orbits are disjoint. (Contributed by Thierry Arnoux, 15-Oct-2023.) |
| ⊢ 𝐺 = (SymGrp‘𝐴) & ⊢ 𝐵 = (Base‘𝐺) & ⊢ (𝜑 → 𝑋 ∈ 𝐵) & ⊢ (𝜑 → 𝑌 ∈ 𝐵) & ⊢ (𝜑 → (𝑋 ↾ 𝐸) = ( I ↾ 𝐸)) & ⊢ (𝜑 → (𝑌 ↾ 𝐹) = ( I ↾ 𝐹)) & ⊢ (𝜑 → (𝐸 ∩ 𝐹) = ∅) & ⊢ (𝜑 → (𝐸 ∪ 𝐹) = 𝐴) ⇒ ⊢ (𝜑 → (𝑋 ∘ 𝑌) = (𝑌 ∘ 𝑋)) | ||
| Theorem | symgcom2 33041 | Two permutations 𝑋 and 𝑌 commute if their orbits are disjoint. (Contributed by Thierry Arnoux, 17-Nov-2023.) |
| ⊢ 𝐺 = (SymGrp‘𝐴) & ⊢ 𝐵 = (Base‘𝐺) & ⊢ (𝜑 → 𝑋 ∈ 𝐵) & ⊢ (𝜑 → 𝑌 ∈ 𝐵) & ⊢ (𝜑 → (dom (𝑋 ∖ I ) ∩ dom (𝑌 ∖ I )) = ∅) ⇒ ⊢ (𝜑 → (𝑋 ∘ 𝑌) = (𝑌 ∘ 𝑋)) | ||
| Theorem | symgcntz 33042* | All elements of a (finite) set of permutations commute if their orbits are disjoint. (Contributed by Thierry Arnoux, 20-Nov-2023.) |
| ⊢ 𝑆 = (SymGrp‘𝐷) & ⊢ 𝐵 = (Base‘𝑆) & ⊢ 𝑍 = (Cntz‘𝑆) & ⊢ (𝜑 → 𝐴 ⊆ 𝐵) & ⊢ (𝜑 → Disj 𝑥 ∈ 𝐴 dom (𝑥 ∖ I )) ⇒ ⊢ (𝜑 → 𝐴 ⊆ (𝑍‘𝐴)) | ||
| Theorem | odpmco 33043 | The composition of two odd permutations is even. (Contributed by Thierry Arnoux, 15-Oct-2023.) |
| ⊢ 𝑆 = (SymGrp‘𝐷) & ⊢ 𝐵 = (Base‘𝑆) & ⊢ 𝐴 = (pmEven‘𝐷) ⇒ ⊢ ((𝐷 ∈ Fin ∧ 𝑋 ∈ (𝐵 ∖ 𝐴) ∧ 𝑌 ∈ (𝐵 ∖ 𝐴)) → (𝑋 ∘ 𝑌) ∈ 𝐴) | ||
| Theorem | symgsubg 33044 | The value of the group subtraction operation of the symmetric group. (Contributed by Thierry Arnoux, 15-Oct-2023.) |
| ⊢ 𝐺 = (SymGrp‘𝐴) & ⊢ 𝐵 = (Base‘𝐺) & ⊢ − = (-g‘𝐺) ⇒ ⊢ ((𝑋 ∈ 𝐵 ∧ 𝑌 ∈ 𝐵) → (𝑋 − 𝑌) = (𝑋 ∘ ◡𝑌)) | ||
| Theorem | pmtrprfv2 33045 | In a transposition of two given points, each maps to the other. (Contributed by Thierry Arnoux, 22-Aug-2020.) |
| ⊢ 𝑇 = (pmTrsp‘𝐷) ⇒ ⊢ ((𝐷 ∈ 𝑉 ∧ (𝑋 ∈ 𝐷 ∧ 𝑌 ∈ 𝐷 ∧ 𝑋 ≠ 𝑌)) → ((𝑇‘{𝑋, 𝑌})‘𝑌) = 𝑋) | ||
| Theorem | pmtrcnel 33046 | Composing a permutation 𝐹 with a transposition which results in moving at least one less point. Here the set of points moved by a permutation 𝐹 is expressed as dom (𝐹 ∖ I ). (Contributed by Thierry Arnoux, 16-Nov-2023.) |
| ⊢ 𝑆 = (SymGrp‘𝐷) & ⊢ 𝑇 = (pmTrsp‘𝐷) & ⊢ 𝐵 = (Base‘𝑆) & ⊢ 𝐽 = (𝐹‘𝐼) & ⊢ (𝜑 → 𝐷 ∈ 𝑉) & ⊢ (𝜑 → 𝐹 ∈ 𝐵) & ⊢ (𝜑 → 𝐼 ∈ dom (𝐹 ∖ I )) ⇒ ⊢ (𝜑 → dom (((𝑇‘{𝐼, 𝐽}) ∘ 𝐹) ∖ I ) ⊆ (dom (𝐹 ∖ I ) ∖ {𝐼})) | ||
| Theorem | pmtrcnel2 33047 | Variation on pmtrcnel 33046. (Contributed by Thierry Arnoux, 16-Nov-2023.) |
| ⊢ 𝑆 = (SymGrp‘𝐷) & ⊢ 𝑇 = (pmTrsp‘𝐷) & ⊢ 𝐵 = (Base‘𝑆) & ⊢ 𝐽 = (𝐹‘𝐼) & ⊢ (𝜑 → 𝐷 ∈ 𝑉) & ⊢ (𝜑 → 𝐹 ∈ 𝐵) & ⊢ (𝜑 → 𝐼 ∈ dom (𝐹 ∖ I )) ⇒ ⊢ (𝜑 → (dom (𝐹 ∖ I ) ∖ {𝐼, 𝐽}) ⊆ dom (((𝑇‘{𝐼, 𝐽}) ∘ 𝐹) ∖ I )) | ||
| Theorem | pmtrcnelor 33048 | Composing a permutation 𝐹 with a transposition which results in moving one or two less points. (Contributed by Thierry Arnoux, 16-Nov-2023.) |
| ⊢ 𝑆 = (SymGrp‘𝐷) & ⊢ 𝑇 = (pmTrsp‘𝐷) & ⊢ 𝐵 = (Base‘𝑆) & ⊢ 𝐽 = (𝐹‘𝐼) & ⊢ (𝜑 → 𝐷 ∈ 𝑉) & ⊢ (𝜑 → 𝐹 ∈ 𝐵) & ⊢ (𝜑 → 𝐼 ∈ dom (𝐹 ∖ I )) & ⊢ 𝐸 = dom (𝐹 ∖ I ) & ⊢ 𝐴 = dom (((𝑇‘{𝐼, 𝐽}) ∘ 𝐹) ∖ I ) ⇒ ⊢ (𝜑 → (𝐴 = (𝐸 ∖ {𝐼, 𝐽}) ∨ 𝐴 = (𝐸 ∖ {𝐼}))) | ||
| Theorem | fzo0pmtrlast 33049* | Reorder a half-open integer range based at 0, so that the given index 𝐼 is at the end. (Contributed by Thierry Arnoux, 27-May-2025.) |
| ⊢ 𝐽 = (0..^𝑁) & ⊢ (𝜑 → 𝐼 ∈ 𝐽) ⇒ ⊢ (𝜑 → ∃𝑠(𝑠:𝐽–1-1-onto→𝐽 ∧ (𝑠‘(𝑁 − 1)) = 𝐼)) | ||
| Theorem | wrdpmtrlast 33050* | Reorder a word, so that the symbol given at index 𝐼 is at the end. (Contributed by Thierry Arnoux, 27-May-2025.) |
| ⊢ 𝐽 = (0..^(♯‘𝑊)) & ⊢ (𝜑 → 𝐼 ∈ 𝐽) & ⊢ (𝜑 → 𝑊 ∈ Word 𝑆) & ⊢ 𝑈 = ((𝑊 ∘ 𝑠) prefix ((♯‘𝑊) − 1)) ⇒ ⊢ (𝜑 → ∃𝑠(𝑠:𝐽–1-1-onto→𝐽 ∧ (𝑊 ∘ 𝑠) = (𝑈 ++ 〈“(𝑊‘𝐼)”〉))) | ||
| Theorem | pmtridf1o 33051 | Transpositions of 𝑋 and 𝑌 (understood to be the identity when 𝑋 = 𝑌), are bijections. (Contributed by Thierry Arnoux, 1-Jan-2022.) |
| ⊢ (𝜑 → 𝐴 ∈ 𝑉) & ⊢ (𝜑 → 𝑋 ∈ 𝐴) & ⊢ (𝜑 → 𝑌 ∈ 𝐴) & ⊢ 𝑇 = if(𝑋 = 𝑌, ( I ↾ 𝐴), ((pmTrsp‘𝐴)‘{𝑋, 𝑌})) ⇒ ⊢ (𝜑 → 𝑇:𝐴–1-1-onto→𝐴) | ||
| Theorem | pmtridfv1 33052 | Value at X of the transposition of 𝑋 and 𝑌 (understood to be the identity when X = Y ). (Contributed by Thierry Arnoux, 3-Jan-2022.) |
| ⊢ (𝜑 → 𝐴 ∈ 𝑉) & ⊢ (𝜑 → 𝑋 ∈ 𝐴) & ⊢ (𝜑 → 𝑌 ∈ 𝐴) & ⊢ 𝑇 = if(𝑋 = 𝑌, ( I ↾ 𝐴), ((pmTrsp‘𝐴)‘{𝑋, 𝑌})) ⇒ ⊢ (𝜑 → (𝑇‘𝑋) = 𝑌) | ||
| Theorem | pmtridfv2 33053 | Value at Y of the transposition of 𝑋 and 𝑌 (understood to be the identity when X = Y ). (Contributed by Thierry Arnoux, 3-Jan-2022.) |
| ⊢ (𝜑 → 𝐴 ∈ 𝑉) & ⊢ (𝜑 → 𝑋 ∈ 𝐴) & ⊢ (𝜑 → 𝑌 ∈ 𝐴) & ⊢ 𝑇 = if(𝑋 = 𝑌, ( I ↾ 𝐴), ((pmTrsp‘𝐴)‘{𝑋, 𝑌})) ⇒ ⊢ (𝜑 → (𝑇‘𝑌) = 𝑋) | ||
| Theorem | psgnid 33054 | Permutation sign of the identity. (Contributed by Thierry Arnoux, 21-Aug-2020.) |
| ⊢ 𝑆 = (pmSgn‘𝐷) ⇒ ⊢ (𝐷 ∈ Fin → (𝑆‘( I ↾ 𝐷)) = 1) | ||
| Theorem | psgndmfi 33055 | For a finite base set, the permutation sign is defined for all permutations. (Contributed by Thierry Arnoux, 22-Aug-2020.) |
| ⊢ 𝑆 = (pmSgn‘𝐷) & ⊢ 𝐺 = (Base‘(SymGrp‘𝐷)) ⇒ ⊢ (𝐷 ∈ Fin → 𝑆 Fn 𝐺) | ||
| Theorem | pmtrto1cl 33056 | Useful lemma for the following theorems. (Contributed by Thierry Arnoux, 21-Aug-2020.) |
| ⊢ 𝐷 = (1...𝑁) & ⊢ 𝑇 = (pmTrsp‘𝐷) ⇒ ⊢ ((𝐾 ∈ ℕ ∧ (𝐾 + 1) ∈ 𝐷) → (𝑇‘{𝐾, (𝐾 + 1)}) ∈ ran 𝑇) | ||
| Theorem | psgnfzto1stlem 33057* | Lemma for psgnfzto1st 33062. Our permutation of rank (𝑛 + 1) can be written as a permutation of rank 𝑛 composed with a transposition. (Contributed by Thierry Arnoux, 21-Aug-2020.) |
| ⊢ 𝐷 = (1...𝑁) ⇒ ⊢ ((𝐾 ∈ ℕ ∧ (𝐾 + 1) ∈ 𝐷) → (𝑖 ∈ 𝐷 ↦ if(𝑖 = 1, (𝐾 + 1), if(𝑖 ≤ (𝐾 + 1), (𝑖 − 1), 𝑖))) = (((pmTrsp‘𝐷)‘{𝐾, (𝐾 + 1)}) ∘ (𝑖 ∈ 𝐷 ↦ if(𝑖 = 1, 𝐾, if(𝑖 ≤ 𝐾, (𝑖 − 1), 𝑖))))) | ||
| Theorem | fzto1stfv1 33058* | Value of our permutation 𝑃 at 1. (Contributed by Thierry Arnoux, 23-Aug-2020.) |
| ⊢ 𝐷 = (1...𝑁) & ⊢ 𝑃 = (𝑖 ∈ 𝐷 ↦ if(𝑖 = 1, 𝐼, if(𝑖 ≤ 𝐼, (𝑖 − 1), 𝑖))) ⇒ ⊢ (𝐼 ∈ 𝐷 → (𝑃‘1) = 𝐼) | ||
| Theorem | fzto1st1 33059* | Special case where the permutation defined in psgnfzto1st 33062 is the identity. (Contributed by Thierry Arnoux, 21-Aug-2020.) |
| ⊢ 𝐷 = (1...𝑁) & ⊢ 𝑃 = (𝑖 ∈ 𝐷 ↦ if(𝑖 = 1, 𝐼, if(𝑖 ≤ 𝐼, (𝑖 − 1), 𝑖))) ⇒ ⊢ (𝐼 = 1 → 𝑃 = ( I ↾ 𝐷)) | ||
| Theorem | fzto1st 33060* | The function moving one element to the first position (and shifting all elements before it) is a permutation. (Contributed by Thierry Arnoux, 21-Aug-2020.) |
| ⊢ 𝐷 = (1...𝑁) & ⊢ 𝑃 = (𝑖 ∈ 𝐷 ↦ if(𝑖 = 1, 𝐼, if(𝑖 ≤ 𝐼, (𝑖 − 1), 𝑖))) & ⊢ 𝐺 = (SymGrp‘𝐷) & ⊢ 𝐵 = (Base‘𝐺) ⇒ ⊢ (𝐼 ∈ 𝐷 → 𝑃 ∈ 𝐵) | ||
| Theorem | fzto1stinvn 33061* | Value of the inverse of our permutation 𝑃 at 𝐼. (Contributed by Thierry Arnoux, 23-Aug-2020.) |
| ⊢ 𝐷 = (1...𝑁) & ⊢ 𝑃 = (𝑖 ∈ 𝐷 ↦ if(𝑖 = 1, 𝐼, if(𝑖 ≤ 𝐼, (𝑖 − 1), 𝑖))) & ⊢ 𝐺 = (SymGrp‘𝐷) & ⊢ 𝐵 = (Base‘𝐺) ⇒ ⊢ (𝐼 ∈ 𝐷 → (◡𝑃‘𝐼) = 1) | ||
| Theorem | psgnfzto1st 33062* | The permutation sign for moving one element to the first position. (Contributed by Thierry Arnoux, 21-Aug-2020.) |
| ⊢ 𝐷 = (1...𝑁) & ⊢ 𝑃 = (𝑖 ∈ 𝐷 ↦ if(𝑖 = 1, 𝐼, if(𝑖 ≤ 𝐼, (𝑖 − 1), 𝑖))) & ⊢ 𝐺 = (SymGrp‘𝐷) & ⊢ 𝐵 = (Base‘𝐺) & ⊢ 𝑆 = (pmSgn‘𝐷) ⇒ ⊢ (𝐼 ∈ 𝐷 → (𝑆‘𝑃) = (-1↑(𝐼 + 1))) | ||
| Syntax | ctocyc 33063 | Extend class notation with the permutation cycle builder. |
| class toCyc | ||
| Definition | df-tocyc 33064* | Define a convenience permutation cycle builder. Given a list of elements to be cycled, in the form of a word, this function produces the corresponding permutation cycle. See definition in [Lang] p. 30. (Contributed by Thierry Arnoux, 19-Sep-2023.) |
| ⊢ toCyc = (𝑑 ∈ V ↦ (𝑤 ∈ {𝑢 ∈ Word 𝑑 ∣ 𝑢:dom 𝑢–1-1→𝑑} ↦ (( I ↾ (𝑑 ∖ ran 𝑤)) ∪ ((𝑤 cyclShift 1) ∘ ◡𝑤)))) | ||
| Theorem | tocycval 33065* | Value of the cycle builder. (Contributed by Thierry Arnoux, 22-Sep-2023.) |
| ⊢ 𝐶 = (toCyc‘𝐷) ⇒ ⊢ (𝐷 ∈ 𝑉 → 𝐶 = (𝑤 ∈ {𝑢 ∈ Word 𝐷 ∣ 𝑢:dom 𝑢–1-1→𝐷} ↦ (( I ↾ (𝐷 ∖ ran 𝑤)) ∪ ((𝑤 cyclShift 1) ∘ ◡𝑤)))) | ||
| Theorem | tocycfv 33066 | Function value of a permutation cycle built from a word. (Contributed by Thierry Arnoux, 18-Sep-2023.) |
| ⊢ 𝐶 = (toCyc‘𝐷) & ⊢ (𝜑 → 𝐷 ∈ 𝑉) & ⊢ (𝜑 → 𝑊 ∈ Word 𝐷) & ⊢ (𝜑 → 𝑊:dom 𝑊–1-1→𝐷) ⇒ ⊢ (𝜑 → (𝐶‘𝑊) = (( I ↾ (𝐷 ∖ ran 𝑊)) ∪ ((𝑊 cyclShift 1) ∘ ◡𝑊))) | ||
| Theorem | tocycfvres1 33067 | A cyclic permutation is a cyclic shift on its orbit. (Contributed by Thierry Arnoux, 15-Oct-2023.) |
| ⊢ 𝐶 = (toCyc‘𝐷) & ⊢ (𝜑 → 𝐷 ∈ 𝑉) & ⊢ (𝜑 → 𝑊 ∈ Word 𝐷) & ⊢ (𝜑 → 𝑊:dom 𝑊–1-1→𝐷) ⇒ ⊢ (𝜑 → ((𝐶‘𝑊) ↾ ran 𝑊) = ((𝑊 cyclShift 1) ∘ ◡𝑊)) | ||
| Theorem | tocycfvres2 33068 | A cyclic permutation is the identity outside of its orbit. (Contributed by Thierry Arnoux, 15-Oct-2023.) |
| ⊢ 𝐶 = (toCyc‘𝐷) & ⊢ (𝜑 → 𝐷 ∈ 𝑉) & ⊢ (𝜑 → 𝑊 ∈ Word 𝐷) & ⊢ (𝜑 → 𝑊:dom 𝑊–1-1→𝐷) ⇒ ⊢ (𝜑 → ((𝐶‘𝑊) ↾ (𝐷 ∖ ran 𝑊)) = ( I ↾ (𝐷 ∖ ran 𝑊))) | ||
| Theorem | cycpmfvlem 33069 | Lemma for cycpmfv1 33070 and cycpmfv2 33071. (Contributed by Thierry Arnoux, 22-Sep-2023.) |
| ⊢ 𝐶 = (toCyc‘𝐷) & ⊢ (𝜑 → 𝐷 ∈ 𝑉) & ⊢ (𝜑 → 𝑊 ∈ Word 𝐷) & ⊢ (𝜑 → 𝑊:dom 𝑊–1-1→𝐷) & ⊢ (𝜑 → 𝑁 ∈ (0..^(♯‘𝑊))) ⇒ ⊢ (𝜑 → ((𝐶‘𝑊)‘(𝑊‘𝑁)) = (((𝑊 cyclShift 1) ∘ ◡𝑊)‘(𝑊‘𝑁))) | ||
| Theorem | cycpmfv1 33070 | Value of a cycle function for any element but the last. (Contributed by Thierry Arnoux, 22-Sep-2023.) |
| ⊢ 𝐶 = (toCyc‘𝐷) & ⊢ (𝜑 → 𝐷 ∈ 𝑉) & ⊢ (𝜑 → 𝑊 ∈ Word 𝐷) & ⊢ (𝜑 → 𝑊:dom 𝑊–1-1→𝐷) & ⊢ (𝜑 → 𝑁 ∈ (0..^((♯‘𝑊) − 1))) ⇒ ⊢ (𝜑 → ((𝐶‘𝑊)‘(𝑊‘𝑁)) = (𝑊‘(𝑁 + 1))) | ||
| Theorem | cycpmfv2 33071 | Value of a cycle function for the last element of the orbit. (Contributed by Thierry Arnoux, 22-Sep-2023.) |
| ⊢ 𝐶 = (toCyc‘𝐷) & ⊢ (𝜑 → 𝐷 ∈ 𝑉) & ⊢ (𝜑 → 𝑊 ∈ Word 𝐷) & ⊢ (𝜑 → 𝑊:dom 𝑊–1-1→𝐷) & ⊢ (𝜑 → 0 < (♯‘𝑊)) & ⊢ (𝜑 → 𝑁 = ((♯‘𝑊) − 1)) ⇒ ⊢ (𝜑 → ((𝐶‘𝑊)‘(𝑊‘𝑁)) = (𝑊‘0)) | ||
| Theorem | cycpmfv3 33072 | Values outside of the orbit are unchanged by a cycle. (Contributed by Thierry Arnoux, 22-Sep-2023.) |
| ⊢ 𝐶 = (toCyc‘𝐷) & ⊢ (𝜑 → 𝐷 ∈ 𝑉) & ⊢ (𝜑 → 𝑊 ∈ Word 𝐷) & ⊢ (𝜑 → 𝑊:dom 𝑊–1-1→𝐷) & ⊢ (𝜑 → 𝑋 ∈ 𝐷) & ⊢ (𝜑 → ¬ 𝑋 ∈ ran 𝑊) ⇒ ⊢ (𝜑 → ((𝐶‘𝑊)‘𝑋) = 𝑋) | ||
| Theorem | cycpmcl 33073 | Cyclic permutations are permutations. (Contributed by Thierry Arnoux, 24-Sep-2023.) |
| ⊢ 𝐶 = (toCyc‘𝐷) & ⊢ (𝜑 → 𝐷 ∈ 𝑉) & ⊢ (𝜑 → 𝑊 ∈ Word 𝐷) & ⊢ (𝜑 → 𝑊:dom 𝑊–1-1→𝐷) & ⊢ 𝑆 = (SymGrp‘𝐷) ⇒ ⊢ (𝜑 → (𝐶‘𝑊) ∈ (Base‘𝑆)) | ||
| Theorem | tocycf 33074* | The permutation cycle builder as a function. (Contributed by Thierry Arnoux, 25-Sep-2023.) |
| ⊢ 𝐶 = (toCyc‘𝐷) & ⊢ 𝑆 = (SymGrp‘𝐷) & ⊢ 𝐵 = (Base‘𝑆) ⇒ ⊢ (𝐷 ∈ 𝑉 → 𝐶:{𝑤 ∈ Word 𝐷 ∣ 𝑤:dom 𝑤–1-1→𝐷}⟶𝐵) | ||
| Theorem | tocyc01 33075 | Permutation cycles built from the empty set or a singleton are the identity. (Contributed by Thierry Arnoux, 21-Nov-2023.) |
| ⊢ 𝐶 = (toCyc‘𝐷) ⇒ ⊢ ((𝐷 ∈ 𝑉 ∧ 𝑊 ∈ (dom 𝐶 ∩ (◡♯ “ {0, 1}))) → (𝐶‘𝑊) = ( I ↾ 𝐷)) | ||
| Theorem | cycpm2tr 33076 | A cyclic permutation of 2 elements is a transposition. (Contributed by Thierry Arnoux, 24-Sep-2023.) |
| ⊢ 𝐶 = (toCyc‘𝐷) & ⊢ (𝜑 → 𝐷 ∈ 𝑉) & ⊢ (𝜑 → 𝐼 ∈ 𝐷) & ⊢ (𝜑 → 𝐽 ∈ 𝐷) & ⊢ (𝜑 → 𝐼 ≠ 𝐽) & ⊢ 𝑇 = (pmTrsp‘𝐷) ⇒ ⊢ (𝜑 → (𝐶‘〈“𝐼𝐽”〉) = (𝑇‘{𝐼, 𝐽})) | ||
| Theorem | cycpm2cl 33077 | Closure for the 2-cycles. (Contributed by Thierry Arnoux, 24-Sep-2023.) |
| ⊢ 𝐶 = (toCyc‘𝐷) & ⊢ (𝜑 → 𝐷 ∈ 𝑉) & ⊢ (𝜑 → 𝐼 ∈ 𝐷) & ⊢ (𝜑 → 𝐽 ∈ 𝐷) & ⊢ (𝜑 → 𝐼 ≠ 𝐽) & ⊢ 𝑆 = (SymGrp‘𝐷) ⇒ ⊢ (𝜑 → (𝐶‘〈“𝐼𝐽”〉) ∈ (Base‘𝑆)) | ||
| Theorem | cyc2fv1 33078 | Function value of a 2-cycle at the first point. (Contributed by Thierry Arnoux, 24-Sep-2023.) |
| ⊢ 𝐶 = (toCyc‘𝐷) & ⊢ (𝜑 → 𝐷 ∈ 𝑉) & ⊢ (𝜑 → 𝐼 ∈ 𝐷) & ⊢ (𝜑 → 𝐽 ∈ 𝐷) & ⊢ (𝜑 → 𝐼 ≠ 𝐽) & ⊢ 𝑆 = (SymGrp‘𝐷) ⇒ ⊢ (𝜑 → ((𝐶‘〈“𝐼𝐽”〉)‘𝐼) = 𝐽) | ||
| Theorem | cyc2fv2 33079 | Function value of a 2-cycle at the second point. (Contributed by Thierry Arnoux, 24-Sep-2023.) |
| ⊢ 𝐶 = (toCyc‘𝐷) & ⊢ (𝜑 → 𝐷 ∈ 𝑉) & ⊢ (𝜑 → 𝐼 ∈ 𝐷) & ⊢ (𝜑 → 𝐽 ∈ 𝐷) & ⊢ (𝜑 → 𝐼 ≠ 𝐽) & ⊢ 𝑆 = (SymGrp‘𝐷) ⇒ ⊢ (𝜑 → ((𝐶‘〈“𝐼𝐽”〉)‘𝐽) = 𝐼) | ||
| Theorem | trsp2cyc 33080* | Exhibit the word a transposition corresponds to, as a cycle. (Contributed by Thierry Arnoux, 25-Sep-2023.) |
| ⊢ 𝑇 = ran (pmTrsp‘𝐷) & ⊢ 𝐶 = (toCyc‘𝐷) ⇒ ⊢ ((𝐷 ∈ 𝑉 ∧ 𝑃 ∈ 𝑇) → ∃𝑖 ∈ 𝐷 ∃𝑗 ∈ 𝐷 (𝑖 ≠ 𝑗 ∧ 𝑃 = (𝐶‘〈“𝑖𝑗”〉))) | ||
| Theorem | cycpmco2f1 33081 | The word U used in cycpmco2 33090 is injective, so it can represent a cycle and form a cyclic permutation (𝑀‘𝑈). (Contributed by Thierry Arnoux, 4-Jan-2024.) |
| ⊢ 𝑀 = (toCyc‘𝐷) & ⊢ 𝑆 = (SymGrp‘𝐷) & ⊢ (𝜑 → 𝐷 ∈ 𝑉) & ⊢ (𝜑 → 𝑊 ∈ dom 𝑀) & ⊢ (𝜑 → 𝐼 ∈ (𝐷 ∖ ran 𝑊)) & ⊢ (𝜑 → 𝐽 ∈ ran 𝑊) & ⊢ 𝐸 = ((◡𝑊‘𝐽) + 1) & ⊢ 𝑈 = (𝑊 splice 〈𝐸, 𝐸, 〈“𝐼”〉〉) ⇒ ⊢ (𝜑 → 𝑈:dom 𝑈–1-1→𝐷) | ||
| Theorem | cycpmco2rn 33082 | The orbit of the composition of a cyclic permutation and a well-chosen transposition is one element more than the orbit of the original permutation. (Contributed by Thierry Arnoux, 4-Jan-2024.) |
| ⊢ 𝑀 = (toCyc‘𝐷) & ⊢ 𝑆 = (SymGrp‘𝐷) & ⊢ (𝜑 → 𝐷 ∈ 𝑉) & ⊢ (𝜑 → 𝑊 ∈ dom 𝑀) & ⊢ (𝜑 → 𝐼 ∈ (𝐷 ∖ ran 𝑊)) & ⊢ (𝜑 → 𝐽 ∈ ran 𝑊) & ⊢ 𝐸 = ((◡𝑊‘𝐽) + 1) & ⊢ 𝑈 = (𝑊 splice 〈𝐸, 𝐸, 〈“𝐼”〉〉) ⇒ ⊢ (𝜑 → ran 𝑈 = (ran 𝑊 ∪ {𝐼})) | ||
| Theorem | cycpmco2lem1 33083 | Lemma for cycpmco2 33090. (Contributed by Thierry Arnoux, 4-Jan-2024.) |
| ⊢ 𝑀 = (toCyc‘𝐷) & ⊢ 𝑆 = (SymGrp‘𝐷) & ⊢ (𝜑 → 𝐷 ∈ 𝑉) & ⊢ (𝜑 → 𝑊 ∈ dom 𝑀) & ⊢ (𝜑 → 𝐼 ∈ (𝐷 ∖ ran 𝑊)) & ⊢ (𝜑 → 𝐽 ∈ ran 𝑊) & ⊢ 𝐸 = ((◡𝑊‘𝐽) + 1) & ⊢ 𝑈 = (𝑊 splice 〈𝐸, 𝐸, 〈“𝐼”〉〉) ⇒ ⊢ (𝜑 → ((𝑀‘𝑊)‘((𝑀‘〈“𝐼𝐽”〉)‘𝐼)) = ((𝑀‘𝑊)‘𝐽)) | ||
| Theorem | cycpmco2lem2 33084 | Lemma for cycpmco2 33090. (Contributed by Thierry Arnoux, 4-Jan-2024.) |
| ⊢ 𝑀 = (toCyc‘𝐷) & ⊢ 𝑆 = (SymGrp‘𝐷) & ⊢ (𝜑 → 𝐷 ∈ 𝑉) & ⊢ (𝜑 → 𝑊 ∈ dom 𝑀) & ⊢ (𝜑 → 𝐼 ∈ (𝐷 ∖ ran 𝑊)) & ⊢ (𝜑 → 𝐽 ∈ ran 𝑊) & ⊢ 𝐸 = ((◡𝑊‘𝐽) + 1) & ⊢ 𝑈 = (𝑊 splice 〈𝐸, 𝐸, 〈“𝐼”〉〉) ⇒ ⊢ (𝜑 → (𝑈‘𝐸) = 𝐼) | ||
| Theorem | cycpmco2lem3 33085 | Lemma for cycpmco2 33090. (Contributed by Thierry Arnoux, 4-Jan-2024.) |
| ⊢ 𝑀 = (toCyc‘𝐷) & ⊢ 𝑆 = (SymGrp‘𝐷) & ⊢ (𝜑 → 𝐷 ∈ 𝑉) & ⊢ (𝜑 → 𝑊 ∈ dom 𝑀) & ⊢ (𝜑 → 𝐼 ∈ (𝐷 ∖ ran 𝑊)) & ⊢ (𝜑 → 𝐽 ∈ ran 𝑊) & ⊢ 𝐸 = ((◡𝑊‘𝐽) + 1) & ⊢ 𝑈 = (𝑊 splice 〈𝐸, 𝐸, 〈“𝐼”〉〉) ⇒ ⊢ (𝜑 → ((♯‘𝑈) − 1) = (♯‘𝑊)) | ||
| Theorem | cycpmco2lem4 33086 | Lemma for cycpmco2 33090. (Contributed by Thierry Arnoux, 4-Jan-2024.) |
| ⊢ 𝑀 = (toCyc‘𝐷) & ⊢ 𝑆 = (SymGrp‘𝐷) & ⊢ (𝜑 → 𝐷 ∈ 𝑉) & ⊢ (𝜑 → 𝑊 ∈ dom 𝑀) & ⊢ (𝜑 → 𝐼 ∈ (𝐷 ∖ ran 𝑊)) & ⊢ (𝜑 → 𝐽 ∈ ran 𝑊) & ⊢ 𝐸 = ((◡𝑊‘𝐽) + 1) & ⊢ 𝑈 = (𝑊 splice 〈𝐸, 𝐸, 〈“𝐼”〉〉) ⇒ ⊢ (𝜑 → ((𝑀‘𝑊)‘((𝑀‘〈“𝐼𝐽”〉)‘𝐼)) = ((𝑀‘𝑈)‘𝐼)) | ||
| Theorem | cycpmco2lem5 33087 | Lemma for cycpmco2 33090. (Contributed by Thierry Arnoux, 4-Jan-2024.) |
| ⊢ 𝑀 = (toCyc‘𝐷) & ⊢ 𝑆 = (SymGrp‘𝐷) & ⊢ (𝜑 → 𝐷 ∈ 𝑉) & ⊢ (𝜑 → 𝑊 ∈ dom 𝑀) & ⊢ (𝜑 → 𝐼 ∈ (𝐷 ∖ ran 𝑊)) & ⊢ (𝜑 → 𝐽 ∈ ran 𝑊) & ⊢ 𝐸 = ((◡𝑊‘𝐽) + 1) & ⊢ 𝑈 = (𝑊 splice 〈𝐸, 𝐸, 〈“𝐼”〉〉) & ⊢ (𝜑 → 𝐾 ∈ ran 𝑊) & ⊢ (𝜑 → (◡𝑈‘𝐾) = ((♯‘𝑈) − 1)) ⇒ ⊢ (𝜑 → ((𝑀‘𝑈)‘𝐾) = ((𝑀‘𝑊)‘𝐾)) | ||
| Theorem | cycpmco2lem6 33088 | Lemma for cycpmco2 33090. (Contributed by Thierry Arnoux, 4-Jan-2024.) |
| ⊢ 𝑀 = (toCyc‘𝐷) & ⊢ 𝑆 = (SymGrp‘𝐷) & ⊢ (𝜑 → 𝐷 ∈ 𝑉) & ⊢ (𝜑 → 𝑊 ∈ dom 𝑀) & ⊢ (𝜑 → 𝐼 ∈ (𝐷 ∖ ran 𝑊)) & ⊢ (𝜑 → 𝐽 ∈ ran 𝑊) & ⊢ 𝐸 = ((◡𝑊‘𝐽) + 1) & ⊢ 𝑈 = (𝑊 splice 〈𝐸, 𝐸, 〈“𝐼”〉〉) & ⊢ (𝜑 → 𝐾 ∈ ran 𝑊) & ⊢ (𝜑 → 𝐾 ≠ 𝐼) & ⊢ (𝜑 → (◡𝑈‘𝐾) ∈ (𝐸..^((♯‘𝑈) − 1))) ⇒ ⊢ (𝜑 → ((𝑀‘𝑈)‘𝐾) = ((𝑀‘𝑊)‘𝐾)) | ||
| Theorem | cycpmco2lem7 33089 | Lemma for cycpmco2 33090. (Contributed by Thierry Arnoux, 4-Jan-2024.) |
| ⊢ 𝑀 = (toCyc‘𝐷) & ⊢ 𝑆 = (SymGrp‘𝐷) & ⊢ (𝜑 → 𝐷 ∈ 𝑉) & ⊢ (𝜑 → 𝑊 ∈ dom 𝑀) & ⊢ (𝜑 → 𝐼 ∈ (𝐷 ∖ ran 𝑊)) & ⊢ (𝜑 → 𝐽 ∈ ran 𝑊) & ⊢ 𝐸 = ((◡𝑊‘𝐽) + 1) & ⊢ 𝑈 = (𝑊 splice 〈𝐸, 𝐸, 〈“𝐼”〉〉) & ⊢ (𝜑 → 𝐾 ∈ ran 𝑊) & ⊢ (𝜑 → 𝐾 ≠ 𝐽) & ⊢ (𝜑 → (◡𝑈‘𝐾) ∈ (0..^𝐸)) ⇒ ⊢ (𝜑 → ((𝑀‘𝑈)‘𝐾) = ((𝑀‘𝑊)‘𝐾)) | ||
| Theorem | cycpmco2 33090 | The composition of a cyclic permutation and a transposition of one element in the cycle and one outside the cycle results in a cyclic permutation with one more element in its orbit. (Contributed by Thierry Arnoux, 2-Jan-2024.) |
| ⊢ 𝑀 = (toCyc‘𝐷) & ⊢ 𝑆 = (SymGrp‘𝐷) & ⊢ (𝜑 → 𝐷 ∈ 𝑉) & ⊢ (𝜑 → 𝑊 ∈ dom 𝑀) & ⊢ (𝜑 → 𝐼 ∈ (𝐷 ∖ ran 𝑊)) & ⊢ (𝜑 → 𝐽 ∈ ran 𝑊) & ⊢ 𝐸 = ((◡𝑊‘𝐽) + 1) & ⊢ 𝑈 = (𝑊 splice 〈𝐸, 𝐸, 〈“𝐼”〉〉) ⇒ ⊢ (𝜑 → ((𝑀‘𝑊) ∘ (𝑀‘〈“𝐼𝐽”〉)) = (𝑀‘𝑈)) | ||
| Theorem | cyc2fvx 33091 | Function value of a 2-cycle outside of its orbit. (Contributed by Thierry Arnoux, 19-Sep-2023.) |
| ⊢ 𝐶 = (toCyc‘𝐷) & ⊢ 𝑆 = (SymGrp‘𝐷) & ⊢ (𝜑 → 𝐷 ∈ 𝑉) & ⊢ (𝜑 → 𝐼 ∈ 𝐷) & ⊢ (𝜑 → 𝐽 ∈ 𝐷) & ⊢ (𝜑 → 𝐾 ∈ 𝐷) & ⊢ (𝜑 → 𝐼 ≠ 𝐽) & ⊢ (𝜑 → 𝐽 ≠ 𝐾) & ⊢ (𝜑 → 𝐾 ≠ 𝐼) ⇒ ⊢ (𝜑 → ((𝐶‘〈“𝐼𝐽”〉)‘𝐾) = 𝐾) | ||
| Theorem | cycpm3cl 33092 | Closure of the 3-cycles in the permutations. (Contributed by Thierry Arnoux, 19-Sep-2023.) |
| ⊢ 𝐶 = (toCyc‘𝐷) & ⊢ 𝑆 = (SymGrp‘𝐷) & ⊢ (𝜑 → 𝐷 ∈ 𝑉) & ⊢ (𝜑 → 𝐼 ∈ 𝐷) & ⊢ (𝜑 → 𝐽 ∈ 𝐷) & ⊢ (𝜑 → 𝐾 ∈ 𝐷) & ⊢ (𝜑 → 𝐼 ≠ 𝐽) & ⊢ (𝜑 → 𝐽 ≠ 𝐾) & ⊢ (𝜑 → 𝐾 ≠ 𝐼) ⇒ ⊢ (𝜑 → (𝐶‘〈“𝐼𝐽𝐾”〉) ∈ (Base‘𝑆)) | ||
| Theorem | cycpm3cl2 33093 | Closure of the 3-cycles in the class of 3-cycles. (Contributed by Thierry Arnoux, 19-Sep-2023.) |
| ⊢ 𝐶 = (toCyc‘𝐷) & ⊢ 𝑆 = (SymGrp‘𝐷) & ⊢ (𝜑 → 𝐷 ∈ 𝑉) & ⊢ (𝜑 → 𝐼 ∈ 𝐷) & ⊢ (𝜑 → 𝐽 ∈ 𝐷) & ⊢ (𝜑 → 𝐾 ∈ 𝐷) & ⊢ (𝜑 → 𝐼 ≠ 𝐽) & ⊢ (𝜑 → 𝐽 ≠ 𝐾) & ⊢ (𝜑 → 𝐾 ≠ 𝐼) ⇒ ⊢ (𝜑 → (𝐶‘〈“𝐼𝐽𝐾”〉) ∈ (𝐶 “ (◡♯ “ {3}))) | ||
| Theorem | cyc3fv1 33094 | Function value of a 3-cycle at the first point. (Contributed by Thierry Arnoux, 19-Sep-2023.) |
| ⊢ 𝐶 = (toCyc‘𝐷) & ⊢ 𝑆 = (SymGrp‘𝐷) & ⊢ (𝜑 → 𝐷 ∈ 𝑉) & ⊢ (𝜑 → 𝐼 ∈ 𝐷) & ⊢ (𝜑 → 𝐽 ∈ 𝐷) & ⊢ (𝜑 → 𝐾 ∈ 𝐷) & ⊢ (𝜑 → 𝐼 ≠ 𝐽) & ⊢ (𝜑 → 𝐽 ≠ 𝐾) & ⊢ (𝜑 → 𝐾 ≠ 𝐼) ⇒ ⊢ (𝜑 → ((𝐶‘〈“𝐼𝐽𝐾”〉)‘𝐼) = 𝐽) | ||
| Theorem | cyc3fv2 33095 | Function value of a 3-cycle at the second point. (Contributed by Thierry Arnoux, 19-Sep-2023.) |
| ⊢ 𝐶 = (toCyc‘𝐷) & ⊢ 𝑆 = (SymGrp‘𝐷) & ⊢ (𝜑 → 𝐷 ∈ 𝑉) & ⊢ (𝜑 → 𝐼 ∈ 𝐷) & ⊢ (𝜑 → 𝐽 ∈ 𝐷) & ⊢ (𝜑 → 𝐾 ∈ 𝐷) & ⊢ (𝜑 → 𝐼 ≠ 𝐽) & ⊢ (𝜑 → 𝐽 ≠ 𝐾) & ⊢ (𝜑 → 𝐾 ≠ 𝐼) ⇒ ⊢ (𝜑 → ((𝐶‘〈“𝐼𝐽𝐾”〉)‘𝐽) = 𝐾) | ||
| Theorem | cyc3fv3 33096 | Function value of a 3-cycle at the third point. (Contributed by Thierry Arnoux, 19-Sep-2023.) |
| ⊢ 𝐶 = (toCyc‘𝐷) & ⊢ 𝑆 = (SymGrp‘𝐷) & ⊢ (𝜑 → 𝐷 ∈ 𝑉) & ⊢ (𝜑 → 𝐼 ∈ 𝐷) & ⊢ (𝜑 → 𝐽 ∈ 𝐷) & ⊢ (𝜑 → 𝐾 ∈ 𝐷) & ⊢ (𝜑 → 𝐼 ≠ 𝐽) & ⊢ (𝜑 → 𝐽 ≠ 𝐾) & ⊢ (𝜑 → 𝐾 ≠ 𝐼) ⇒ ⊢ (𝜑 → ((𝐶‘〈“𝐼𝐽𝐾”〉)‘𝐾) = 𝐼) | ||
| Theorem | cyc3co2 33097 | Represent a 3-cycle as a composition of two 2-cycles. (Contributed by Thierry Arnoux, 19-Sep-2023.) |
| ⊢ 𝐶 = (toCyc‘𝐷) & ⊢ 𝑆 = (SymGrp‘𝐷) & ⊢ (𝜑 → 𝐷 ∈ 𝑉) & ⊢ (𝜑 → 𝐼 ∈ 𝐷) & ⊢ (𝜑 → 𝐽 ∈ 𝐷) & ⊢ (𝜑 → 𝐾 ∈ 𝐷) & ⊢ (𝜑 → 𝐼 ≠ 𝐽) & ⊢ (𝜑 → 𝐽 ≠ 𝐾) & ⊢ (𝜑 → 𝐾 ≠ 𝐼) & ⊢ · = (+g‘𝑆) ⇒ ⊢ (𝜑 → (𝐶‘〈“𝐼𝐽𝐾”〉) = ((𝐶‘〈“𝐼𝐾”〉) · (𝐶‘〈“𝐼𝐽”〉))) | ||
| Theorem | cycpmconjvlem 33098 | Lemma for cycpmconjv 33099. (Contributed by Thierry Arnoux, 9-Oct-2023.) |
| ⊢ (𝜑 → 𝐹:𝐷–1-1-onto→𝐷) & ⊢ (𝜑 → 𝐵 ⊆ 𝐷) ⇒ ⊢ (𝜑 → ((𝐹 ↾ (𝐷 ∖ 𝐵)) ∘ ◡𝐹) = ( I ↾ (𝐷 ∖ ran (𝐹 ↾ 𝐵)))) | ||
| Theorem | cycpmconjv 33099 | A formula for computing conjugacy classes of cyclic permutations. Formula in property (b) of [Lang] p. 32. (Contributed by Thierry Arnoux, 9-Oct-2023.) |
| ⊢ 𝑆 = (SymGrp‘𝐷) & ⊢ 𝑀 = (toCyc‘𝐷) & ⊢ + = (+g‘𝑆) & ⊢ − = (-g‘𝑆) & ⊢ 𝐵 = (Base‘𝑆) ⇒ ⊢ ((𝐷 ∈ 𝑉 ∧ 𝐺 ∈ 𝐵 ∧ 𝑊 ∈ dom 𝑀) → ((𝐺 + (𝑀‘𝑊)) − 𝐺) = (𝑀‘(𝐺 ∘ 𝑊))) | ||
| Theorem | cycpmrn 33100 | The range of the word used to build a cycle is the cycle's orbit, i.e., the set of points it moves. (Contributed by Thierry Arnoux, 20-Nov-2023.) |
| ⊢ 𝑀 = (toCyc‘𝐷) & ⊢ (𝜑 → 𝐷 ∈ 𝑉) & ⊢ (𝜑 → 𝑊 ∈ Word 𝐷) & ⊢ (𝜑 → 𝑊:dom 𝑊–1-1→𝐷) & ⊢ (𝜑 → 1 < (♯‘𝑊)) ⇒ ⊢ (𝜑 → ran 𝑊 = dom ((𝑀‘𝑊) ∖ I )) | ||
| < Previous Next > |
| Copyright terms: Public domain | < Previous Next > |