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

"Unable to handle arbitrary u+k <= v constraints" should probably be an Error, not an Anomaly (polyproj) #114

Open JasonGross opened 10 years ago

JasonGross commented 10 years ago
Inductive test : $(let U := type of Type in exact U)$ := t.
(* Anomaly: Unable to handle arbitrary u+k <= v constraints. Please report. *)