aboutsummaryrefslogtreecommitdiffhomepage
path: root/vernac
diff options
context:
space:
mode:
authorGravatar Gaëtan Gilbert <gaetan.gilbert@skyskimmer.net>2017-11-10 13:23:32 +0100
committerGravatar Gaëtan Gilbert <gaetan.gilbert@skyskimmer.net>2018-02-10 01:34:19 +0100
commit1ed0836a7e0c8e05b0288f85e344ef5249d5d228 (patch)
treee36199b1ff1f6a7ddf83ba164c131339b5061f6c /vernac
parent35fba70509d9fb219b2a88f8e7bd246b2671b39b (diff)
Inference of inductive subtyping does not need an evar map.
Diffstat (limited to 'vernac')
-rw-r--r--vernac/comInductive.ml2
-rw-r--r--vernac/record.ml11
2 files changed, 2 insertions, 11 deletions
diff --git a/vernac/comInductive.ml b/vernac/comInductive.ml
index 3f8d413b7..faac16802 100644
--- a/vernac/comInductive.ml
+++ b/vernac/comInductive.ml
@@ -356,7 +356,7 @@ let interp_mutual_inductive (paramsl,indl) notations cum poly prv finite =
}
in
(if poly && cum then
- Inductiveops.infer_inductive_subtyping env_ar sigma mind_ent
+ Inductiveops.infer_inductive_subtyping env_ar mind_ent
else mind_ent), Evd.universe_binders sigma, impls
(* Very syntactical equality *)
diff --git a/vernac/record.ml b/vernac/record.ml
index 31c0483b4..6e35ac4db 100644
--- a/vernac/record.ml
+++ b/vernac/record.ml
@@ -423,16 +423,7 @@ let declare_structure finite ubinders univs id idbuild paramimpls params arity t
mind_entry_universes = univs;
}
in
- let mie =
- match ctx with
- | Polymorphic_const_entry ctx ->
- let env = Global.env () in
- let env' = Environ.push_context ctx env in
- let evd = Evd.from_env env' in
- Inductiveops.infer_inductive_subtyping env' evd mie
- | Monomorphic_const_entry _ ->
- mie
- in
+ let mie = Inductiveops.infer_inductive_subtyping (Global.env ()) mie in
let kn = ComInductive.declare_mutual_inductive_with_eliminations mie ubinders [(paramimpls,[])] in
let rsp = (kn,0) in (* This is ind path of idstruc *)
let cstr = (rsp,1) in