diff src/Universes.v @ 436:5d5e44f905c7

Changes during more coqdoc hacking
author Adam Chlipala <adam@chlipala.net>
date Fri, 27 Jul 2012 15:41:06 -0400
parents a54a4a2ea6e4
children 8077352044b2
line wrap: on
line diff
--- a/src/Universes.v	Thu Jul 26 19:05:12 2012 -0400
+++ b/src/Universes.v	Fri Jul 27 15:41:06 2012 -0400
@@ -776,6 +776,10 @@
     end.
 Qed.
 
+(* begin hide *)
+Require Eqdep_dec.
+(* end hide *)
+
 (** These corollaries are special cases of proof irrelevance.  In developments that only need proof irrelevance for equality, there is no need to assert full irrelevance.
 
    Another facet of proof irrelevance is that, like excluded middle, it is often provable for specific propositions.  For instance, [UIP] is provable whenever the type [A] has a decidable equality operation.  The module [Eqdep_dec] of the standard library contains a proof.  A similar phenomenon applies to other notable cases, including less-than proofs.  Thus, it is often possible to use proof irrelevance without asserting axioms.
@@ -844,6 +848,10 @@
 
   This axiom lets us convert a relational specification [R] into a function implementing that specification.  We need only prove that [R] is truly a function.  An alternate, stronger formulation applies to cases where [R] maps each input to one or more outputs.  We also simplify the statement of the theorem by considering only non-dependent function types. *)
 
+(* begin hide *)
+Require RelationalChoice.
+(* end hide *)
+
 Require Import ClassicalChoice.
 Check choice.
 (** %\vspace{-.15in}% [[