aboutsummaryrefslogtreecommitdiff
path: root/tactics/contradiction.ml
diff options
context:
space:
mode:
authorPierre-Marie Pédrot2015-10-19 14:32:50 +0200
committerPierre-Marie Pédrot2015-10-19 14:57:32 +0200
commitbdddfe4f3f720a65cdb9ea6ab2573d4adaa8694e (patch)
treebc56e2d01553fae61760d643aac9e08fd24acb46 /tactics/contradiction.ml
parent872d88b5f5c5ab382c7a721f7089bd3085de3cc9 (diff)
Removing tclEVARS in various places.
Diffstat (limited to 'tactics/contradiction.ml')
-rw-r--r--tactics/contradiction.ml13
1 files changed, 8 insertions, 5 deletions
diff --git a/tactics/contradiction.ml b/tactics/contradiction.ml
index 22f218b4fb..0253747641 100644
--- a/tactics/contradiction.ml
+++ b/tactics/contradiction.ml
@@ -13,6 +13,8 @@ open Tactics
open Coqlib
open Reductionops
open Misctypes
+open Sigma.Notations
+open Proofview.Notations
(* Absurd *)
@@ -22,18 +24,19 @@ let mk_absurd_proof t =
mkLambda (Names.Name id,t,mkApp (mkRel 2,[|mkRel 1|])))
let absurd c =
- Proofview.Goal.enter begin fun gl ->
+ Proofview.Goal.s_enter { enter = begin fun gl sigma ->
let env = Proofview.Goal.env gl in
- let sigma = Proofview.Goal.sigma gl in
+ let sigma = Sigma.to_evar_map sigma in
let j = Retyping.get_judgment_of env sigma c in
let sigma, j = Coercion.inh_coerce_to_sort Loc.ghost env sigma j in
let t = j.Environ.utj_val in
+ let tac =
Tacticals.New.tclTHENLIST [
- Proofview.Unsafe.tclEVARS sigma;
elim_type (build_coq_False ());
Simple.apply (mk_absurd_proof t)
- ]
- end
+ ] in
+ Sigma.Unsafe.of_pair (tac, sigma)
+ end }
let absurd c = absurd c