aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar Emilio Jesus Gallego Arias <e+git@x80.org>2016-08-19 00:50:19 +0200
committerGravatar Emilio Jesus Gallego Arias <e+git@x80.org>2016-08-19 00:50:19 +0200
commiteb479438328a473ff1cf5fe010ed714194dbf28f (patch)
tree515e01200e6ed3875c57c3ce97b007c65084580d
parentfa141fa1d2df2720f84a3e2c1fc4900a47f9939f (diff)
[pp] Fix newline issues.
This is a followup to 91ee24b4a7843793a84950379277d92992ba1651 , where we got a few cases wrong wrt to newline endings. Thanks to @herbelin for pointing it out. This doesn't yet fix https://coq.inria.fr/bugs/show_bug.cgi?id=4842
-rw-r--r--pretyping/reductionops.ml4
-rw-r--r--proofs/refiner.ml2
-rw-r--r--toplevel/vernac.ml2
3 files changed, 4 insertions, 4 deletions
diff --git a/pretyping/reductionops.ml b/pretyping/reductionops.ml
index 5484e70b6..8259876c2 100644
--- a/pretyping/reductionops.ml
+++ b/pretyping/reductionops.ml
@@ -790,11 +790,11 @@ let rec whd_state_gen ?csts tactic_mode flags env sigma =
(h 0 (str "<<" ++ Termops.print_constr x ++
str "|" ++ cut () ++ Cst_stack.pr cst_l ++
str "|" ++ cut () ++ Stack.pr Termops.print_constr stack ++
- str ">>") ++ fnl ())
+ str ">>"))
in
let fold () =
let () = if !debug_RAKAM then
- let open Pp in Feedback.msg_notice (str "<><><><><>" ++ fnl ()) in
+ let open Pp in Feedback.msg_notice (str "<><><><><>") in
(s,cst_l)
in
match kind_of_term x with
diff --git a/proofs/refiner.ml b/proofs/refiner.ml
index ebd30820b..ea8543b02 100644
--- a/proofs/refiner.ml
+++ b/proofs/refiner.ml
@@ -221,7 +221,7 @@ let tclSHOWHYPS (tac : tactic) (goal: Goal.goal Evd.sigma)
Feedback.msg_notice
(str (emacs_str "<infoH>")
++ (hov 0 (str s))
- ++ (str (emacs_str "</infoH>")) ++ fnl());
+ ++ (str (emacs_str "</infoH>")));
tclIDTAC goal;;
diff --git a/toplevel/vernac.ml b/toplevel/vernac.ml
index f83ada466..0fc56353e 100644
--- a/toplevel/vernac.ml
+++ b/toplevel/vernac.ml
@@ -101,7 +101,7 @@ let verbose_phrase verbch loc =
let s = String.create len in
seek_in ch (fst loc);
really_input ch s 0 len;
- Feedback.msg_notice (str s ++ fnl ())
+ Feedback.msg_notice (str s)
| None -> ()
exception End_of_input