aboutsummaryrefslogtreecommitdiffhomepage
path: root/checker
diff options
context:
space:
mode:
authorGravatar Maxime Dénès <mail@maximedenes.fr>2017-07-31 15:26:39 +0200
committerGravatar Maxime Dénès <mail@maximedenes.fr>2017-07-31 15:26:39 +0200
commit2f349829c125ed0e2d55548935e7b90e7719f12e (patch)
tree2d3003a0072af5ab5f1268c1570b2d83ead70060 /checker
parent9a872809b246bb6af0c177d530581f7c0c36583f (diff)
parente3c247c1d96f39d2c07d120b69598a904b7d9f19 (diff)
Merge PR #761: deprecate Pp.std_ppcmds type and promote Pp.t instead
Diffstat (limited to 'checker')
-rw-r--r--checker/indtypes.mli4
-rw-r--r--checker/univ.ml2
-rw-r--r--checker/univ.mli14
3 files changed, 10 insertions, 10 deletions
diff --git a/checker/indtypes.mli b/checker/indtypes.mli
index 7eaaf65f2..b0554989e 100644
--- a/checker/indtypes.mli
+++ b/checker/indtypes.mli
@@ -12,8 +12,8 @@ open Cic
open Environ
(*i*)
-val prkn : kernel_name -> Pp.std_ppcmds
-val prcon : constant -> Pp.std_ppcmds
+val prkn : kernel_name -> Pp.t
+val prcon : constant -> Pp.t
(*s The different kinds of errors that may result of a malformed inductive
definition. *)
diff --git a/checker/univ.ml b/checker/univ.ml
index e3abc436f..558315c2c 100644
--- a/checker/univ.ml
+++ b/checker/univ.ml
@@ -1071,7 +1071,7 @@ module Instance : sig
val equal : t -> t -> bool
val subst_fn : universe_level_subst_fn -> t -> t
val subst : universe_level_subst -> t -> t
- val pr : t -> Pp.std_ppcmds
+ val pr : t -> Pp.t
val check_eq : t check_function
val length : t -> int
val append : t -> t -> t
diff --git a/checker/univ.mli b/checker/univ.mli
index 7f5aa7626..0a21019b1 100644
--- a/checker/univ.mli
+++ b/checker/univ.mli
@@ -20,7 +20,7 @@ sig
val var : int -> t
- val pr : t -> Pp.std_ppcmds
+ val pr : t -> Pp.t
(** Pretty-printing *)
val equal : t -> t -> bool
@@ -53,7 +53,7 @@ type universe = Universe.t
(** Alias name. *)
-val pr_uni : universe -> Pp.std_ppcmds
+val pr_uni : universe -> Pp.t
(** The universes hierarchy: Type 0- = Prop <= Type 0 = Set <= Type 1 <= ...
Typing of universes: Type 0-, Type 0 : Type 1; Type i : Type (i+1) if i>0 *)
@@ -172,7 +172,7 @@ sig
val subst : universe_level_subst -> t -> t
(** Substitution by a level-to-level function. *)
- val pr : t -> Pp.std_ppcmds
+ val pr : t -> Pp.t
(** Pretty-printing, no comments *)
val check_eq : t check_function
@@ -274,8 +274,8 @@ val check_subtype : universes -> AUContext.t -> AUContext.t -> bool
(** {6 Pretty-printing of universes. } *)
-val pr_constraint_type : constraint_type -> Pp.std_ppcmds
-val pr_constraints : (Level.t -> Pp.std_ppcmds) -> constraints -> Pp.std_ppcmds
-val pr_universe_context : (Level.t -> Pp.std_ppcmds) -> universe_context -> Pp.std_ppcmds
+val pr_constraint_type : constraint_type -> Pp.t
+val pr_constraints : (Level.t -> Pp.t) -> constraints -> Pp.t
+val pr_universe_context : (Level.t -> Pp.t) -> universe_context -> Pp.t
-val pr_universes : universes -> Pp.std_ppcmds
+val pr_universes : universes -> Pp.t