summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/4603.v
blob: e7567623a6594b57423bb5368c1ae12e179dfeb9 (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.