aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2016-10-22 12:22:00 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2016-10-22 12:22:40 +0200
commit46462c3cc69e97bf3260f1aad5faaa6eaf6c2722 (patch)
tree67eeabc6becc6476c030c4060524c1fab1ae5320
parentc28a2a3a1297098ee73ad5b26e714164b6167d2b (diff)
parent80d5779409bf33fbe5043275b96775a5f04a3b2c (diff)
Merge branch 'v8.5' into v8.6
-rw-r--r--ltac/tacinterp.ml3
-rw-r--r--test-suite/output/ltac.out1
-rw-r--r--test-suite/output/ltac.v5
3 files changed, 9 insertions, 0 deletions
diff --git a/ltac/tacinterp.ml b/ltac/tacinterp.ml
index 08e67a0c2..52208979c 100644
--- a/ltac/tacinterp.ml
+++ b/ltac/tacinterp.ml
@@ -875,6 +875,9 @@ let rec message_of_value v =
Ftactic.return (pr_closed_glob_env (pf_env gl)
(project gl) c)
end }
+ else if has_type v (topwit wit_var) then
+ let id = out_gen (topwit wit_var) v in
+ Ftactic.nf_enter { enter = begin fun gl -> Ftactic.return (pr_id id) end }
else match Value.to_list v with
| Some l ->
Ftactic.List.map message_of_value l >>= fun l ->
diff --git a/test-suite/output/ltac.out b/test-suite/output/ltac.out
index f4254e4e2..a62f4312e 100644
--- a/test-suite/output/ltac.out
+++ b/test-suite/output/ltac.out
@@ -26,3 +26,4 @@ The command has indeed failed with message:
In nested Ltac calls to "h" and "injection (destruction_arg)", last call
failed.
Error: No primitive equality found.
+Hx
diff --git a/test-suite/output/ltac.v b/test-suite/output/ltac.v
index dfa60eeda..fb1dab799 100644
--- a/test-suite/output/ltac.v
+++ b/test-suite/output/ltac.v
@@ -43,3 +43,8 @@ Goal True -> False.
Fail h I.
intro H.
Fail h H.
+
+(* Check printing of the "var" argument "Hx" *)
+Ltac m H := idtac H; exact H.
+Goal True.
+let a:=constr:(let Hx := 0 in ltac:(m Hx)) in idtac.