Content deleted Content added
→When A is countably infinite: Added "Indeed," to the beginning of a sentence so that the sentence does not start with a mathematical symbol, as is often accepted as bad style. I think this does not change the meaning of the sentence |
|||
(37 intermediate revisions by 18 users not shown) | |||
Line 4:
{{SpecialChars}}
In mathematical [[set theory]], '''Cantor's theorem''' is a fundamental result which states that, for any [[Set (mathematics)|set]] <math>A</math>, the set of all [[subset]]s of <math>A,</math> known as the [[power set]] of <math>A,</math> has a strictly greater [[cardinality]] than <math>A</math> itself.
For [[finite set]]s, Cantor's theorem can be seen to be true by simple [[enumeration]] of the number of subsets. Counting the [[empty set]] as a subset, a set with <math>n</math> elements has a total of <math>2^n</math> subsets, and the theorem holds because <math>2^n > n</math> for all [[non-negative integers]].
Line 10:
Much more significant is Cantor's discovery of an argument that is applicable to any set, and shows that the theorem holds for [[infinite set|infinite]] sets also. As a consequence, the cardinality of the [[real number]]s, which is the same as that of the power set of the [[integer]]s, is strictly larger than the cardinality of the integers; see [[Cardinality of the continuum]] for details.
The theorem is named for
==Proof==
Line 16:
{{math theorem|name=Theorem (Cantor)|math_statement=Let <math>f</math> be a map from set <math>A</math> to its power set <math>\mathcal{P}(A)</math>. Then <math>f : A \to \mathcal{P}(A)</math> is not [[surjective]]. As a consequence, <math>\operatorname{card}(A) < \operatorname{card}(\mathcal{P}(A))</math> holds for any set <math>A</math>.}}
{{math proof|
By definition of cardinality, we have <math>\operatorname{card}(X) < \operatorname{card}(Y)</math> for any two sets <math>X</math> and <math>Y</math> if and only if there is an [[injective function]] but no [[Bijective Function|bijective function]] from <math>X</math>
:<math>B=\{x\in A \mid x\not\in f(x)\}.</math>
This means, by definition, that for all
Equivalently, and slightly more formally, we have just proved that the existence of
▲Equivalently, and slightly more formally, we just proved that the existence of ξ ∈ ''A'' such that ''f''(ξ) = ''B'' implies the following [[contradiction]]:
:<math>\begin{aligned}
\xi\
\xi \in B &\iff \xi \in f(\xi) && \text{(by assumption that }f(\xi)=B\text{)}
\end{aligned}</math>
Therefore, by [[reductio ad absurdum]], the assumption must be false.<ref name="Priest2002"/> Thus there is no
Finally, to complete the proof, we need to exhibit an injective function from
Another way to think of the proof is that
Because of the double occurrence of <math>x</math> in the expression "<math>x\in f(x)</math>", this is a [[Cantor's diagonal argument|diagonal argument]]. For a countable (or finite) set, the argument of the proof given above can be illustrated by constructing a table in which
Because of the double occurrence of ''x'' in the expression "''x'' ∉ ''f''(''x'')", this is a [[Cantor's diagonal argument|diagonal argument]]. For a countable (or finite) set, the argument of the proof given above can be illustrated by constructing a table in which each row is labelled by a unique ''x'' from ''A'' = {''x''<sub>1</sub>, ''x''<sub>2</sub>, ...}, in this order. ''A'' is assumed to admit a [[Total order|linear order]] so that such table can be constructed. Each column of the table is labelled by a unique ''y'' from the [[power set]] of ''A''; the columns are ordered by the argument to ''f'', i.e. the column labels are ''f''(''x''<sub>1</sub>), ''f''(''x''<sub>2</sub>), ..., in this order. The intersection of each row ''x'' and column ''y'' records a true/false bit whether ''x'' ∈ ''y''. Given the order chosen for the row and column labels, the main diagonal ''D'' of this table thus records whether ''x'' ∈ ''f''(''x'') for each ''x'' ∈ ''A''. The set ''B'' constructed in the previous paragraphs coincides with the row labels for the subset of entries on this main diagonal ''D'' where the table records that ''x'' ∈ ''f''(''x'') is false.<ref name="Priest2002">{{cite book|author=Graham Priest|title=Beyond the Limits of Thought|year=2002|publisher=Oxford University Press|isbn=978-0-19-925405-7|pages=118–119}}<!--note that the page numbers differ between the OUP and CUP editions of Priest's book!--></ref> Each column records the values of the [[indicator function]] of the set corresponding to the column. The indicator function of ''B'' coincides with the [[logical negation|logically negated]] (swap "true" and "false") entries of the main diagonal. Thus the indicator function of ''B'' does not agree with any column in at least one entry. Consequently, no column represents ''B''.▼
# each row is labelled by a unique <math>x</math> from <math>A=\{x_1 ,x_2 , \ldots \}</math>, in this order. <math>A</math> is assumed to admit a [[Total order|linear order]] so that such table can be constructed.
# each column of the table is labelled by a unique <math>y</math> from the [[power set]] of <math>A</math>; the columns are ordered by the argument to <math>f</math>, i.e. the column labels are <math>f(x_1),f(x_2)</math>, ..., in this order.
# the intersection of each row <math>x</math> and column <math>y</math> records a true/false bit whether <math>x\in y</math>.
Given the order chosen for the row and column labels, the main diagonal <math>D</math> of this table thus records whether <math>x\in f(x)</math> for each <math>x\in A</math>. One such table will be the following:
<math display="block">\begin{array}{cccccc}
& f(x_1) & f(x_2) & f(x_3) & f(x_4) & \cdots \\
\hline
x_1 & {\color{red} T} & T & F & T & \cdots \\
x_2 & T & {\color{red} F} & F & F & \cdots \\
x_3 & F & F & {\color{red} T} & T & \cdots \\
x_4 & F & T & T & {\color{red} T} & \cdots \\
\vdots & \vdots & \vdots & \vdots & \vdots & \ddots
\end{array}</math>
▲
Despite the simplicity of the above proof, it is rather difficult for an [[automated theorem prover]] to produce it. The main difficulty lies in an automated discovery of the Cantor diagonal set. [[Lawrence Paulson]] noted in 1992 that [[Otter (theorem prover)|Otter]] could not do it, whereas [[Isabelle (proof assistant)|Isabelle]] could, albeit with a certain amount of direction in terms of tactics that might perhaps be considered cheating.<ref name="Paulson1992"/>
==When ''A'' is countably infinite==
Let us examine the proof for the specific case when <math>A</math> is [[countably infinite]]. [[Without loss of generality]], we may take
Suppose that
:<math>\mathcal{P}(\mathbb{N})=\{\varnothing,\{1, 2\}, \{1, 2, 3\}, \{4\}, \{1, 5\}, \{3, 4, 6\}, \{2, 4, 6,\dots\},\dots\}.</math>
Now that we have an idea of what the elements of
:<math>\mathbb{N}\begin{Bmatrix} 1 & \longleftrightarrow & \{4, 5\}\\ 2 & \longleftrightarrow & \{1, 2, 3\} \\ 3 & \longleftrightarrow & \{4, 5, 6\} \\ 4 & \longleftrightarrow & \{1, 3, 5\} \\ \vdots & \vdots & \vdots \end{Bmatrix}\mathcal{P}(\mathbb{N}).</math>
Line 56 ⟶ 71:
Given such a pairing, some natural numbers are paired with [[subset]]s that contain the very same number. For instance, in our example the number 2 is paired with the subset {1, 2, 3}, which contains 2 as a member. Let us call such numbers ''selfish''. Other natural numbers are paired with [[subset]]s that do not contain them. For instance, in our example the number 1 is paired with the subset {4, 5}, which does not contain the number 1. Call these numbers ''non-selfish''. Likewise, 3 and 4 are non-selfish.
Using this idea, let us build a special set of natural numbers. This set will provide the [[proof by contradiction|contradiction]] we seek. Let
Since there is no natural number which can be paired with
Note that the set
Through this [[proof by contradiction]] we have proven that the [[cardinality]] of
==Related paradoxes==
Line 85 ⟶ 100:
==History==
Cantor gave essentially this proof in a paper published in 1891 "Über eine elementare Frage der Mannigfaltigkeitslehre",<ref>{{Citation|language=de|first=Georg|last=Cantor|url=http://gdz.sub.uni-goettingen.de/dms/load/img/?PID=GDZPPN002113910&physid=PHYS_0084 <!--http://resolver.sub.uni-goettingen.de/purl?GDZPPN002113910-->|title=Über eine elementare Frage der Mannigfaltigskeitslehre|journal=Jahresbericht der Deutschen Mathematiker-Vereinigung|volume=1|year=1891|pages=75–78}}, also in ''Georg Cantor, Gesammelte Abhandlungen mathematischen und philosophischen Inhalts'', E. Zermelo, 1932.</ref> where the [[Cantor's diagonal argument|diagonal argument]] for the uncountability of the [[real number|reals]] also first appears (he had [[Cantor's first uncountability proof|earlier proved the uncountability of the reals by other methods]]). The version of this argument he gave in that paper was phrased in terms of indicator functions on a set rather than subsets of a set.<ref>A. Kanamori, "[https://math.bu.edu/people/aki/8.pdf The Empty Set, the Singleton, and the Ordered Pair]", p.276. Bulletin of Symbolic Logic vol. 9, no. 3, (2003). Accessed 21 August 2023.</ref> He showed that if ''f'' is a function defined on ''X'' whose values are 2-valued functions on ''X'', then the 2-valued function ''G''(''x'') = 1 − ''f''(''x'')(''x'') is not in the range of ''f''.
[[Bertrand Russell]] has a very similar proof in ''[[Principles of Mathematics]]'' (1903, section 348), where he shows that there are more [[propositional function]]s than objects. "For suppose a correlation of all objects and some propositional functions to have been affected, and let phi-''x'' be the correlate of ''x''. Then "not-phi-''x''(''x'')," i.e. "phi-''x'' does not hold of ''x''" is a propositional function not contained in this correlation; for it is true or false of ''x'' according as phi-''x'' is false or true of ''x'', and therefore it differs from phi-''x'' for every value of ''x''." He attributes the idea behind the proof to Cantor.
Line 92 ⟶ 107:
==Generalizations==
==See also==
|