summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/4035.v
blob: ec246d097ba90856dea6f4dfe4154107e9851ef5 (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
(* Supporting tactic notations within Ltac in the presence of an
  "ident" entry which does not expect a fresh ident *)
(* Of course, this is a matter of convention of what "ident" is
   supposed to denote, but in practice, it seems more convenient to
   have less constraints on ident at interpretation time, as
   otherwise more ad hoc entries would be necessary (as e.g. a special
   "quantified_hypothesis" entry for dependent destruction). *)
Require Import Program.
Goal nat -> Type.
  intro x.
  lazymatch goal with
  | [ x : nat |- _ ] => dependent destruction x
  end.