blob: 08bf62493da0e3cf2dfe806c1ac2c9d37e682d59 (
plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
|
Axiom P : nat -> Prop.
Axiom admit : forall n : nat, P n -> P n -> n = S n.
Axiom foo : forall n, P n.
Create HintDb bar.
Hint Extern 3 => symmetry : bar.
Hint Resolve admit : bar.
Hint Immediate foo : bar.
Lemma qux : forall n : nat, n = S n.
Proof.
intros n.
eauto with bar.
Defined.
Goal True.
pose (e := eq_refl (qux 0)); unfold qux in e.
match type of e with context [eq_sym] => fail 1 | _ => idtac end.
|