aboutsummaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/bug_3326.v
blob: 1c126853530d758a22cdde2291ce07b120ebad01 (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
Class ORDER A := Order {
  LEQ : A -> A -> bool;
  leqRefl: forall x, true = LEQ x x
}.

Section XXX.

Variable A:Type.
Variable (O:ORDER A).
Definition aLeqRefl := @leqRefl _ O.

Lemma OK : forall x, true = LEQ x x.
Proof.
  intros.
  unfold LEQ.
  destruct O.
  clear.
  Fail apply aLeqRefl.
Abort.
End XXX.