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: variable n unbound. (using [transparent assert]) #126

Open RobertoZunino opened 9 years ago

RobertoZunino commented 9 years ago
Require Import HoTT.

Goal True.
Proof.
assert {m:nat & True} as n.
exists 0.
exact tt.

transparent assert (H: True).
destruct n.
(* Anomaly: variable n unbound. Please report. *)

Using assert instead works fine.