coq-club AT inria.fr
Subject: The Coq mailing list
List archive
- From: Hugo Herbelin <Hugo.Herbelin AT inria.fr>
- To: Jonathan <jonikelee AT gmail.com>
- Cc: coq-club AT inria.fr
- Subject: Re: [Coq-Club] problem with tactic-generated terms
- Date: Sat, 13 Sep 2014 17:59:04 +0200
Hi,
On Fri, Sep 12, 2014 at 09:41:12PM -0400, Jonathan wrote:
> On 09/12/2014 07:59 PM, Robert Dockins wrote:
> >
> >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.
> >
>
> I needed to add Import Hurkens.NoRetractFromSmallPropositionToProp.
> and use "paradox" unqualified, for some reason - but otherwise it
> does work (I'm using a trunk version). Are things just as bad if I
> limit Erasable to be over Set instead of Type?
In the Set-impredicative version of the Calculus of Inductive
Constructions, you can (relevantly) interpret Prop as impredicative
Set and define an injective erasable over types in Set. Up to
impredicativity that Prop has but Type not, this is Matthieu's claim
that there is a proof-relevant model of Erasable (with its restriction
to Set needed).
Hugo Herbelin
- Re: [Coq-Club] problem with tactic-generated terms, (continued)
- 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/13/2014
- Re: [Coq-Club] problem with tactic-generated terms, Daniel Schepler, 09/13/2014
- Re: [Coq-Club] problem with tactic-generated terms, Daniel Schepler, 09/13/2014
Archive powered by MHonArc 2.6.18.