aboutsummaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/bug_12529.v
blob: bc3c9a28bd79576caeff4b0c2d60417ffa74dd6a (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
Goal SProp.
match goal with |- SProp => idtac end.
Fail match goal with |- Prop => idtac end.
Abort.

Goal Prop.
Fail match goal with |- SProp => idtac end.
match goal with |- Prop => idtac end.
Abort.

Class F A := f : A.

Inductive pFalse : Prop  := .
Inductive sFalse : SProp := .

Hint Extern 0 (F Prop) => exact pFalse : typeclass_instances.
Definition pf := f : Prop.

Hint Extern 0 (F SProp) => exact sFalse : typeclass_instances.
Definition sf := (f : SProp).
Definition pf' := (f : Prop).