coq-club AT inria.fr
Subject: The Coq mailing list
List archive
- From: Lionel Elie Mamane <lionel AT mamane.lu>
- To: coq-club AT pauillac.inria.fr
- Subject: [Coq-Club] Anomaly: Evar was not declared.
- Date: Thu, 1 Sep 2005 16:04:49 +0200
- List-archive: <http://pauillac.inria.fr/pipermail/coq-club/>
Hi,
Given this code:
Definition twopower: nat -> nat.
Admitted.
Definition log2': forall x:nat, {y:nat | twopower y <= x < twopower
(y+1)}+{x=0}.
intros.
case x.
right; apply (refl_equal 0).
clear x; intros Px.
set (x:=(S Px)).
left.
refine (exist _ ((fix lg (n:nat) {struct n}:nat:= _ ) _) _).
I get at this refine an anomaly:
Anomaly: Evar ?13 was not declared. Please report.
So I report it "par la présente".
Have fun,
--
Lionel
- [Coq-Club] Anomaly: Evar was not declared., Lionel Elie Mamane
- <Possible follow-ups>
- [Coq-Club] Anomaly: Evar was not declared., Lionel Elie Mamane
Archive powered by MhonArc 2.6.16.