aboutsummaryrefslogtreecommitdiffhomepage
path: root/vernac/class.ml
diff options
context:
space:
mode:
authorGravatar Gaƫtan Gilbert <gaetan.gilbert@skyskimmer.net>2017-09-09 14:00:42 +0200
committerGravatar Matthieu Sozeau <mattam@mattam.org>2017-09-19 10:28:03 +0200
commitcd29948855c2cbd3f4065170e41f8dbe625e1921 (patch)
treee747c92a12074f2d0753b902c5fe00261d0a0fe4 /vernac/class.ml
parentc2b881aae9c71a34199d2c66282512f2bdb19cf6 (diff)
Don't lose names in UState.universe_context.
We dont care about the order of the binder map ([map] in the code) so no need to do tricky things with it.
Diffstat (limited to 'vernac/class.ml')
-rw-r--r--vernac/class.ml3
1 files changed, 2 insertions, 1 deletions
diff --git a/vernac/class.ml b/vernac/class.ml
index be682977e..3915148a0 100644
--- a/vernac/class.ml
+++ b/vernac/class.ml
@@ -222,9 +222,10 @@ let build_id_coercion idf_opt source poly =
Id.of_string ("Id_"^(ident_key_of_class source)^"_"^
(ident_key_of_class cl))
in
+ let univs = (snd (Evd.universe_context ~names:[] ~extensible:true sigma)) in
let constr_entry = (* Cast is necessary to express [val_f] is identity *)
DefinitionEntry
- (definition_entry ~types:typ_f ~poly ~univs:(snd (Evd.universe_context sigma))
+ (definition_entry ~types:typ_f ~poly ~univs
~inline:true (mkCast (val_f, DEFAULTcast, typ_f)))
in
let decl = (constr_entry, IsDefinition IdentityCoercion) in