aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/eqdecide.ml4
diff options
context:
space:
mode:
Diffstat (limited to 'tactics/eqdecide.ml4')
-rw-r--r--tactics/eqdecide.ml44
1 files changed, 2 insertions, 2 deletions
diff --git a/tactics/eqdecide.ml4 b/tactics/eqdecide.ml4
index ac6e944fb..cc6547bc3 100644
--- a/tactics/eqdecide.ml4
+++ b/tactics/eqdecide.ml4
@@ -130,7 +130,7 @@ let solveArg eqonleft op a1 a2 tac =
let solveEqBranch rectype =
Proofview.tclORELSE
begin
- Goal.concl >>- fun concl ->
+ Proofview.Goal.concl >>- fun concl ->
match_eqdec concl >= fun (eqonleft,op,lhs,rhs,_) ->
let (mib,mip) = Global.lookup_inductive rectype in
let nparams = mib.mind_nparams in
@@ -155,7 +155,7 @@ let hd_app c = match kind_of_term c with
let decideGralEquality =
Proofview.tclORELSE
begin
- Goal.concl >>- fun concl ->
+ Proofview.Goal.concl >>- fun concl ->
match_eqdec concl >= fun eqonleft,_,c1,c2,typ ->
Tacmach.New.of_old (fun g -> hd_app (pf_compute g typ)) >>- fun headtyp ->
begin match kind_of_term headtyp with