aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Init/Specif.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/Init/Specif.v')
-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 *)