Skip to content
Snippets Groups Projects
Commit 658dbe78 authored by François Clément's avatar François Clément
Browse files

Mv lemma earlier to be able to compile Set_dec earlier.

parent 8491ab46
No related branches found
No related tags found
No related merge requests found
......@@ -16,6 +16,7 @@ COPYING file for more details.
(** Basic operations on sets (definitions). *)
From Coq Require Import Classical_Pred_Type.
From Coq Require Import PropExtensionality FunctionalExtensionality.
......@@ -177,6 +178,14 @@ intros HA; induction HA as [x Hx]; exists x; easy.
intros [x Hx]; eapply ne, Hx.
Qed.
Lemma nonempty_equiv_alt :
forall (A : set U), nonempty A <-> ~ empty A.
Proof.
intros A; split; intros HA.
induction HA as [x Hx]; intros H; apply (H x); easy.
destruct (not_all_not_ex _ _ HA) as [x Hx]; eapply ne, Hx.
Qed.
(** Extensionality of sets. *)
Lemma set_ext : forall (A B : set U), same A B -> A = B.
......
0% Loading or .
You are about to add 0 people to the discussion. Proceed with caution.
Finish editing this message first!
Please register or to comment