aboutsummaryrefslogtreecommitdiff
path: root/test-suite/bugs/opened/bug_3370.v
blob: d6fc88a03a6d66a545d427eae0de5bcd127551dd (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
Require Import String.

Local Ltac set_strings :=
  let s := match goal with |- context[String ?s1 ?s2] => constr:(String s1 s2) end in
  let H := fresh s in
  set (H := s).

Local Open Scope string_scope.

Goal "asdf" = "bds".
Fail set_strings. (* Error: Ltac variable s is bound to "asdf" which cannot be coerced to
a fresh identifier. *)
Abort.