coq-club AT inria.fr
Subject: The Coq mailing list
List archive
- From: Chad E Brown <cebrown2323 AT yahoo.com>
- To: coq-club AT inria.fr
- Subject: Re: [Coq-Club] An axiom about parametricity
- Date: Wed, 22 Sep 2010 08:52:25 -0700 (PDT)
- Domainkey-signature: a=rsa-sha1; q=dns; c=nofws; s=s1024; d=yahoo.com; h=Message-ID:X-YMail-OSG:Received:X-Mailer:References:Date:From:Subject:To:In-Reply-To:MIME-Version:Content-Type; b=tGRPeQr4s8LVB2ZEIejSAI/W4Yb7uMpg4gQWjcFAhJr74Q5AolkAQq8yfCQvTyfqZIkX/N25IQjCqf2XhZtsUfhUI1SBiJESxzvLnFF4q5vTPZvsWqL0gRXdKKVRocTSXl3RADPGGgqPJsrTtvVzGuQ8X10qJaetqu40fnPwPqc=;
Hi Xinyu, and all,
The axiom as you gave it is inconsistent with Coq. A proof is below. Maybe you meant something else?
Axiom pa : forall (F : Type -> Type) (f g : forall t, F t) (t : Type), f t = g t -> f = g.
Definition f_ (X : Type) : Type := X -> False.
Definition g_ (X : Type) : Type := False -> X.
Goal False.
cut (f_ = g_). intros e.
cut (g_ True). rewrite <- e. auto.
unfold g_. auto.
apply (pa (fun X => Type) f_ g_ False).
auto.
Qed.
- Chad
From: Xinyu Jiang <xj27 AT pantheon.yale.edu>
To: coq-club AT inria.fr
Sent: Wed, September 22, 2010 4:22:11 PM
Subject: [Coq-Club] An axiom about parametricity
The axiom as you gave it is inconsistent with Coq. A proof is below. Maybe you meant something else?
Axiom pa : forall (F : Type -> Type) (f g : forall t, F t) (t : Type), f t = g t -> f = g.
Definition f_ (X : Type) : Type := X -> False.
Definition g_ (X : Type) : Type := False -> X.
Goal False.
cut (f_ = g_). intros e.
cut (g_ True). rewrite <- e. auto.
unfold g_. auto.
apply (pa (fun X => Type) f_ g_ False).
auto.
Qed.
- Chad
From: Xinyu Jiang <xj27 AT pantheon.yale.edu>
To: coq-club AT inria.fr
Sent: Wed, September 22, 2010 4:22:11 PM
Subject: [Coq-Club] An axiom about parametricity
Hi all,
I would like to add an axiom somehow like:
"forall (F : Type -> Type) (f g : forall t, F t) (t : Type), f t = g t -> f = g"
to Coq. It seems to be reasonable because of the parametricity of Coq's logic. But I wonder if the axiom is indeed consistent with Coq.
If so, would it collide against other axioms like exclusive of the middle? If not, what would the counter example be like? Thanks very much.
I would like to add an axiom somehow like:
"forall (F : Type -> Type) (f g : forall t, F t) (t : Type), f t = g t -> f = g"
to Coq. It seems to be reasonable because of the parametricity of Coq's logic. But I wonder if the axiom is indeed consistent with Coq.
If so, would it collide against other axioms like exclusive of the middle? If not, what would the counter example be like? Thanks very much.
- [Coq-Club] An axiom about parametricity, Xinyu Jiang
- Message not available
- Message not available
- [Coq-Club] An axiom about parametricity,
Xinyu Jiang
- Re: [Coq-Club] An axiom about parametricity, Chad E Brown
- Re: [Coq-Club] An axiom about parametricity, AUGER Cedric
- Message not available
- Re: [Coq-Club] An axiom about parametricity,
Bruno Barras
- Re: [Coq-Club] An axiom about parametricity, Thorsten Altenkirch
- Re: [Coq-Club] An axiom about parametricity,
Bruno Barras
- [Coq-Club] An axiom about parametricity,
Xinyu Jiang
- Message not available
- Message not available
- Message not available
- Message not available
- Re: [Coq-Club] An axiom about parametricity, Arthur Charguéraud
- Message not available
- Message not available
- Re: [Coq-Club] An axiom about parametricity,
Taral
- Re: [Coq-Club] An axiom about parametricity, Thorsten Altenkirch
- <Possible follow-ups>
- Re: [Coq-Club] An axiom about parametricity, xinyu . jiang
- Message not available
Archive powered by MhonArc 2.6.16.