cardinality of sets

0.0(0)
studied byStudied by 0 people
0.0(0)
full-widthCall Kai
learnLearn
examPractice Test
spaced repetitionSpaced Repetition
heart puzzleMatch
flashcardsFlashcards
GameKnowt Play
Card Sorting

1/36

encourage image

There's no tags or description

Looks like no tags are added yet.

Study Analytics
Name
Mastery
Learn
Test
Matching
Spaced

No study sessions yet.

37 Terms

1
New cards

Define N_n.

For n\in\mathbb{N}, N_n=\{1,2,3,\ldots,n\}=\{k\in\mathbb{N}\mid 1\le k\le n\}.

2
New cards

Rigorous definition: what does it mean that a finite set A has cardinality n?

There exists a bijection f:N_n\to A. We write |A|=n and define |\varnothing|=0.

3
New cards

How can you certify |A|=n without 'counting'?

Exhibit a bijection f:Nn\to A (i.e. label elements a1,\dots,an with f(i)=ai).

4
New cards

State Lemma: If there is an injection f:Nm\to Nn, what inequality holds?

m\le n.

5
New cards

Why is the lemma f:Nm\to Nn means M\le N useful for finite cardinality?

It shows cardinality is well-defined: if A is in bijection with both Nm and Nn, then m=n.

6
New cards

State precisely: when is finite cardinality well-defined?

If there are bijections f:Nm\to A and g:Nn\to A, then m=n.

7
New cards

What does an injection f:A\to B imply for finite sets?

|A|\le |B|; and if f is a bijection then |A|=|B|.

8
New cards

State the Pigeonhole Principle in cardinality language.

For finite sets, if |A|>|B| then no function f:A\to B is injective (some two elements of A map to the same element of B).

9
New cards

Cardinality of the union of disjoint finite sets?

If A\cap B=\varnothing, then |A\cup B|=|A|+|B|.

10
New cards

Generalise the previous result to finitely many pairwise-disjoint finite sets.

If A1,\dots,An are pairwise disjoint and finite, then \bigl|\bigcup{i=1}^n Ai\bigr|=\sum{i=1}^n |Ai|.

11
New cards

State the Inclusion–Exclusion principle for two finite sets.

|A\cup B|=|A|+|B|-|A\cap B|.

12
New cards

Define: sets A,B are equipotent.

There exists a bijection between A and B (they have the same cardinality).

13
New cards

Example of equipotent infinite sets on \mathbb{R}.

The intervals (0,1) and (0,2) are equipotent via f(x)=2x.

14
New cards

Define: denumerable set and the symbol for its size.

A is denumerable if there is a bijection f:\mathbb{N}\to A. We write |A|=\aleph_0.

15
New cards

Define: countable set.

A is countable if it is finite or denumerable.

16
New cards

Equivalent characterisation: how do we \list\ a denumerable set?

A is denumerable iff we can write A=\{a1,a2,\dots\} (a bijection with \mathbb{N} given by f(i)=a_i).

17
New cards

Example: show the even positive integers \{2k\mid k\in\mathbb{N}\} are denumerable.

Bijection f:\mathbb{N}\to A with f(k)=2k.

18
New cards

Example: show the squares \{k^2\mid k\in\mathbb{N}\} are denumerable.

Bijection f:\mathbb{N}\to B with f(k)=k^2.

19
New cards

Give an explicit bijection \mathbb{N}\to\mathbb{Z} to prove \mathbb{Z} is denumerable.

f(n)=\begin{cases}n/2,&n\text{ even}\\-(n-1)/2,&n\text{ odd}\end{cases}.

20
New cards

State Dedekind's characterisation of infinite sets.

A set A is infinite iff it is equipotent to a proper subset of itself.

21
New cards

Show: the union of two countable sets is countable.

If A and B are countable, list them as a1,a2,\dots and b1,b2,\dots; interleave to list A\cup B, hence it is countable.

22
New cards

Show: the product of two countable sets is countable (diagonal argument).

Arrange (ai,bj) in a grid and traverse along diagonals to list A\times B; thus countable.

23
New cards

Generalise: finite unions and finite products of countable sets are countable.

If A1,\dots,An are countable then both \bigcup{i=1}^n Ai and \prod{i=1}^n Ai are countable.

24
New cards

State: \mathbb{Q} is denumerable (idea of proof).

Since \mathbb{Z}\times\mathbb{Z} is countable and \mathbb{Q}=\{a/b\mid a,b\in\mathbb{Z},\,b>0,\,\gcd(a,b)=1\} injects into it, \mathbb{Q} is denumerable.

25
New cards

State Cantor's theorem: \mathbb{R} is uncountable (core diagonal step).

Assume $[0,1] is listed as an=0.a{n1}a{n2}\ldots and define b=0.b1b2\ldots with bn\ne a{nn} (e.g. bn=1 if a{nn}\ne 1, else bn=2). Then b$$ is missing from the list, contradiction.

26
New cards

Compare sizes: |\mathbb{N}|,|\mathbb{Z}|,|\mathbb{Q}|,|\mathbb{R}|.

|\mathbb{N}|=|\mathbb{Z}|=|\mathbb{Q}|=\aleph_0<|\mathbb{R}|=:\mathfrak{c}.

27
New cards

What is |\mathbb{R}\times\mathbb{R}|?

|\mathbb{R}\times\mathbb{R}|=\mathfrak{c} (same cardinality as \mathbb{R}).

28
New cards

Define the power set \mathcal{P}(A).

\mathcal{P}(A)=\{B\mid B\subseteq A\}.

29
New cards

State Cantor's power-set theorem.

For every set A, |\mathcal{P}(A)|>|A|.

30
New cards

Consequence of the power-set theorem for \mathbb{R}.

|\mathcal{P}(\mathbb{R})|>|\mathbb{R}|=\mathfrak{c}, so there are infinitely many strictly larger infinities.

31
New cards

Technique tip: how to prove a set is countable in practice?

Either exhibit a bijection \mathbb{N}\to A (list it), or inject A into a known countable set, or surject \mathbb{N} onto A.

32
New cards

If |A|>|B| for finite sets and f:A\to B, what must happen? Why?

By the Pigeonhole Principle, f is not injective; some two elements of A share an image.

33
New cards

Compute |A\cup B| when |A|=7,|B|=10,|A\cap B|=4 (finite sets).

|A\cup B|=7+10-4=13.

34
New cards

Give a quick test to recognise an infinite set using Dedekind's idea.

Find an injection A\to A that misses at least one element (e.g. n\mapsto n+1 on \mathbb{N}).

35
New cards

Is a subset of a denumerable set always countable?

Yes: any subset is either finite or denumerable, hence countable.

36
New cards

Why doesn't the diagonal proof contradict that (0,1) and (0,2) are equipotent?

Both sets are uncountable of size \mathfrak{c}; a bijection like x\mapsto 2x exists between them. Diagonalisation only rules out listing them by \mathbb{N}.

37
New cards

TEST—rendering check: show this matrix as a square not a line.

\begin{pmatrix}1 & 0 & 0\\0 & 1 & 0\\0 & 0 & 1\end{pmatrix}