aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-04-20 08:49:15 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-04-20 08:49:15 +0000
commitde5631d1793834eb26f17f82d5e198b778008f64 (patch)
tree480012375450c2d58242c445dcd5c470cd9ead5a /tactics
parentdc1a605a165f85244f80ef6af17c59cba66587a5 (diff)
Fixed bug #2999 (destruct was not refreshing universes of what it generalized *)
+ changed printing of universe Type(0) to Set, so not to show that the implementation starts numbering with Set=Type(0) while documentation uses Type(0) for the common type of Prop and Set. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12956 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'tactics')
-rw-r--r--tactics/tactics.ml1
1 files changed, 1 insertions, 0 deletions
diff --git a/tactics/tactics.ml b/tactics/tactics.ml
index 51aa86613..41fab4e71 100644
--- a/tactics/tactics.ml
+++ b/tactics/tactics.ml
@@ -2903,6 +2903,7 @@ let apply_induction_with_discharge induct_tac elim indhyps destopt avoid names t
let apply_induction_in_context hyp0 elim indvars names induct_tac gl =
let env = pf_env gl in
let statuslists,lhyp0,indhyps,deps = cook_sign hyp0 indvars env in
+ let deps = List.map (on_pi3 refresh_universes_strict) deps in
let tmpcl = it_mkNamedProd_or_LetIn (pf_concl gl) deps in
let dephyps = List.map (fun (id,_,_) -> id) deps in
let deps_cstr =