aboutsummaryrefslogtreecommitdiffhomepage
path: root/translate/ppvernacnew.ml
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-05-13 22:10:03 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-05-13 22:10:03 +0000
commit1d77fef0f749dc3a629f8ebd29dfebe1311eb497 (patch)
tree883ee1b75202153a3e9c7c9fe6df845c4c3a2467 /translate/ppvernacnew.ml
parent6006880b1ab124ae7c229dc3dc513b49229c9813 (diff)
Separation entre les propositions de syntaxe - suite
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4005 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'translate/ppvernacnew.ml')
-rw-r--r--translate/ppvernacnew.ml12
1 files changed, 7 insertions, 5 deletions
diff --git a/translate/ppvernacnew.ml b/translate/ppvernacnew.ml
index e0e2c4a65..4a16fbaee 100644
--- a/translate/ppvernacnew.ml
+++ b/translate/ppvernacnew.ml
@@ -243,7 +243,7 @@ let anonymize_binder na c =
else c
let sep_fields () =
- if !Options.p1 then str ";" ++ spc () else fnl ()
+ if !Options.p1 then fnl () else str ";" ++ spc ()
let surround_binder p =
if !Options.p1 then str"(" ++ p ++ str")" else p
@@ -708,7 +708,7 @@ let rec pr_vernac = function
(* Solving *)
| VernacSolve (i,tac,deftac) ->
- (if i = 1 then mt() else int i ++ str ": ") ++
+ (if i = 1 then mt() else int i ++ str ": ") ++
(if !Options.p1 then mt () else str "By ") ++
(if deftac then mt() else str "!! ") ++
pr_raw_tactic_goal i tac
@@ -753,9 +753,11 @@ let rec pr_vernac = function
(List.map (fun ((_,id),_) -> (id,Lib.make_path id)) l)
(Global.env()) body in
hov 1
- ((* Rec by default: (if rc then str "Recursive " else mt()) ++ *)
- str "Ltac " ++
- prlist_with_sep (fun () -> fnl() ++ str"with ") pr_tac_body l)
+ ((if !Options.p1 then
+ (if rc then str "Recursive " else mt()) ++
+ str "Tactic Definition " else
+ (* Rec by default *) str "Ltac ") ++
+ prlist_with_sep (fun () -> fnl() ++ str"with ") pr_tac_body l)
| VernacHints (dbnames,h) -> pr_hints dbnames h pr_constr
| VernacHintDestruct (id,loc,c,i,tac) ->
hov 2 (str"HintDestruct " ++ pr_destruct_location loc ++ spc() ++