coq-club AT inria.fr
Subject: The Coq mailing list
List archive
- From: Cody Roux <cody.roux AT andrew.cmu.edu>
- To: coq-club AT inria.fr
- Subject: Re: [Coq-Club] coercing equality proofs
- Date: Tue, 28 Jan 2014 17:17:30 -0500
Of course, prop_ext in inconsistent with the current version of Coq, so this proof shouldn't come as a surprise... :) On 01/28/2014 04:51 PM, Jason Gross wrote: You don't even need bracket types if you have
prop_ext:
Axiom prop_ext: forall (p q : Prop), (p <-> q)
-> p = q.
Goal forall (a b : Prop), @eq Type a b -> @eq Prop a
b.
Proof.
intros a b H.
apply prop_ext.
split; destruct H; apply id.
Defined.
On Tue, Jan 28, 2014 at 4:45 PM, Jeremy
Avigad <avigad AT cmu.edu>
wrote:
It should be possible to do using the "bracket type" projection Type -> Prop but I am not sure how exactly it works in Coq since I do not use Prop. (Sorry for the lousy proof scripts. I have been away from Coq for a while.) Best wishes, Jeremy ********************** Axiom prop_ext: forall (p q : Prop), (p <-> q) -> p = q. Section Test. Variables a b : Prop. Variable p : @eq Type a b. Definition bracket (A : Type) : Prop := forall (P : Prop), (A -> P) -> P. Lemma bracket_eq (x : Prop): bracket x = x. apply prop_ext. split. intro H. apply (H x). intro H1. apply H1. intros H P H1. apply (H1 H). Qed. Lemma coerce: @eq Prop a b. transitivity (bracket a). symmetry. apply bracket_eq. transitivity (bracket b). rewrite p. reflexivity. apply bracket_eq. Qed. End Test. On 01/28/2014 03:50 PM, Vladimir Voevodsky wrote:
It should be possible to do using the "bracket type" projection Type -> Prop but I am not sure how exactly it works in Coq since I do not use Prop. |
- [Coq-Club] coercing equality proofs, Leonardo de Moura, 01/28/2014
- Re: [Coq-Club] coercing equality proofs, Jason Gross, 01/28/2014
- Re: [Coq-Club] coercing equality proofs, Vladimir Voevodsky, 01/28/2014
- Re: [Coq-Club] coercing equality proofs, Jeremy Avigad, 01/28/2014
- Re: [Coq-Club] coercing equality proofs, Jason Gross, 01/28/2014
- Re: [Coq-Club] coercing equality proofs, Cody Roux, 01/28/2014
- Re: [Coq-Club] coercing equality proofs, Jason Gross, 01/28/2014
- Re: [Coq-Club] coercing equality proofs, Cody Roux, 01/28/2014
- Re: [Coq-Club] coercing equality proofs, Jason Gross, 01/28/2014
- Re: [Coq-Club] coercing equality proofs, Cody Roux, 01/28/2014
- Re: [Coq-Club] coercing equality proofs, Vladimir Voevodsky, 01/28/2014
- Re: [Coq-Club] coercing equality proofs, Bas Spitters, 01/29/2014
- Re: [Coq-Club] coercing equality proofs, Arnaud Spiwack, 01/29/2014
- Re: [Coq-Club] coercing equality proofs, Jason Gross, 01/28/2014
- Re: [Coq-Club] coercing equality proofs, Jason Gross, 01/28/2014
- Re: [Coq-Club] coercing equality proofs, Jeremy Avigad, 01/28/2014
- Re: [Coq-Club] coercing equality proofs, Vladimir Voevodsky, 01/28/2014
- Re: [Coq-Club] coercing equality proofs, Jason Gross, 01/28/2014
Archive powered by MHonArc 2.6.18.