aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/hintdb_in_ltac_bis.v
blob: f5c25540effd22e8d00ccc5d8ed9c568dd6fa27b (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
Parameter Foo : Prop.
Axiom H : Foo.

Hint Resolve H : mybase.

Ltac foo base := eauto with base.

Tactic Notation "bar" ident(base) :=
  typeclasses eauto with base.

Goal Foo.
  progress foo mybase.
  Undo.
  progress bar mybase.
Qed.