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

Add inhabited_prod.

parent b30e378c
No related branches found
No related tags found
No related merge requests found
......@@ -1633,6 +1633,12 @@ Section Prod_Facts.
Context {U1 U2 : Type}. (* Universes. *)
Lemma inhabited_prod :
inhabited U1 -> inhabited U2 -> inhabited (U1 * U2).
Proof.
intros [x1] [x2]; apply (inhabits (x1, x2)).
Qed.
Lemma prod_emptyset_l :
forall A2, prod emptyset A2 = @emptyset (U1 * U2).
Proof.
......
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