HoTT / coq

Coq is a formal proof management system. It provides a formal language to write mathematical definitions, executable algorithms and theorems together with an environment for semi-interactive development of machine-checked proofs.
http://coq.inria.fr/
GNU Lesser General Public License v2.1
27 stars 5 forks source link

Primitive projections should be valid targets of coercions (polyproj) #81

Closed JasonGross closed 10 years ago

JasonGross commented 10 years ago
Set Primitive Projections.
Set Implicit Arguments.
Set Universe Polymorphism.

Record category :=
  { ob :> Type;
    hom : ob -> ob -> Type
  }.

Record foo := { C : category; x : ob C; y :> hom x x }.
(* Toplevel input, characters 20-75:
Error: Cannot find the target class. *)
mattam82 commented 10 years ago

Fixed in trunk