aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
-rw-r--r--plugins/firstorder/g_ground.ml46
-rw-r--r--printing/ppconstr.ml2
-rw-r--r--printing/pptactic.ml11
-rw-r--r--printing/ppvernac.ml2
-rw-r--r--theories/Relations/Operators_Properties.v3
5 files changed, 13 insertions, 11 deletions
diff --git a/plugins/firstorder/g_ground.ml4 b/plugins/firstorder/g_ground.ml4
index c3ae05de6..10e2e1773 100644
--- a/plugins/firstorder/g_ground.ml4
+++ b/plugins/firstorder/g_ground.ml4
@@ -106,9 +106,9 @@ open Pp
open Genarg
open Ppconstr
open Printer
-let pr_firstorder_using_raw _ _ _ = prlist_with_sep pr_comma pr_reference
-let pr_firstorder_using_glob _ _ _ = prlist_with_sep pr_comma (pr_or_var (fun x -> (pr_global (snd x))))
-let pr_firstorder_using_typed _ _ _ = prlist_with_sep pr_comma pr_global
+let pr_firstorder_using_raw _ _ _ l = str "using " ++ prlist_with_sep pr_comma pr_reference l
+let pr_firstorder_using_glob _ _ _ l = str "using " ++ prlist_with_sep pr_comma (pr_or_var (fun x -> (pr_global (snd x)))) l
+let pr_firstorder_using_typed _ _ _ l = str "using " ++ prlist_with_sep pr_comma pr_global l
ARGUMENT EXTEND firstorder_using
PRINTED BY pr_firstorder_using_typed
diff --git a/printing/ppconstr.ml b/printing/ppconstr.ml
index b38cfa664..fb40e90d3 100644
--- a/printing/ppconstr.ml
+++ b/printing/ppconstr.ml
@@ -451,7 +451,7 @@ let pr pr sep inherited a =
lfix
| CProdN _ ->
let (bl,a) = extract_prod_binders a in
- hov 2 (
+ hov 0 (
hov 2 (pr_delimited_binders pr_forall spc
(pr mt ltop) bl) ++
str "," ++ pr spc ltop a),
diff --git a/printing/pptactic.ml b/printing/pptactic.ml
index 42a7e894a..02a21ced6 100644
--- a/printing/pptactic.ml
+++ b/printing/pptactic.ml
@@ -420,8 +420,9 @@ let pr_in_hyp_as pr_id = function
pr_in (spc () ++ pr_clear_flag clear pr_id id) ++ pr_as_ipat ipat
let pr_clauses default_is_concl pr_id = function
- | { onhyps=Some []; concl_occs=AllOccurrences }
- when (match default_is_concl with Some true -> true | _ -> false) -> mt ()
+ | { onhyps=Some []; concl_occs=occs }
+ when (match default_is_concl with Some true -> true | _ -> false) ->
+ pr_with_occurrences mt (occs,())
| { onhyps=None; concl_occs=AllOccurrences }
when (match default_is_concl with Some false -> true | _ -> false) -> mt ()
| { onhyps=None; concl_occs=NoOccurrences } ->
@@ -706,8 +707,8 @@ and pr_atom1 = function
hov 1 (str "pose" ++ pr_pose pr_constr pr_lconstr na c)
| TacLetTac (na,c,cl,b,e) ->
hov 1 ((if b then str "set" else str "remember") ++
- (if b then pr_pose pr_lconstr else pr_pose_as_style)
- pr_constr na c ++
+ (if b then pr_pose pr_constr pr_lconstr na c
+ else pr_pose_as_style pr_constr na c) ++
pr_opt (fun p -> pr_eqn_ipat p ++ spc ()) e ++
pr_clauses (Some b) pr_ident cl)
(* | TacInstantiate (n,c,ConclLocation ()) ->
@@ -853,7 +854,7 @@ let rec pr_tac inherited tac =
lfun
| TacThens (t,tl) ->
hov 1 (pr_tac (lseq,E) t ++ pr_then () ++ spc () ++
- pr_seq_body (pr_tac ltop) tl),
+ pr_seq_body (pr_opt_tactic (pr_tac ltop)) tl),
lseq
| TacThen (t1,t2) ->
hov 1 (pr_tac (lseq,E) t1 ++ pr_then () ++ spc () ++
diff --git a/printing/ppvernac.ml b/printing/ppvernac.ml
index d01e6a028..666c0c6d3 100644
--- a/printing/ppvernac.ml
+++ b/printing/ppvernac.ml
@@ -130,7 +130,7 @@ let pr_search a b pr_p = match a with
| SearchRewrite c -> str"SearchRewrite" ++ spc() ++ pr_p c ++ pr_in_out_modules b
| SearchAbout sl -> str"Search" ++ spc() ++ prlist_with_sep spc pr_search_about sl ++ pr_in_out_modules b
-let pr_locality local = if local then str "Local" ++ spc () else mt ()
+let pr_locality local = if local then str "Local " else mt ()
let pr_explanation (e,b,f) =
let a = match e with
diff --git a/theories/Relations/Operators_Properties.v b/theories/Relations/Operators_Properties.v
index c2cd9628b..cf1aa9baf 100644
--- a/theories/Relations/Operators_Properties.v
+++ b/theories/Relations/Operators_Properties.v
@@ -35,7 +35,8 @@ Section Properties.
Section Clos_Refl_Trans.
- Local Notation "R *" := (clos_refl_trans R) (at level 8, left associativity).
+ Local Notation "R *" := (clos_refl_trans R)
+ (at level 8, left associativity, format "R *").
(** Correctness of the reflexive-transitive closure operator *)