coq-club AT inria.fr
Subject: The Coq mailing list
List archive
- From: Brian Huffman <brianh AT cs.pdx.edu>
- To: coq-club AT inria.fr
- Subject: Re: [Coq-Club] Prove inductive type implies false in cycle
- Date: Mon, 1 Aug 2011 21:07:32 -0700
On Mon, Aug 1, 2011 at 8:16 PM, S3
<scubed2 AT gmail.com>
wrote:
> Start with a simple definition for divides evenly:
[...]
> Inductive divides: nat -> nat -> Prop :=
> | divides_0 n: divides 0 n
> | divides_n n m: divides n m -> divides (n + m) m
> .
[...]
> But, how would I prove that:
> forall n, divides (S n) 0 -> False.
I managed to prove this by proving a related lemma first:
Lemma divides_zero :
forall n m, divides n m -> m = 0 -> n = 0.
Formulated this way, divides_zero can be proved by a straightforward
induction on the "divides" predicate.
Your original goal, "forall n, divides (S n) 0 -> False" can be
derived fairly directly from divides_zero.
- Brian
- [Coq-Club] Prove inductive type implies false in cycle, S3
- [Coq-Club] Prove inductive type implies false in cycle,
S3
- Re: [Coq-Club] Prove inductive type implies false in cycle, Brian Huffman
- Message not available
- Re: [Coq-Club] Prove inductive type implies false in cycle, Pierre Casteran
- Re: [Coq-Club] Prove inductive type implies false in cycle, AUGER Cedric
- [Coq-Club] Prove inductive type implies false in cycle,
S3
Archive powered by MhonArc 2.6.16.