aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Init/Datatypes.v
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <mattam@mattam.org>2014-04-28 13:47:25 +0200
committerGravatar Matthieu Sozeau <mattam@mattam.org>2014-05-06 09:59:01 +0200
commit902da7d2949464ff54dafc3fda1d44365270d2e1 (patch)
treee8af894bb79090b316df4fbd247e09fb464bd2ac /theories/Init/Datatypes.v
parent6869b22e2546b69acb74e18dc491029897ba36a3 (diff)
Try a new way of handling template universe levels
Diffstat (limited to 'theories/Init/Datatypes.v')
-rw-r--r--theories/Init/Datatypes.v6
1 files changed, 3 insertions, 3 deletions
diff --git a/theories/Init/Datatypes.v b/theories/Init/Datatypes.v
index 9b5d7ffb0..c8d18f766 100644
--- a/theories/Init/Datatypes.v
+++ b/theories/Init/Datatypes.v
@@ -153,10 +153,10 @@ Inductive option (A:Type) : Type :=
Arguments None [A].
-Definition option_map (A B:Type) (f:A->B) o :=
+Definition option_map (A B:Type) (f:A->B) (o : option A) : option B :=
match o with
- | Some a => Some (f a)
- | None => None
+ | Some a => @Some B (f a)
+ | None => @None B
end.
(** [sum A B], written [A + B], is the disjoint sum of [A] and [B] *)