Skip to content

Commit

Permalink
closed_bigcup (#991)
Browse files Browse the repository at this point in the history
  • Loading branch information
affeldt-aist authored Jul 31, 2023
1 parent 84fcbd6 commit 902670c
Show file tree
Hide file tree
Showing 2 changed files with 12 additions and 0 deletions.
3 changes: 3 additions & 0 deletions CHANGELOG_UNRELEASED.md
Original file line number Diff line number Diff line change
Expand Up @@ -93,6 +93,9 @@
- in `classical_sets.v`:
+ lemma `bigcup_bigcup`

- in `topology.v`:
+ lemma `closed_bigcup`

### Changed

- moved from `lebesgue_measure.v` to `real_interval.v`:
Expand Down
9 changes: 9 additions & 0 deletions theories/topology.v
Original file line number Diff line number Diff line change
Expand Up @@ -2761,6 +2761,15 @@ move=> scF; rewrite big_seq.
by elim/big_ind : _ => //; [exact: closed0|exact: closedU].
Qed.

Lemma closed_bigcup (T : topologicalType) (I : choiceType) (A : set I)
(F : I -> set T) :
finite_set A -> (forall i, A i -> closed (F i)) ->
closed (\bigcup_(i in A) F i).
Proof.
move=> finA cF; rewrite -bigsetU_fset_set//; apply: closed_bigsetU => i.
by rewrite in_fset_set// inE; exact: cF.
Qed.

Section closure_lemmas.
Variable T : topologicalType.
Implicit Types E A B U : set T.
Expand Down

0 comments on commit 902670c

Please sign in to comment.