Require Import ssreflect.
Axiom odd : nat -> Prop.
Lemma simple :
forall x, 3 <= x -> forall y, odd (y+x) -> x = y -> True.
Proof.
move=> >x_ge_3 >xy_odd.
lazymatch goal with
| |- ?x = ?y -> True => done
end.
Qed.
Lemma simple2 :
forall x, 3 <= x -> forall y, odd (y+x) -> x = y -> True.
Proof.
move=> >; move=>x_ge_3; move=> >; move=>xy_odd.
lazymatch goal with
| |- ?x = ?y -> True => done
end.
Qed.
Definition stuff x := 3 <= x -> forall y, odd (y+x) -> x = y -> True.
Lemma harder : forall x, stuff x.
Proof.
move=> >x_ge_3 >xy_odd.
lazymatch goal with
| |- ?x = ?y -> True => done
end.
Qed.
Lemma harder2 : forall x, stuff x.
Proof.
move=> >; move=>x_ge_3;move=> >; move=>xy_odd.
lazymatch goal with
| |- ?x = ?y -> True => done
end.
Qed.
Lemma homotop : forall x : nat, forall e : x = x, e = e -> True.
Proof.
move=> >eq_ee.
lazymatch goal with
| |- True => done
end.
Qed.
¤ Dauer der Verarbeitung: 0.0 Sekunden
(vorverarbeitet)
¤
|
Haftungshinweis
Die Informationen auf dieser Webseite wurden
nach bestem Wissen sorgfältig zusammengestellt. Es wird jedoch weder Vollständigkeit, noch Richtigkeit,
noch Qualität der bereit gestellten Informationen zugesichert.
Bemerkung:
Die farbliche Syntaxdarstellung ist noch experimentell.
|