aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Init/Datatypes.v
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-03-21 14:41:53 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-03-21 14:41:53 +0000
commit94d72b73a6db3918796ca1fa8cb4b21b793dc561 (patch)
tree8cebb2b802593e50c7b8154fd2a55ddafe3e76ed /theories/Init/Datatypes.v
parent637e67a78096cb59ae309329df7ddc6fc9a6149d (diff)
Init: some results in Type should rather be Defined than Qed
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@13920 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Init/Datatypes.v')
-rw-r--r--theories/Init/Datatypes.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Init/Datatypes.v b/theories/Init/Datatypes.v
index 9895bd30b..d7e4b1ff6 100644
--- a/theories/Init/Datatypes.v
+++ b/theories/Init/Datatypes.v
@@ -271,7 +271,7 @@ Hint Unfold CompSpec CompSpecT.
Lemma CompSpec2Type : forall A (eq lt:A->A->Prop) x y c,
CompSpec eq lt x y c -> CompSpecT eq lt x y c.
-Proof. intros. apply CompareSpec2Type; assumption. Qed.
+Proof. intros. apply CompareSpec2Type; assumption. Defined.
(** Identity *)