aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/tactics.ml
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2016-11-29 16:30:00 +0100
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2017-02-14 17:30:44 +0100
commitd549d9d3d169fbfc5f555e3e4f22f46301161d53 (patch)
tree4cb4052135639414c1f46e3f61a2064ed74d94eb /tactics/tactics.ml
parent4e9cebb0641927f11a21cbb50828974f910cfe47 (diff)
Do not ask for a normalized goal to get hypotheses and conclusions.
This is now useless as this returns evar-constrs, so that all functions acting on them should be insensitive to evar-normalization.
Diffstat (limited to 'tactics/tactics.ml')
-rw-r--r--tactics/tactics.ml12
1 files changed, 6 insertions, 6 deletions
diff --git a/tactics/tactics.ml b/tactics/tactics.ml
index 4bf848a9c..de3572155 100644
--- a/tactics/tactics.ml
+++ b/tactics/tactics.ml
@@ -208,7 +208,7 @@ let convert_concl ?(check=true) ty k =
Proofview.Goal.enter { enter = begin fun gl ->
let env = Proofview.Goal.env gl in
let store = Proofview.Goal.extra gl in
- let conclty = Proofview.Goal.raw_concl gl in
+ let conclty = Proofview.Goal.concl gl in
Refine.refine ~unsafe:true { run = begin fun sigma ->
let Sigma ((), sigma, p) =
if check then begin
@@ -228,7 +228,7 @@ let convert_hyp ?(check=true) d =
Proofview.Goal.enter { enter = begin fun gl ->
let env = Proofview.Goal.env gl in
let sigma = Tacmach.New.project gl in
- let ty = Proofview.Goal.raw_concl gl in
+ let ty = Proofview.Goal.concl gl in
let store = Proofview.Goal.extra gl in
let sign = convert_hyp check (named_context_val env) sigma d in
let env = reset_with_named_context sign env in
@@ -328,7 +328,7 @@ let move_hyp id dest =
Proofview.Goal.enter { enter = begin fun gl ->
let env = Proofview.Goal.env gl in
let sigma = Tacmach.New.project gl in
- let ty = Proofview.Goal.raw_concl gl in
+ let ty = Proofview.Goal.concl gl in
let store = Proofview.Goal.extra gl in
let sign = named_context_val env in
let sign' = move_hyp_in_named_context sigma id dest sign in
@@ -756,7 +756,7 @@ let e_reduct_option ?(check=false) redfun = function
let e_change_in_concl (redfun,sty) =
Proofview.Goal.s_enter { s_enter = begin fun gl ->
let sigma = Proofview.Goal.sigma gl in
- let Sigma (c, sigma, p) = redfun.e_redfun (Proofview.Goal.env gl) sigma (Proofview.Goal.raw_concl gl) in
+ let Sigma (c, sigma, p) = redfun.e_redfun (Proofview.Goal.env gl) sigma (Proofview.Goal.concl gl) in
Sigma (convert_concl_no_check c sty, sigma, p)
end }
@@ -4340,7 +4340,7 @@ let pose_induction_arg_then isrec with_evars (is_arg_pure_hyp,from_prefix) elim
Proofview.Goal.s_enter { s_enter = begin fun gl ->
let sigma = Proofview.Goal.sigma gl in
let env = Proofview.Goal.env gl in
- let ccl = Proofview.Goal.raw_concl gl in
+ let ccl = Proofview.Goal.concl gl in
let store = Proofview.Goal.extra gl in
let check = check_enough_applied env sigma elim in
let Sigma (c, sigma', p) = use_bindings env sigma elim false (c0,lbind) t0 in
@@ -4409,7 +4409,7 @@ let induction_gen clear_flag isrec with_evars elim
let env = Proofview.Goal.env gl in
let sigma = Proofview.Goal.sigma gl in
let evd = Sigma.to_evar_map sigma in
- let ccl = Proofview.Goal.raw_concl gl in
+ let ccl = Proofview.Goal.concl gl in
let cls = Option.default allHypsAndConcl cls in
let t = typ_of env sigma c in
let is_arg_pure_hyp =