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

Error: No such section variable or assumption: U' at section end (HoTT/coq) #116

Closed JasonGross closed 10 years ago

JasonGross commented 10 years ago
Set Universe Polymorphism.
Section foo.
  Let U := Type.
  Let U' : Type.
  Proof.
    let U' := constr:(Type) in
    let U_le_U' := constr:(fun x : U => (x : U')) in
    exact U'.
  Defined.
  Inductive t : U' := .
End foo.
(* Toplevel input, characters 15-23:
Error: No such section variable or assumption: U'. *)

This bug is closed in trunk-polyproj, so I'll close it immediately; I'm reporting it so I have a number to give the bug in my test-suite.