aboutsummaryrefslogtreecommitdiffhomepage
path: root/dev/top_printers.mli
diff options
context:
space:
mode:
authorGravatar Gaëtan Gilbert <gaetan.gilbert@skyskimmer.net>2017-12-16 11:00:36 +0100
committerGravatar Gaëtan Gilbert <gaetan.gilbert@skyskimmer.net>2017-12-22 16:41:33 +0100
commit871272d959ac8f2b528cac3677230f2eb33a78c4 (patch)
treeb8784fe607544bf942d6941f1b2b58b9a57421bf /dev/top_printers.mli
parent87cbd64254f33439882156d9a297a6a2f6886057 (diff)
Cleanup top_printers.mli
Diffstat (limited to 'dev/top_printers.mli')
-rw-r--r--dev/top_printers.mli99
1 files changed, 70 insertions, 29 deletions
diff --git a/dev/top_printers.mli b/dev/top_printers.mli
index 44c0c7365..7b5e4a0b6 100644
--- a/dev/top_printers.mli
+++ b/dev/top_printers.mli
@@ -1,5 +1,18 @@
+(************************************************************************)
+(* v * The Coq Proof Assistant / The Coq Development Team *)
+(* <O___,, * INRIA - CNRS - LIX - LRI - PPS - Copyright 1999-2017 *)
+(* \VV/ **************************************************************)
+(* // * This file is distributed under the terms of the *)
+(* * GNU Lesser General Public License Version 2.1 *)
+(************************************************************************)
+
+(** Printers for the ocaml toplevel. *)
+
val pp : Pp.t -> unit
+val pP : Pp.t -> unit (* with surrounding box *)
+
val ppfuture : 'a Future.computation -> unit
+
val ppid : Names.Id.t -> unit
val pplab : Names.Label.t -> unit
val ppmbid : Names.MBId.t -> unit
@@ -9,44 +22,60 @@ val ppcon : Names.Constant.t -> unit
val ppproj : Names.Projection.t -> unit
val ppkn : Names.KerName.t -> unit
val ppmind : Names.MutInd.t -> unit
-val ppind : Names.MutInd.t * int -> unit
+val ppind : Names.inductive -> unit
+
val ppsp : Libnames.full_path -> unit
val ppqualid : Libnames.qualid -> unit
+
val ppclindex : Classops.cl_index -> unit
+
val ppscheme : 'a Ind_tables.scheme_kind -> unit
+
val prrecarg : Declarations.recarg -> Pp.t
val ppwf_paths : Declarations.recarg Rtree.t -> unit
-val envpp : (Environ.env -> Evd.evar_map -> 'a) -> 'a
-val rawdebug : bool ref
+
+val pr_evar : Evar.t -> Pp.t
val ppevar : Evar.t -> unit
-val ppconstr : Constr.t -> unit
-val ppeconstr : EConstr.constr -> unit
-val ppconstr_expr : Constrexpr.constr_expr -> unit
-val ppsconstr : Constr.constr Mod_subst.substituted -> unit
+
+(* Multiple printers for Constr.t *)
+val ppconstr : Constr.t -> unit (* by Termops printer *)
val ppconstr_univ : Constr.t -> unit
+
+(* Extern as type *)
+val pptype : Constr.types -> unit
+
+val ppsconstr : Constr.constr Mod_subst.substituted -> unit
+val ppeconstr : EConstr.constr -> unit (* Termops printer *)
+val ppconstr_expr : Constrexpr.constr_expr -> unit
val ppglob_constr : 'a Glob_term.glob_constr_g -> unit
val pppattern : Pattern.constr_pattern -> unit
-val pptype : Constr.types -> unit
val ppfconstr : CClosure.fconstr -> unit
+
val ppbigint : Bigint.bigint -> unit
-val prset : ('a -> Pp.t) -> 'a list -> Pp.t
+
val ppintset : Int.Set.t -> unit
val ppidset : Names.Id.Set.t -> unit
-val prset' : ('a -> Pp.t) -> 'a list -> Pp.t
+
val pridmap : (Names.Id.Map.key -> 'a -> Pp.t) -> 'a Names.Id.Map.t -> Pp.t
val ppidmap : (Names.Id.Map.key -> 'a -> Pp.t) -> 'a Names.Id.Map.t -> unit
+
val pridmapgen : 'a Names.Id.Map.t -> Pp.t
val ppidmapgen : 'a Names.Id.Map.t -> unit
-val ppevarsubst :
- (Constr.t * Constr.t option * Names.Id.Map.key) list Names.Id.Map.t -> unit
+
val prididmap : Names.Id.t Names.Id.Map.t -> Pp.t
val ppididmap : Names.Id.t Names.Id.Map.t -> unit
+
val prconstrunderbindersidmap :
(Names.Id.t list * EConstr.constr) Names.Id.Map.t -> Pp.t
val ppconstrunderbindersidmap :
(Names.Id.t list * EConstr.constr) Names.Id.Map.t -> unit
+
+val ppevarsubst :
+ (Constr.t * Constr.t option * Names.Id.Map.key) list Names.Id.Map.t -> unit
+
val ppunbound_ltac_var_map :
'a Genarg.generic_argument Names.Id.Map.t -> unit
+
val pr_closure : Ltac_pretype.closure -> Pp.t
val pr_closed_glob_constr_idmap :
Ltac_pretype.closed_glob_constr Names.Id.Map.t -> Pp.t
@@ -55,40 +84,54 @@ val ppclosure : Ltac_pretype.closure -> unit
val ppclosedglobconstr : Ltac_pretype.closed_glob_constr -> unit
val ppclosedglobconstridmap :
Ltac_pretype.closed_glob_constr Names.Id.Map.t -> unit
-val pP : Pp.t -> unit
-val safe_pr_global : Globnames.global_reference -> unit
+
val ppglobal : Globnames.global_reference -> unit
+
val ppconst :
Names.KerName.t * (Constr.constr, 'a) Environ.punsafe_judgment -> unit
val ppvar : Names.Id.t * Constr.constr -> unit
+
val genppj : ('a -> Pp.t * Pp.t) -> 'a -> Pp.t
val ppj : EConstr.unsafe_judgment -> unit
+
val ppsubst : Mod_subst.substitution -> unit
val ppdelta : Mod_subst.delta_resolver -> unit
+
val pp_idpred : Names.Id.Pred.t -> unit
val pp_cpred : Names.Cpred.t -> unit
val pp_transparent_state : Names.transparent_state -> unit
+
val pp_stack_t : Constr.t Reductionops.Stack.t -> unit
val pp_cst_stack_t : Reductionops.Cst_stack.t -> unit
val pp_state_t : Reductionops.state -> unit
-val pr_evar : Evar.t -> Pp.t
+
val ppmetas : Evd.Metaset.t -> unit
val ppevm : Evd.evar_map -> unit
val ppevmall : Evd.evar_map -> unit
+
val pr_existentialset : Evar.Set.t -> Pp.t
val ppexistentialset : Evar.Set.t -> unit
+
val ppexistentialfilter : Evd.Filter.t -> unit
+
val ppclenv : Clenv.clausenv -> unit
+
val ppgoalgoal : Goal.goal -> unit
+
val ppgoal : Proof_type.goal Evd.sigma -> unit
+(* also print evar map *)
val ppgoalsigma : Proof_type.goal Evd.sigma -> unit
+
val pphintdb : Hints.Hint_db.t -> unit
val ppproofview : Proofview.proofview -> unit
val ppopenconstr : Evd.open_constr -> unit
+
val pproof : Proof.t -> unit
+
+(* Universes *)
val ppuni : Univ.Universe.t -> unit
-val ppuni_level : Univ.Level.t -> unit
-val prlev : Univ.Level.t -> Pp.t
+val ppuni_level : Univ.Level.t -> unit (* raw *)
+val prlev : Univ.Level.t -> Pp.t (* with global names (does this work?) *)
val ppuniverse_set : Univ.LSet.t -> unit
val ppuniverse_instance : Univ.Instance.t -> unit
val ppuniverse_context : Univ.UContext.t -> unit
@@ -103,30 +146,28 @@ val ppuniverse_context_future : Univ.UContext.t Future.computation -> unit
val ppcumulativity_info : Univ.CumulativityInfo.t -> unit
val ppabstract_cumulativity_info : Univ.ACumulativityInfo.t -> unit
val ppuniverses : UGraph.t -> unit
+
val ppnamedcontextval : Environ.named_context_val -> unit
val ppenv : Environ.env -> unit
val ppenvwithcst : Environ.env -> unit
+
val pptac : Tacexpr.glob_tactic_expr -> unit
+
val ppobj : Libobject.obj -> unit
-val cnt : int ref
+
+(* Some super raw printers *)
val cast_kind_display : Constr.cast_kind -> string
val constr_display : Constr.constr -> unit
val print_pure_constr : Constr.types -> unit
+
val pploc : Loc.t -> unit
+
val pp_argument_type : Genarg.argument_type -> unit
val pp_generic_argument : 'a Genarg.generic_argument -> unit
+
val prgenarginfo : Geninterp.Val.t -> Pp.t
val ppgenarginfo : Geninterp.Val.t -> unit
+
val ppgenargargt : ('a, 'b, 'c) Genarg.ArgT.tag -> unit
+
val ppist : Geninterp.interp_sign -> unit
-val in_current_context :
- (Constr.constr -> 'a) -> Constrexpr.constr_expr -> 'a
-val encode_path :
- ?loc:Loc.t ->
- string ->
- (Names.ModPath.t * Names.DirPath.t) option ->
- Names.module_ident list -> Names.Id.t -> Libnames.reference
-val raw_string_of_ref :
- ?loc:Loc.t -> 'a -> Globnames.global_reference -> Libnames.reference
-val short_string_of_ref :
- ?loc:Loc.t -> 'a -> Globnames.global_reference -> Libnames.reference