aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/leminv.ml
diff options
context:
space:
mode:
authorGravatar Gaëtan Gilbert <gaetan.gilbert@skyskimmer.net>2017-09-08 14:58:28 +0200
committerGravatar Gaëtan Gilbert <gaetan.gilbert@skyskimmer.net>2017-09-08 18:42:37 +0200
commitb71e68fb78ccde52f1aaa63ef26f0135b92e9be5 (patch)
treefd07ca12f3aa602a082cc960a82f031ea72fa7c3 /tactics/leminv.ml
parentb1fbec7e3945fe2965f4ba9f80c8c31b821dbce1 (diff)
Parse directly to Sorts.family when appropriate.
When we used to parse to a glob_sort but always give an empty list in the GType case we can now parse directly to Sorts.family.
Diffstat (limited to 'tactics/leminv.ml')
-rw-r--r--tactics/leminv.ml4
1 files changed, 2 insertions, 2 deletions
diff --git a/tactics/leminv.ml b/tactics/leminv.ml
index aeb80ae57..967ec2a71 100644
--- a/tactics/leminv.ml
+++ b/tactics/leminv.ml
@@ -248,9 +248,9 @@ let add_inversion_lemma_exn na com comsort bool tac =
let env = Global.env () in
let evd = ref (Evd.from_env env) in
let c = Constrintern.interp_type_evars env evd com in
- let sigma, sort = Pretyping.interp_sort !evd comsort in
+ let evd, sort = Evd.fresh_sort_in_family ~rigid:univ_rigid env !evd comsort in
try
- add_inversion_lemma na env sigma c sort bool tac
+ add_inversion_lemma na env evd c sort bool tac
with
| UserError (Some "Case analysis",s) -> (* Reference to Indrec *)
user_err ~hdr:"Inv needs Nodep Prop Set" s