Skip to Content.
Sympa Menu

coq-club - Re: [Coq-Club] Question about equality

coq-club AT inria.fr

Subject: The Coq mailing list

List archive

Re: [Coq-Club] Question about equality


chronological Thread 
  • From: Andr� Hirschowitz <ah AT unice.fr>
  • To: Edsko de Vries <devriese AT cs.tcd.ie>
  • Cc: coq-club AT pauillac.inria.fr
  • Subject: Re: [Coq-Club] Question about equality
  • Date: Sat, 21 Mar 2009 10:36:07 +0100
  • List-archive: <http://pauillac.inria.fr/pipermail/coq-club/>
  • Organization: UNS

Hello,

My first impression is that you cannot:
Take A:=B = bool.
a=b=true
and
f (true) =Id, f(false) = -Id
Probably you oversimplified your problem?

ah
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

--------------------------------------------------------
Bug reports: http://logical.saclay.inria.fr/coq-bugs
Archives: http://pauillac.inria.fr/pipermail/coq-club
          http://pauillac.inria.fr/bin/wilma/coq-club
Info: http://pauillac.inria.fr/mailman/listinfo/coq-club





Archive powered by MhonArc 2.6.16.

Top of Page