Download as pdf or txt
Download as pdf or txt
You are on page 1of 2

Simple topology results

Anon K
December 2020

1 Functions
Lemma 1.1. If A and B are subsets of X and f a function from X to Y , then

1. f (A − B) ⊃ f (A) − f (B)
2. If {Aα } is a collection of subsets of X, then f (∩α Aα ) ⊂ ∩α Aα .
3. If {Aα } is a collection of subsets of X, then f (∪α Aα ) = ∪α f (Aα ).
Proof. 1. If y ∈ f (A) − f (B), then ∃x ∈ A and x ∈
/ B such that f (x) = y. That is y ∈ f (A − B).
The inclusion can be proper: consider the function f : {1, 2} → {5} defined as f (x) = 5. Then
{5} = f ({1} − {2}) 6= f ({1}) − f ({2}) = ∅.
2. If y ∈ f (∩α Aα ), ∃x ∈ ∩α Aα such that y = f (x). That is y ∈ Aα ∀α.
The inclusion can be proper: consider the function f : {1, 2} → {5} defined as f (x) = 5. Then
∅ = f ({1} ∩ {2}) 6= f ({1}) ∩ f ({2}) = {5}.

3. If y ∈ f (∪α Aα ), ∃x ∈ Aα0 for some α0 such that y = f (x). Therefore y ∈ ∪α Aα . Conversely, if


y ∈ ∪α f (Aα ), y ∈ f (Aα0 ) =⇒ ∃x ∈ Aα0 for some α0 such that y = f (x). Therefore y ∈ f (∪α Aα ).

Lemma 1.2. If A and B are subsets of X and f a function from X to Y , then

1. f −1 (A ∪ B) = f −1 (A) ∪ f −1 (B)
2. f −1 (A ∩ B) = f −1 (A) ∩ f −1 (B)
3. f −1 (A − B) = f −1 (A) − f −1 (B)
Proof. Note that the statements 1 and 2 can be generalized for arbitrary unions and intersections.

1. x ∈ f −1 (A ∪ B) =⇒ f (x) ∈ A ∪ B =⇒ f (x) ∈ A or f (x) ∈ B. So, x ∈ f −1 (A) ∪ f −1 (B).


Suppose x ∈ f −1 (A) ∪ f −1 (B), then x ∈ f −1 (A) or x ∈ f −1 (B) =⇒ f (x) ∈ A textorf (x) ∈ B.
Therefore x ∈ f −1 (A ∪ B).
2. x ∈ f −1 (A ∩ B) =⇒ f (x) ∈ A ∩ B =⇒ f (x) ∈ A and f (x) ∈ B. So, x ∈ f −1 (A) ∩ f −1 (B).
Suppose x ∈ f −1 (A) ∩ f −1 (B), then x ∈ f −1 (A) and x ∈ f −1 (B) =⇒ f (x) ∈ A textandf (x) ∈ B.
Therefore x ∈ f −1 (A ∩ B).
3. x ∈ f −1 (A − B) =⇒ f (x) ∈ A − B =⇒ f (x) ∈ A and f (x) ∈
/ B, therefore x ∈ f −1 (A) − f −1 (B).
−1 −1
If x ∈ f (A) − f (B) =⇒ f (x) ∈ A and f (x) ∈/ B. This means f (x) ∈ A − B.

Lemma 1.3. If p : X → Y is a closed map and U is an open set in X containing p−1 (y), then there exist
W open set in Y containing y such that p−1 (y) ⊂ p−1 (W ) ⊂ U

1
Proof. p−1 (W ) ⊂ U ⇐⇒ [p(x) ∈ W =⇒ x ∈ U ] ⇐⇒ [x ∈ / U =⇒ p(x) ∈ / W ] ⇐⇒ [x ∈ (X − U ) =⇒
p(x) ∈ (Y − W )] ⇐⇒ p(X − U ) ⊂ (Y − W ). That is p(X − U ) ∩ W = ∅
If y ∈ Y and p−1 (y) ∈ U , since U is open (X − U ) is closed. Therefore p(X − U ) is closed and does not
contain y. Hence there is a neighbourhood W of y which does not intersect (X − U ). From the previous
paragraph, p−1 (W ) ⊂ U .

You might also like