aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs/refiner.ml
diff options
context:
space:
mode:
authorGravatar ppedrot <ppedrot@85f007b7-540e-0410-9357-904b9bb8a0f7>2013-04-29 16:02:46 +0000
committerGravatar ppedrot <ppedrot@85f007b7-540e-0410-9357-904b9bb8a0f7>2013-04-29 16:02:46 +0000
commit943e6b23229b5eed2fb8265089563ce0a25b9b44 (patch)
tree803aa037f3413c21e76650c62e7ea9173ba3c918 /proofs/refiner.ml
parent4490dfcb94057dd6518963a904565e3a4a354bac (diff)
Merging Context and Sign.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@16463 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'proofs/refiner.ml')
-rw-r--r--proofs/refiner.ml4
1 files changed, 2 insertions, 2 deletions
diff --git a/proofs/refiner.ml b/proofs/refiner.ml
index 04d125804..5a71b6816 100644
--- a/proofs/refiner.ml
+++ b/proofs/refiner.ml
@@ -190,10 +190,10 @@ let tclNOTSAMEGOAL (tac : tactic) goal =
something similar (better?) in the xml protocol. *)
let tclSHOWHYPS (tac : tactic) (goal: Goal.goal Evd.sigma)
:Proof_type.goal list Evd.sigma =
- let oldhyps:Sign.named_context = pf_hyps goal in
+ let oldhyps:Context.named_context = pf_hyps goal in
let rslt:Proof_type.goal list Evd.sigma = tac goal in
let {it=gls;sigma=sigma} = rslt in
- let hyps:Sign.named_context list =
+ let hyps:Context.named_context list =
List.map (fun gl -> pf_hyps { it = gl; sigma=sigma}) gls in
let newhyps =
List.map (fun hypl -> List.subtract hypl oldhyps) hyps in