aboutsummaryrefslogtreecommitdiffhomepage
path: root/parsing/printer.mli
diff options
context:
space:
mode:
Diffstat (limited to 'parsing/printer.mli')
-rw-r--r--parsing/printer.mli40
1 files changed, 22 insertions, 18 deletions
diff --git a/parsing/printer.mli b/parsing/printer.mli
index ff3179c7d..67434ee31 100644
--- a/parsing/printer.mli
+++ b/parsing/printer.mli
@@ -6,6 +6,7 @@ open Pp
open Names
open Term
open Sign
+open Environ
open Rawterm
open Pattern
(*i*)
@@ -13,40 +14,43 @@ open Pattern
(* These are the entry points for printing terms, context, tac, ... *)
val gentacpr : Coqast.t -> std_ppcmds
-val prterm_env : 'a assumptions -> constr -> std_ppcmds
-val prterm_env_at_top : 'a assumptions -> constr -> std_ppcmds
+val prterm_env : env -> constr -> std_ppcmds
+val prterm_env_at_top : env -> constr -> std_ppcmds
val prterm : constr -> std_ppcmds
-val prtype_env : 'a assumptions -> typed_type -> std_ppcmds
+val prtype_env : env -> typed_type -> std_ppcmds
val prtype : typed_type -> std_ppcmds
val prjudge_env :
- 'a assumptions -> Environ.unsafe_judgment -> std_ppcmds * std_ppcmds
+ env -> Environ.unsafe_judgment -> std_ppcmds * std_ppcmds
val prjudge : Environ.unsafe_judgment -> std_ppcmds * std_ppcmds
val pr_rawterm : Rawterm.rawconstr -> std_ppcmds
val pr_cases_pattern : Rawterm.cases_pattern -> std_ppcmds
-val pr_constant : 'a assumptions -> constant -> std_ppcmds
-val pr_existential : 'a assumptions -> existential -> std_ppcmds
-val pr_constructor : 'a assumptions -> constructor -> std_ppcmds
-val pr_inductive : 'a assumptions -> inductive -> std_ppcmds
+val pr_constant : env -> constant -> std_ppcmds
+val pr_existential : env -> existential -> std_ppcmds
+val pr_constructor : env -> constructor -> std_ppcmds
+val pr_inductive : env -> inductive -> std_ppcmds
val pr_ref_label : constr_label -> std_ppcmds
val pr_pattern : constr_pattern -> std_ppcmds
-val pr_pattern_env : 'a assumptions -> constr_pattern -> std_ppcmds
+val pr_pattern_env : names_context -> constr_pattern -> std_ppcmds
-val pr_ne_env : std_ppcmds -> path_kind -> context -> std_ppcmds
+val pr_ne_context_of : std_ppcmds -> path_kind -> env -> std_ppcmds
-val pr_sign : var_context -> std_ppcmds
-val pr_env_opt : context -> std_ppcmds
+val pr_var_decl : env -> var_declaration -> std_ppcmds
+val pr_rel_decl : env -> rel_declaration -> std_ppcmds
-val emacs_str : string -> string
+val pr_var_context_of : env -> std_ppcmds
+val pr_rel_context : env -> rel_context -> std_ppcmds
+val pr_context_of : env -> std_ppcmds
-(* For compatibility *)
-val term0 : 'a assumptions -> constr -> std_ppcmds
+val emacs_str : string -> string
-val fprterm_env : 'a assumptions -> constr -> std_ppcmds
+(*i*)
+val fprterm_env : env -> constr -> std_ppcmds
val fprterm : constr -> std_ppcmds
-val fprtype_env : 'a assumptions -> typed_type -> std_ppcmds
+val fprtype_env : env -> typed_type -> std_ppcmds
val fprtype : typed_type -> std_ppcmds
(* For compatibility *)
-val fterm0 : 'a assumptions -> constr -> std_ppcmds
+val fterm0 : env -> constr -> std_ppcmds
+(*i*)