aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Init
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-05-12 18:25:06 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-05-12 18:25:06 +0000
commit15bbdcfa63dd7fee30b3d03f98cf0795e4baf087 (patch)
treed547b755963a3f6c59fb2da66d30ab81ae4fa4de /theories/Init
parent651a23b4b21045733d44a4bc944b6b56d449fe2e (diff)
MAJ et bricoles diverses
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10923 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Init')
-rw-r--r--theories/Init/Specif.v3
1 files changed, 3 insertions, 0 deletions
diff --git a/theories/Init/Specif.v b/theories/Init/Specif.v
index 4f642a73e..2244e1b9a 100644
--- a/theories/Init/Specif.v
+++ b/theories/Init/Specif.v
@@ -115,6 +115,9 @@ Proof. destruct 1 as (x,H); exists x; trivial. Defined.
Lemma sigT_of_sig : forall (A:Type) (P:A->Prop), sig P -> sigT P.
Proof. destruct 1 as (x,H); exists x; trivial. Defined.
+Coercion sigT_of_sig : sig >-> sigT.
+Coercion sig_of_sigT : sigT >-> sig.
+
(** [sumbool] is a boolean type equipped with the justification of
their value *)