Skip to content

Commit

Permalink
[B] Move FiniteTypes.finite_couple to Finite_sets
Browse files Browse the repository at this point in the history
This ensures that `FiniteTypes.v` contains only lemmas & theorems
concerning `FiniteT`.
Use `Finite_sets.finite_couple` instead now.
  • Loading branch information
Columbus240 committed Jun 17, 2022
1 parent bd08c83 commit a60c821
Show file tree
Hide file tree
Showing 3 changed files with 11 additions and 11 deletions.
2 changes: 1 addition & 1 deletion theories/ZornsLemma/CountableTypes.v
Original file line number Diff line number Diff line change
Expand Up @@ -2,7 +2,7 @@ From Coq Require Export Relation_Definitions QArith ZArith.
From Coq Require Import Arith ArithRing FunctionalExtensionality
Program.Subset ClassicalChoice.
From ZornsLemma Require Import InfiniteTypes CSB DecidableDec
DependentTypeChoice.
DependentTypeChoice Finite_sets.
From ZornsLemma Require Export FiniteTypes IndexedFamilies.

Local Close Scope Q_scope.
Expand Down
8 changes: 0 additions & 8 deletions theories/ZornsLemma/FiniteTypes.v
Original file line number Diff line number Diff line change
Expand Up @@ -979,11 +979,3 @@ Proof.
+ intros. destruct x as [[]|]; intuition.
+ intros. destruct y as [|]; intuition.
Qed.

Lemma finite_couple {X} (x y : X) :
Finite (Couple x y).
Proof.
rewrite <- Couple_as_union.
apply Union_preserves_Finite.
all: apply Singleton_is_finite.
Qed.
12 changes: 10 additions & 2 deletions theories/ZornsLemma/Finite_sets.v
Original file line number Diff line number Diff line change
@@ -1,6 +1,14 @@
From Coq Require Import Classical.
From Coq Require Export Finite_sets.
From ZornsLemma Require Import EnsemblesImplicit FiniteImplicit.
From Coq Require Export Finite_sets Finite_sets_facts.
From ZornsLemma Require Import EnsemblesImplicit FiniteImplicit Powerset_facts.

Lemma finite_couple {X} (x y : X) :
Finite (Couple x y).
Proof.
rewrite <- Couple_as_union.
apply Union_preserves_Finite.
all: apply Singleton_is_finite.
Qed.

(* This is like a choice property for finite sets. And [P] is about pairs, so
that's the meaning of the name. It is similar to
Expand Down

0 comments on commit a60c821

Please sign in to comment.