![]() |
Metamath Proof Explorer |
< Previous
Next >
Nearby theorems |
|
Mirrors > Home > MPE Home > Th. List > ecopover | Structured version Visualization version GIF version |
Description: Assuming that operation 𝐹 is commutative (second hypothesis), closed (third hypothesis), associative (fourth hypothesis), and has the cancellation property (fifth hypothesis), show that the relation ∼, specified by the first hypothesis, is an equivalence relation. (Contributed by NM, 16-Feb-1996.) (Revised by Mario Carneiro, 12-Aug-2015.) (Proof shortened by AV, 1-May-2021.) |
Ref | Expression |
---|---|
ecopopr.1 | ⊢ ∼ = {〈𝑥, 𝑦〉 ∣ ((𝑥 ∈ (𝑆 × 𝑆) ∧ 𝑦 ∈ (𝑆 × 𝑆)) ∧ ∃𝑧∃𝑤∃𝑣∃𝑢((𝑥 = 〈𝑧, 𝑤〉 ∧ 𝑦 = 〈𝑣, 𝑢〉) ∧ (𝑧 + 𝑢) = (𝑤 + 𝑣)))} |
ecopopr.com | ⊢ (𝑥 + 𝑦) = (𝑦 + 𝑥) |
ecopopr.cl | ⊢ ((𝑥 ∈ 𝑆 ∧ 𝑦 ∈ 𝑆) → (𝑥 + 𝑦) ∈ 𝑆) |
ecopopr.ass | ⊢ ((𝑥 + 𝑦) + 𝑧) = (𝑥 + (𝑦 + 𝑧)) |
ecopopr.can | ⊢ ((𝑥 ∈ 𝑆 ∧ 𝑦 ∈ 𝑆) → ((𝑥 + 𝑦) = (𝑥 + 𝑧) → 𝑦 = 𝑧)) |
Ref | Expression |
---|---|
ecopover | ⊢ ∼ Er (𝑆 × 𝑆) |
Step | Hyp | Ref | Expression |
---|---|---|---|
1 | ecopopr.1 | . . 3 ⊢ ∼ = {〈𝑥, 𝑦〉 ∣ ((𝑥 ∈ (𝑆 × 𝑆) ∧ 𝑦 ∈ (𝑆 × 𝑆)) ∧ ∃𝑧∃𝑤∃𝑣∃𝑢((𝑥 = 〈𝑧, 𝑤〉 ∧ 𝑦 = 〈𝑣, 𝑢〉) ∧ (𝑧 + 𝑢) = (𝑤 + 𝑣)))} | |
2 | 1 | relopabi 5540 | . 2 ⊢ Rel ∼ |
3 | ecopopr.com | . . 3 ⊢ (𝑥 + 𝑦) = (𝑦 + 𝑥) | |
4 | 1, 3 | ecopovsym 8197 | . 2 ⊢ (𝑓 ∼ 𝑔 → 𝑔 ∼ 𝑓) |
5 | ecopopr.cl | . . 3 ⊢ ((𝑥 ∈ 𝑆 ∧ 𝑦 ∈ 𝑆) → (𝑥 + 𝑦) ∈ 𝑆) | |
6 | ecopopr.ass | . . 3 ⊢ ((𝑥 + 𝑦) + 𝑧) = (𝑥 + (𝑦 + 𝑧)) | |
7 | ecopopr.can | . . 3 ⊢ ((𝑥 ∈ 𝑆 ∧ 𝑦 ∈ 𝑆) → ((𝑥 + 𝑦) = (𝑥 + 𝑧) → 𝑦 = 𝑧)) | |
8 | 1, 3, 5, 6, 7 | ecopovtrn 8198 | . 2 ⊢ ((𝑓 ∼ 𝑔 ∧ 𝑔 ∼ ℎ) → 𝑓 ∼ ℎ) |
9 | vex 3411 | . . . . . . . . 9 ⊢ 𝑔 ∈ V | |
10 | vex 3411 | . . . . . . . . 9 ⊢ ℎ ∈ V | |
11 | 9, 10, 3 | caovcom 7159 | . . . . . . . 8 ⊢ (𝑔 + ℎ) = (ℎ + 𝑔) |
12 | 1 | ecopoveq 8196 | . . . . . . . 8 ⊢ (((𝑔 ∈ 𝑆 ∧ ℎ ∈ 𝑆) ∧ (𝑔 ∈ 𝑆 ∧ ℎ ∈ 𝑆)) → (〈𝑔, ℎ〉 ∼ 〈𝑔, ℎ〉 ↔ (𝑔 + ℎ) = (ℎ + 𝑔))) |
13 | 11, 12 | mpbiri 250 | . . . . . . 7 ⊢ (((𝑔 ∈ 𝑆 ∧ ℎ ∈ 𝑆) ∧ (𝑔 ∈ 𝑆 ∧ ℎ ∈ 𝑆)) → 〈𝑔, ℎ〉 ∼ 〈𝑔, ℎ〉) |
14 | 13 | anidms 559 | . . . . . 6 ⊢ ((𝑔 ∈ 𝑆 ∧ ℎ ∈ 𝑆) → 〈𝑔, ℎ〉 ∼ 〈𝑔, ℎ〉) |
15 | 14 | rgen2a 3169 | . . . . 5 ⊢ ∀𝑔 ∈ 𝑆 ∀ℎ ∈ 𝑆 〈𝑔, ℎ〉 ∼ 〈𝑔, ℎ〉 |
16 | breq12 4930 | . . . . . . 7 ⊢ ((𝑓 = 〈𝑔, ℎ〉 ∧ 𝑓 = 〈𝑔, ℎ〉) → (𝑓 ∼ 𝑓 ↔ 〈𝑔, ℎ〉 ∼ 〈𝑔, ℎ〉)) | |
17 | 16 | anidms 559 | . . . . . 6 ⊢ (𝑓 = 〈𝑔, ℎ〉 → (𝑓 ∼ 𝑓 ↔ 〈𝑔, ℎ〉 ∼ 〈𝑔, ℎ〉)) |
18 | 17 | ralxp 5558 | . . . . 5 ⊢ (∀𝑓 ∈ (𝑆 × 𝑆)𝑓 ∼ 𝑓 ↔ ∀𝑔 ∈ 𝑆 ∀ℎ ∈ 𝑆 〈𝑔, ℎ〉 ∼ 〈𝑔, ℎ〉) |
19 | 15, 18 | mpbir 223 | . . . 4 ⊢ ∀𝑓 ∈ (𝑆 × 𝑆)𝑓 ∼ 𝑓 |
20 | 19 | rspec 3150 | . . 3 ⊢ (𝑓 ∈ (𝑆 × 𝑆) → 𝑓 ∼ 𝑓) |
21 | opabssxp 5489 | . . . . . 6 ⊢ {〈𝑥, 𝑦〉 ∣ ((𝑥 ∈ (𝑆 × 𝑆) ∧ 𝑦 ∈ (𝑆 × 𝑆)) ∧ ∃𝑧∃𝑤∃𝑣∃𝑢((𝑥 = 〈𝑧, 𝑤〉 ∧ 𝑦 = 〈𝑣, 𝑢〉) ∧ (𝑧 + 𝑢) = (𝑤 + 𝑣)))} ⊆ ((𝑆 × 𝑆) × (𝑆 × 𝑆)) | |
22 | 1, 21 | eqsstri 3884 | . . . . 5 ⊢ ∼ ⊆ ((𝑆 × 𝑆) × (𝑆 × 𝑆)) |
23 | 22 | ssbri 4970 | . . . 4 ⊢ (𝑓 ∼ 𝑓 → 𝑓((𝑆 × 𝑆) × (𝑆 × 𝑆))𝑓) |
24 | brxp 5449 | . . . . 5 ⊢ (𝑓((𝑆 × 𝑆) × (𝑆 × 𝑆))𝑓 ↔ (𝑓 ∈ (𝑆 × 𝑆) ∧ 𝑓 ∈ (𝑆 × 𝑆))) | |
25 | 24 | simplbi 490 | . . . 4 ⊢ (𝑓((𝑆 × 𝑆) × (𝑆 × 𝑆))𝑓 → 𝑓 ∈ (𝑆 × 𝑆)) |
26 | 23, 25 | syl 17 | . . 3 ⊢ (𝑓 ∼ 𝑓 → 𝑓 ∈ (𝑆 × 𝑆)) |
27 | 20, 26 | impbii 201 | . 2 ⊢ (𝑓 ∈ (𝑆 × 𝑆) ↔ 𝑓 ∼ 𝑓) |
28 | 2, 4, 8, 27 | iseri 8114 | 1 ⊢ ∼ Er (𝑆 × 𝑆) |
Colors of variables: wff setvar class |
Syntax hints: → wi 4 ↔ wb 198 ∧ wa 387 = wceq 1508 ∃wex 1743 ∈ wcel 2051 ∀wral 3081 〈cop 4441 class class class wbr 4925 {copab 4987 × cxp 5401 (class class class)co 6974 Er wer 8084 |
This theorem was proved from axioms: ax-mp 5 ax-1 6 ax-2 7 ax-3 8 ax-gen 1759 ax-4 1773 ax-5 1870 ax-6 1929 ax-7 1966 ax-8 2053 ax-9 2060 ax-10 2080 ax-11 2094 ax-12 2107 ax-13 2302 ax-ext 2743 ax-sep 5056 ax-nul 5063 ax-pr 5182 |
This theorem depends on definitions: df-bi 199 df-an 388 df-or 835 df-3an 1071 df-tru 1511 df-ex 1744 df-nf 1748 df-sb 2017 df-mo 2548 df-eu 2585 df-clab 2752 df-cleq 2764 df-clel 2839 df-nfc 2911 df-ral 3086 df-rex 3087 df-rab 3090 df-v 3410 df-sbc 3675 df-csb 3780 df-dif 3825 df-un 3827 df-in 3829 df-ss 3836 df-nul 4173 df-if 4345 df-sn 4436 df-pr 4438 df-op 4442 df-uni 4709 df-iun 4790 df-br 4926 df-opab 4988 df-xp 5409 df-rel 5410 df-cnv 5411 df-co 5412 df-dm 5413 df-iota 6149 df-fv 6193 df-ov 6977 df-er 8087 |
This theorem is referenced by: enqer 10139 enrer 10281 |
Copyright terms: Public domain | W3C validator |