GoalType*Type.Proof.split.par:exactType.Qed.GoalType.Proof.exactType.Qed.(* (* coqide test, note the delegated proofs seem to get an empty dirpath? or I got confused because I had lemma foo in file foo *)Definition U := Type.Lemma foo : U.Proof. exact Type.Qed.Lemma foo1 : Type.Proof. exact (U:Type).Qed.Print foo.*)