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

Anomaly: unknown meta ?190. Please report. (HoTT/coq) #117

Closed JasonGross closed 10 years ago

JasonGross commented 10 years ago
(* File reduced by coq-bug-finder from original input, then from 1461 lines to 81 lines, then from 84 lines to 40 lines, then from 50\
 lines to 24 lines *)

Inductive paths {A : Type} (a : A) : A -> Type :=
  idpath : paths a a.
Notation "x = y :> A" := (@paths A x y) : type_scope.
Notation "x = y" := (x = y :>_) : type_scope.
Class Contr_internal (A : Type) := BuildContr {
  center : A ;
  contr : (forall y : A, center = y)
}.
Class Funext := {}.

Definition path_forall `{Funext} {A : Type} {P : A -> Type} (f g : forall x : A, P x) :
  (forall x, f x = g x) -> f = g.

Admitted.

Inductive Empty : Set := .
Instance contr_from_Empty {_ : Funext} (A : Type) :
  Contr_internal (Empty -> A) :=
  BuildContr _
             (Empty_rect (fun _ => A))
             (fun f => path_forall _ f (fun x => Empty_rect _ x)).
(* Toplevel input, characters 15-220:
Anomaly: unknown meta ?190. Please report. *)

This is a bug in HoTT/coq, but closed in trunk-polyproj, so I'll close it after I open it.