coq-club AT inria.fr
Subject: The Coq mailing list
List archive
- From: Robert Dockins <robdockins AT fastmail.fm>
- To: coq-club AT inria.fr
- Subject: Re: [Coq-Club] problem with tactic-generated terms
- Date: Fri, 12 Sep 2014 16:59:25 -0700
On Sep 12, 2014, at 3:19 PM, Jonathan
<jonikelee AT gmail.com>
wrote:
> On 09/12/2014 06:10 PM, Adam Chlipala wrote:
>> On 09/12/2014 06:04 PM, Jonathan wrote:
>>> Inductive Erasable(A : Type) : Prop :=
>>> erasable: A -> Erasable A.
>>>
>>> Arguments erasable [A] _.
>>>
>>> Axiom Erasable_inj : forall {A : Type}{a b : A}, erasable a=erasable
>>> b -> a=b.
>>
>> We did the same thing in Ynot, and I think this axiom turned out to be
>> inconsistent, period. You don't need to assume any others to run into
>> trouble. I don't remember the details of the proof, though.
>
> Wow - really? Does anyone remember those details?
You can get this from the Hurkens paradox; see below.
Cheers,
Rob
--------------------------------------
Require Hurkens.
Inductive Erasable(A : Type) : Prop := erasable: A -> Erasable A.
Arguments erasable [A] _.
Axiom Erasable_inj : forall {A : Type}{a b : A}, erasable a=erasable b -> a=b.
Definition er_out (X:Erasable Prop) : Prop
:= exists P, X = @erasable Prop P /\ P.
Theorem inconsistent : False.
Proof.
apply (Hurkens.paradox (Erasable Prop) (@erasable Prop) er_out).
intros.
destruct H as [P [H1 H2]].
apply Erasable_inj in H1.
subst A. trivial.
red; intros.
exists A; split; auto.
Qed.
Check inconsistent.
Print Assumptions inconsistent.
- Re: [Coq-Club] problem with tactic-generated terms, (continued)
- Re: [Coq-Club] problem with tactic-generated terms, Adam Chlipala, 09/12/2014
- Re: [Coq-Club] problem with tactic-generated terms, Jonathan, 09/12/2014
- Re: [Coq-Club] problem with tactic-generated terms, Ömer Sinan Ağacan, 09/12/2014
- Re: [Coq-Club] problem with tactic-generated terms, Jonathan, 09/12/2014
- Re: [Coq-Club] problem with tactic-generated terms, Daniel Schepler, 09/12/2014
- Re: [Coq-Club] problem with tactic-generated terms, Greg Morrisett, 09/12/2014
- Re: [Coq-Club] problem with tactic-generated terms, Jonathan, 09/13/2014
- Re: [Coq-Club] problem with tactic-generated terms, Adam Chlipala, 09/13/2014
- Re: [Coq-Club] problem with tactic-generated terms, Jonathan, 09/13/2014
- Re: [Coq-Club] problem with tactic-generated terms, Matthieu Sozeau, 09/13/2014
- Re: [Coq-Club] problem with tactic-generated terms, Robert Dockins, 09/13/2014
- Re: [Coq-Club] problem with tactic-generated terms, Jonathan, 09/13/2014
- Re: [Coq-Club] problem with tactic-generated terms, Matthieu Sozeau, 09/13/2014
- Re: [Coq-Club] problem with tactic-generated terms, Daniel Schepler, 09/13/2014
- Re: [Coq-Club] problem with tactic-generated terms, Hugo Herbelin, 09/13/2014
- Re: [Coq-Club] problem with tactic-generated terms, Jonathan, 09/14/2014
- Re: [Coq-Club] problem with tactic-generated terms, Hugo Herbelin, 09/15/2014
- Re: [Coq-Club] problem with tactic-generated terms, Jonathan, 09/15/2014
- Re: [Coq-Club] problem with tactic-generated terms, Hugo Herbelin, 09/15/2014
- Re: [Coq-Club] problem with tactic-generated terms, Jonathan, 09/13/2014
- Re: [Coq-Club] problem with tactic-generated terms, Greg Morrisett, 09/12/2014
- Re: [Coq-Club] problem with tactic-generated terms, Daniel Schepler, 09/12/2014
- Re: [Coq-Club] problem with tactic-generated terms, Jonathan, 09/12/2014
- Re: [Coq-Club] problem with tactic-generated terms, Ömer Sinan Ağacan, 09/12/2014
- Re: [Coq-Club] problem with tactic-generated terms, Jonathan, 09/13/2014
- Re: [Coq-Club] problem with tactic-generated terms, Daniel Schepler, 09/13/2014
Archive powered by MHonArc 2.6.18.