coq-club AT inria.fr
Subject: The Coq mailing list
List archive
- From: Edsko de Vries <devriese AT cs.tcd.ie>
- To: coq-club AT pauillac.inria.fr
- Subject: [Coq-Club] Question about equality
- Date: Sat, 21 Mar 2009 09:20:28 +0000
- List-archive: <http://pauillac.inria.fr/pipermail/coq-club/>
Hi,
I am stuck in a proof with lots of JMeqs. I've tried to make a minimal example
that shows the problem; hopefully it's not too minimal. The question is
simple:
how can I complete the following proof??
Require Import JMeq.
Section test.
Variables A B : Set.
Variables (a : A) (b : B).
Hypothesis a_equals_b : JMeq a b.
Definition t (cond : bool) : Set :=
match cond with
| true => A -> A
| false => B -> B
end.
Variable f : forall (cond : bool), t cond.
Lemma foo :
JMeq (f true a) (f false b).
Proof.
Any help is greatly appreciated!
Edsko
- [Coq-Club] Question about equality, Edsko de Vries
- Re: [Coq-Club] Question about equality,
André Hirschowitz
- Re: [Coq-Club] Question about equality, Edsko de Vries
- Re: [Coq-Club] Question about equality, Edsko de Vries
- Re: [Coq-Club] Question about equality,
André Hirschowitz
Archive powered by MhonArc 2.6.16.