aboutsummaryrefslogtreecommitdiffhomepage
path: root/translate
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-11-19 14:31:51 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-11-19 14:31:51 +0000
commitcff24d313545efba6bd14116b83bd3fa0b7f44ff (patch)
treea1c77555098c23f0a7271c0d668bad6aee20b97b /translate
parent26f2ff64a641f1767abb1a0d3da3e7449a5835d3 (diff)
Distinction entre 'as _' qui cache le terme filtre (si variable) et rien dans case_item
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4949 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'translate')
-rw-r--r--translate/ppconstrnew.ml5
1 files changed, 5 insertions, 0 deletions
diff --git a/translate/ppconstrnew.ml b/translate/ppconstrnew.ml
index af8fb845d..8104399c0 100644
--- a/translate/ppconstrnew.ml
+++ b/translate/ppconstrnew.ml
@@ -351,12 +351,17 @@ let tm_clash = function
let pr_case_item pr (tm,(na,indnalopt)) =
hov 0 (pr (lcast,E) tm ++
+(*
(match na with
| Name id when not (is_var id tm) -> spc () ++ str "as " ++ pr_id id
| Anonymous when tm_clash (tm,indnalopt) <> None ->
(* hide [tm] name to avoid conflicts *)
spc () ++ str "as _" (* ++ pr_id (out_some (tm_clash (tm,indnalopt)))*)
| _ -> mt ()) ++
+*)
+ (match na with (* Decision of printing "_" or not moved to constrextern.ml *)
+ | Some na -> spc () ++ str "as " ++ pr_name na
+ | None -> mt ()) ++
(match indnalopt with
| None -> mt ()
(*