summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/4603.v
blob: 2c90044dc77c8fd7bb7bedd8522d299109cea591 (plain)
1
2
3
4
5
6
7
8
9
10
Axiom A : Type.

Goal True. exact I.
Check (fun P => P A).
Abort.

Goal True.
Definition foo (A : Type) : Prop:= True. 
  set (x:=foo). split.
Qed.