aboutsummaryrefslogtreecommitdiffhomepage
path: root/contrib/interface/debug_tac.ml4
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-11-12 19:42:43 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-11-12 19:42:43 +0000
commitc37a44c11076bc22f81e2ef9ee75a36f383e436a (patch)
tree0f517b675cd6e7a5076017674b1b68737e522de1 /contrib/interface/debug_tac.ml4
parente95cfce6398e41f0150aa6340bf8bc37eb66799f (diff)
Bug TacId
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4884 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'contrib/interface/debug_tac.ml4')
-rw-r--r--contrib/interface/debug_tac.ml46
1 files changed, 3 insertions, 3 deletions
diff --git a/contrib/interface/debug_tac.ml4 b/contrib/interface/debug_tac.ml4
index ca43d0077..bf596b284 100644
--- a/contrib/interface/debug_tac.ml4
+++ b/contrib/interface/debug_tac.ml4
@@ -355,7 +355,7 @@ let rec reconstruct_success_tac (tac:glob_tactic_expr) =
Report_node(true, n, l) -> tac
| Report_node(false, n, rl) ->
TacThens (a,List.map2 reconstruct_success_tac l rl)
- | Failed n -> TacId
+ | Failed n -> TacId ""
| Tree_fail r -> reconstruct_success_tac a r
| Mismatch (n,p) -> a)
| TacThen (a,b) ->
@@ -367,13 +367,13 @@ let rec reconstruct_success_tac (tac:glob_tactic_expr) =
[in_gen globwit_tactic a;
in_gen globwit_tactic b;
in_gen (wit_list0 globwit_int) selected_indices]))
- | Failed n -> TacId
+ | Failed n -> TacId ""
| Tree_fail r -> reconstruct_success_tac a r
| _ -> error "this error case should not happen in a THEN tactic")
| _ ->
(function
Report_node(true, n, l) -> tac
- | Failed n -> TacId
+ | Failed n -> TacId ""
| _ ->
errorlabstrm
"this error case should not happen on an unknown tactic"