aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs
diff options
context:
space:
mode:
authorGravatar barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-03-04 18:45:10 +0000
committerGravatar barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-03-04 18:45:10 +0000
commit52aff80a4736ccaeb8610185959affb516a6bd9f (patch)
tree99db8c65bdbf66c45c7ce3d313d25ddc3156e8bf /proofs
parentec6ef01a50f874bae1fc2d8cc2513e303f2a575c (diff)
commande Timeout + compaction des traces de debug_tactic
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@11959 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'proofs')
-rw-r--r--proofs/proof_type.ml4
-rw-r--r--proofs/proof_type.mli4
2 files changed, 4 insertions, 4 deletions
diff --git a/proofs/proof_type.ml b/proofs/proof_type.ml
index dabc84ca3..5bd8060ae 100644
--- a/proofs/proof_type.ml
+++ b/proofs/proof_type.ml
@@ -102,8 +102,8 @@ type ltac_call_kind =
| LtacConstrInterp of rawconstr *
((identifier * constr) list * (identifier * identifier option) list)
-type ltac_trace = (loc * ltac_call_kind) list
+type ltac_trace = (int * loc * ltac_call_kind) list
-exception LtacLocated of (ltac_call_kind * ltac_trace * loc) * exn
+exception LtacLocated of (int * ltac_call_kind * ltac_trace * loc) * exn
let abstract_tactic_box = ref (ref None)
diff --git a/proofs/proof_type.mli b/proofs/proof_type.mli
index 1529a07f3..0bd0eaa11 100644
--- a/proofs/proof_type.mli
+++ b/proofs/proof_type.mli
@@ -137,8 +137,8 @@ type ltac_call_kind =
| LtacConstrInterp of rawconstr *
((identifier * constr) list * (identifier * identifier option) list)
-type ltac_trace = (loc * ltac_call_kind) list
+type ltac_trace = (int * loc * ltac_call_kind) list
-exception LtacLocated of (ltac_call_kind * ltac_trace * loc) * exn
+exception LtacLocated of (int * ltac_call_kind * ltac_trace * loc) * exn
val abstract_tactic_box : atomic_tactic_expr option ref ref