aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Init/Datatypes.v
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-02-13 15:51:45 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-02-13 15:51:45 +0000
commit91a8204515286252d0f026fcfc60a014bc57e727 (patch)
tree57b6eef6d83a05423be5f1c0089832b2bb376970 /theories/Init/Datatypes.v
parent2b73159ba68c43c881b6c8a64134cbc473c9dc91 (diff)
CompSpec2Type is used to build functions, it should be Defined, not Qed
This solves in particular the compilation failure of contrib ATBR git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12765 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 4782194a3..092fce996 100644
--- a/theories/Init/Datatypes.v
+++ b/theories/Init/Datatypes.v
@@ -246,7 +246,7 @@ 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.
destruct c; intros H; constructor; inversion_clear H; auto.
-Qed.
+Defined.
(** Identity *)