Skip to content

Instantly share code, notes, and snippets.

@KeenS
Created April 13, 2014 16:10
Show Gist options
  • Save KeenS/10590357 to your computer and use it in GitHub Desktop.
Save KeenS/10590357 to your computer and use it in GitHub Desktop.
Goal forall P Q : nat -> Prop, P 0 -> (forall x , P x -> Q x) -> Q 0.
Proof.
intros.
apply H0.
apply H.
Qed.
Goal forall P : nat -> Prop, P 2 -> (exists y, P (1 + y)).
Proof.
intros.
exists 1.
apply H.
Qed.
Goal forall P : nat -> Prop, (forall n m, P n -> P m) -> (exists p, P p) -> forall q, P q.
Proof.
intros.
destruct H0.
apply (H x q).
apply H0.
Qed.
Sign up for free to join this conversation on GitHub. Already have an account? Sign in to comment