aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Init/Datatypes.v
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2016-09-13 22:12:35 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2017-03-03 09:51:33 +0100
commitd8f42feb4f4e6c4e062678e256499e03454c7ab2 (patch)
tree66049d9a8dbe72a01132d4c6ecdd66ad5d2a6f1d /theories/Init/Datatypes.v
parent1682d4ed9df64937dfaa162e58233020036ff7b3 (diff)
Compatibility of iff wrt not and imp.
This completes the series and cannot hurt.
Diffstat (limited to 'theories/Init/Datatypes.v')
-rw-r--r--theories/Init/Datatypes.v1
1 files changed, 0 insertions, 1 deletions
diff --git a/theories/Init/Datatypes.v b/theories/Init/Datatypes.v
index ddaf08bf7..4e3f2e80f 100644
--- a/theories/Init/Datatypes.v
+++ b/theories/Init/Datatypes.v
@@ -326,7 +326,6 @@ 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. Defined.
-
(******************************************************************)
(** * Misc Other Datatypes *)