DEBSOURCES
Skip Quicknav
sources / coq-doc / 8.20.0-2 / test-suite / bugs / bug_4603.v
12345678910
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.