| Metamath Proof Explorer |
< Previous
Next >
Nearby theorems |
||
| Mirrors > Home > MPE Home > Th. List > sbth | Structured version Visualization version GIF version | ||
| Description: Schroeder-Bernstein
Theorem. Theorem 18 of [Suppes] p. 95. This
theorem states that if set 𝐴 is smaller (has lower cardinality)
than
𝐵 and vice-versa, then 𝐴 and
𝐵
are equinumerous (have the
same cardinality). The interesting thing is that this can be proved
without invoking the Axiom of Choice, as we do here. The theorem can
also be proved from the axiom of choice and the linear order of the
cardinal numbers, but our development does not provide the linear order
of cardinal numbers until much later and in ways that depend on
Schroeder-Bernstein.
The main proof consists of lemmas sbthlem1 9105 through sbthlem10 9114; this final piece mainly changes bound variables to eliminate the hypotheses of sbthlem10 9114. We follow closely the proof in Suppes, which you should consult to understand our proof at a higher level. Note that Suppes' proof, which is credited to J. M. Whitaker, does not require the Axiom of Infinity. In the Intuitionistic Logic Explorer (ILE) the Schroeder-Bernstein Theorem has been proven equivalent to the law of the excluded middle (LEM), and in ILE the LEM is not accepted as necessarily true; see https://us.metamath.org/ileuni/exmidsbth.html 9114. This is Metamath 100 proof #25. (Contributed by NM, 8-Jun-1998.) |
| Ref | Expression |
|---|---|
| sbth | ⊢ ((𝐴 ≼ 𝐵 ∧ 𝐵 ≼ 𝐴) → 𝐴 ≈ 𝐵) |
| Step | Hyp | Ref | Expression |
|---|---|---|---|
| 1 | reldom 8973 | . . . 4 ⊢ Rel ≼ | |
| 2 | 1 | brrelex1i 5721 | . . 3 ⊢ (𝐴 ≼ 𝐵 → 𝐴 ∈ V) |
| 3 | 1 | brrelex1i 5721 | . . 3 ⊢ (𝐵 ≼ 𝐴 → 𝐵 ∈ V) |
| 4 | breq1 5126 | . . . . . 6 ⊢ (𝑧 = 𝐴 → (𝑧 ≼ 𝑤 ↔ 𝐴 ≼ 𝑤)) | |
| 5 | breq2 5127 | . . . . . 6 ⊢ (𝑧 = 𝐴 → (𝑤 ≼ 𝑧 ↔ 𝑤 ≼ 𝐴)) | |
| 6 | 4, 5 | anbi12d 632 | . . . . 5 ⊢ (𝑧 = 𝐴 → ((𝑧 ≼ 𝑤 ∧ 𝑤 ≼ 𝑧) ↔ (𝐴 ≼ 𝑤 ∧ 𝑤 ≼ 𝐴))) |
| 7 | breq1 5126 | . . . . 5 ⊢ (𝑧 = 𝐴 → (𝑧 ≈ 𝑤 ↔ 𝐴 ≈ 𝑤)) | |
| 8 | 6, 7 | imbi12d 344 | . . . 4 ⊢ (𝑧 = 𝐴 → (((𝑧 ≼ 𝑤 ∧ 𝑤 ≼ 𝑧) → 𝑧 ≈ 𝑤) ↔ ((𝐴 ≼ 𝑤 ∧ 𝑤 ≼ 𝐴) → 𝐴 ≈ 𝑤))) |
| 9 | breq2 5127 | . . . . . 6 ⊢ (𝑤 = 𝐵 → (𝐴 ≼ 𝑤 ↔ 𝐴 ≼ 𝐵)) | |
| 10 | breq1 5126 | . . . . . 6 ⊢ (𝑤 = 𝐵 → (𝑤 ≼ 𝐴 ↔ 𝐵 ≼ 𝐴)) | |
| 11 | 9, 10 | anbi12d 632 | . . . . 5 ⊢ (𝑤 = 𝐵 → ((𝐴 ≼ 𝑤 ∧ 𝑤 ≼ 𝐴) ↔ (𝐴 ≼ 𝐵 ∧ 𝐵 ≼ 𝐴))) |
| 12 | breq2 5127 | . . . . 5 ⊢ (𝑤 = 𝐵 → (𝐴 ≈ 𝑤 ↔ 𝐴 ≈ 𝐵)) | |
| 13 | 11, 12 | imbi12d 344 | . . . 4 ⊢ (𝑤 = 𝐵 → (((𝐴 ≼ 𝑤 ∧ 𝑤 ≼ 𝐴) → 𝐴 ≈ 𝑤) ↔ ((𝐴 ≼ 𝐵 ∧ 𝐵 ≼ 𝐴) → 𝐴 ≈ 𝐵))) |
| 14 | vex 3467 | . . . . 5 ⊢ 𝑧 ∈ V | |
| 15 | sseq1 3989 | . . . . . . 7 ⊢ (𝑦 = 𝑥 → (𝑦 ⊆ 𝑧 ↔ 𝑥 ⊆ 𝑧)) | |
| 16 | imaeq2 6054 | . . . . . . . . . 10 ⊢ (𝑦 = 𝑥 → (𝑓 “ 𝑦) = (𝑓 “ 𝑥)) | |
| 17 | 16 | difeq2d 4106 | . . . . . . . . 9 ⊢ (𝑦 = 𝑥 → (𝑤 ∖ (𝑓 “ 𝑦)) = (𝑤 ∖ (𝑓 “ 𝑥))) |
| 18 | 17 | imaeq2d 6058 | . . . . . . . 8 ⊢ (𝑦 = 𝑥 → (𝑔 “ (𝑤 ∖ (𝑓 “ 𝑦))) = (𝑔 “ (𝑤 ∖ (𝑓 “ 𝑥)))) |
| 19 | difeq2 4100 | . . . . . . . 8 ⊢ (𝑦 = 𝑥 → (𝑧 ∖ 𝑦) = (𝑧 ∖ 𝑥)) | |
| 20 | 18, 19 | sseq12d 3997 | . . . . . . 7 ⊢ (𝑦 = 𝑥 → ((𝑔 “ (𝑤 ∖ (𝑓 “ 𝑦))) ⊆ (𝑧 ∖ 𝑦) ↔ (𝑔 “ (𝑤 ∖ (𝑓 “ 𝑥))) ⊆ (𝑧 ∖ 𝑥))) |
| 21 | 15, 20 | anbi12d 632 | . . . . . 6 ⊢ (𝑦 = 𝑥 → ((𝑦 ⊆ 𝑧 ∧ (𝑔 “ (𝑤 ∖ (𝑓 “ 𝑦))) ⊆ (𝑧 ∖ 𝑦)) ↔ (𝑥 ⊆ 𝑧 ∧ (𝑔 “ (𝑤 ∖ (𝑓 “ 𝑥))) ⊆ (𝑧 ∖ 𝑥)))) |
| 22 | 21 | cbvabv 2804 | . . . . 5 ⊢ {𝑦 ∣ (𝑦 ⊆ 𝑧 ∧ (𝑔 “ (𝑤 ∖ (𝑓 “ 𝑦))) ⊆ (𝑧 ∖ 𝑦))} = {𝑥 ∣ (𝑥 ⊆ 𝑧 ∧ (𝑔 “ (𝑤 ∖ (𝑓 “ 𝑥))) ⊆ (𝑧 ∖ 𝑥))} |
| 23 | eqid 2734 | . . . . 5 ⊢ ((𝑓 ↾ ∪ {𝑦 ∣ (𝑦 ⊆ 𝑧 ∧ (𝑔 “ (𝑤 ∖ (𝑓 “ 𝑦))) ⊆ (𝑧 ∖ 𝑦))}) ∪ (◡𝑔 ↾ (𝑧 ∖ ∪ {𝑦 ∣ (𝑦 ⊆ 𝑧 ∧ (𝑔 “ (𝑤 ∖ (𝑓 “ 𝑦))) ⊆ (𝑧 ∖ 𝑦))}))) = ((𝑓 ↾ ∪ {𝑦 ∣ (𝑦 ⊆ 𝑧 ∧ (𝑔 “ (𝑤 ∖ (𝑓 “ 𝑦))) ⊆ (𝑧 ∖ 𝑦))}) ∪ (◡𝑔 ↾ (𝑧 ∖ ∪ {𝑦 ∣ (𝑦 ⊆ 𝑧 ∧ (𝑔 “ (𝑤 ∖ (𝑓 “ 𝑦))) ⊆ (𝑧 ∖ 𝑦))}))) | |
| 24 | vex 3467 | . . . . 5 ⊢ 𝑤 ∈ V | |
| 25 | 14, 22, 23, 24 | sbthlem10 9114 | . . . 4 ⊢ ((𝑧 ≼ 𝑤 ∧ 𝑤 ≼ 𝑧) → 𝑧 ≈ 𝑤) |
| 26 | 8, 13, 25 | vtocl2g 3557 | . . 3 ⊢ ((𝐴 ∈ V ∧ 𝐵 ∈ V) → ((𝐴 ≼ 𝐵 ∧ 𝐵 ≼ 𝐴) → 𝐴 ≈ 𝐵)) |
| 27 | 2, 3, 26 | syl2an 596 | . 2 ⊢ ((𝐴 ≼ 𝐵 ∧ 𝐵 ≼ 𝐴) → ((𝐴 ≼ 𝐵 ∧ 𝐵 ≼ 𝐴) → 𝐴 ≈ 𝐵)) |
| 28 | 27 | pm2.43i 52 | 1 ⊢ ((𝐴 ≼ 𝐵 ∧ 𝐵 ≼ 𝐴) → 𝐴 ≈ 𝐵) |
| Colors of variables: wff setvar class |
| Syntax hints: → wi 4 ∧ wa 395 = wceq 1539 ∈ wcel 2107 {cab 2712 Vcvv 3463 ∖ cdif 3928 ∪ cun 3929 ⊆ wss 3931 ∪ cuni 4887 class class class wbr 5123 ◡ccnv 5664 ↾ cres 5667 “ cima 5668 ≈ cen 8964 ≼ cdom 8965 |
| This theorem was proved from axioms: ax-mp 5 ax-1 6 ax-2 7 ax-3 8 ax-gen 1794 ax-4 1808 ax-5 1909 ax-6 1966 ax-7 2006 ax-8 2109 ax-9 2117 ax-10 2140 ax-12 2176 ax-ext 2706 ax-sep 5276 ax-nul 5286 ax-pow 5345 ax-pr 5412 ax-un 7737 |
| This theorem depends on definitions: df-bi 207 df-an 396 df-or 848 df-3an 1088 df-tru 1542 df-fal 1552 df-ex 1779 df-nf 1783 df-sb 2064 df-mo 2538 df-eu 2567 df-clab 2713 df-cleq 2726 df-clel 2808 df-ral 3051 df-rex 3060 df-rab 3420 df-v 3465 df-dif 3934 df-un 3936 df-in 3938 df-ss 3948 df-nul 4314 df-if 4506 df-pw 4582 df-sn 4607 df-pr 4609 df-op 4613 df-uni 4888 df-br 5124 df-opab 5186 df-id 5558 df-xp 5671 df-rel 5672 df-cnv 5673 df-co 5674 df-dm 5675 df-rn 5676 df-res 5677 df-ima 5678 df-fun 6543 df-fn 6544 df-f 6545 df-f1 6546 df-fo 6547 df-f1o 6548 df-en 8968 df-dom 8969 |
| This theorem is referenced by: sbthb 9116 sdomnsym 9120 domtriord 9145 xpen 9162 limenpsi 9174 phpOLD 9241 onomeneqOLD 9248 unbnn 9314 infxpenlem 10035 fseqen 10049 infpwfien 10084 inffien 10085 alephdom 10103 mappwen 10134 infdjuabs 10227 infunabs 10228 infdju 10229 infdif 10230 infxpabs 10233 infmap2 10239 gchaleph 10693 gchhar 10701 inttsk 10796 inar1 10797 znnen 16231 qnnen 16232 rpnnen 16246 rexpen 16247 mreexfidimd 17665 acsinfdimd 18573 fislw 19612 opnreen 24790 ovolctb2 25464 vitali 25585 aannenlem3 26309 basellem4 27064 lgsqrlem4 27330 upgrex 29038 iccioo01 37303 ctbssinf 37382 phpreu 37586 poimirlem26 37628 pellexlem4 42821 pellexlem5 42822 idomsubgmo 43183 |
| Copyright terms: Public domain | W3C validator |