aboutsummaryrefslogtreecommitdiffhomepage
path: root/printing
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2012-10-06 10:08:51 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2012-10-06 10:08:51 +0000
commit0256a92eb0d0265750bd38a85dce4f9487aefe5b (patch)
treee2786cc2476aebafa664db64da2ab787f18a887a /printing
parent30cf9c6711df3eb583dacad3cb98158adbbf1f5f (diff)
still some more dead code removal
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@15875 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'printing')
-rw-r--r--printing/pptactic.ml12
-rw-r--r--printing/ppvernac.ml4
2 files changed, 0 insertions, 16 deletions
diff --git a/printing/pptactic.ml b/printing/pptactic.ml
index 48a59be05..2ec66bb34 100644
--- a/printing/pptactic.ml
+++ b/printing/pptactic.ml
@@ -980,15 +980,6 @@ let strip_prod_binders_glob_constr n (ty,_) =
| _ -> error "Cannot translate fix tactic: not enough products" in
strip_ty [] n ty
-let strip_prod_binders_constr n ty =
- let rec strip_ty acc n ty =
- if n=0 then (List.rev acc, ty) else
- match Term.kind_of_term ty with
- Term.Prod(na,a,b) ->
- strip_ty (([Loc.ghost,na],a)::acc) (n-1) b
- | _ -> error "Cannot translate fix tactic: not enough products" in
- strip_ty [] n ty
-
let drop_env f _env = f
let pr_constr_or_lconstr_pattern_expr b =
@@ -1030,9 +1021,6 @@ let rec glob_printers =
and pr_glob_tactic_level env n (t:glob_tactic_expr) =
fst (make_pr_tac glob_printers env) n t
-let pr_constr_or_lconstr_pattern b =
- if b then pr_lconstr_pattern else pr_constr_pattern
-
let pr_raw_tactic env = pr_raw_tactic_level env ltop
let pr_glob_tactic env = pr_glob_tactic_level env ltop
diff --git a/printing/ppvernac.ml b/printing/ppvernac.ml
index 3553373fb..686d2ae2d 100644
--- a/printing/ppvernac.ml
+++ b/printing/ppvernac.ml
@@ -175,10 +175,6 @@ let pr_set_option a b =
let pr_topcmd _ = str"(* <Warning> : No printer for toplevel commands *)"
-let pr_destruct_location = function
- | Tacexpr.ConclLocation () -> str"Conclusion"
- | Tacexpr.HypLocation b -> if b then str"Discardable Hypothesis" else str"Hypothesis"
-
let pr_opt_hintbases l = match l with
| [] -> mt()
| _ as z -> str":" ++ spc() ++ prlist_with_sep sep str z