X-Git-Url: http://matita.cs.unibo.it/gitweb/?a=blobdiff_plain;f=helm%2Fsoftware%2Fmatita%2Ftests%2Fa.ma;h=e6dac496cecec0e8cabfab3e6c818274afd3c889;hb=2b3de2b59f301c65cbc9985b18a25f659743a76a;hp=1061544d0b5891ab04689722b1a3057c69673b1e;hpb=42f25c258b0b199ee96dd8eaa3d44c86eb6916ab;p=helm.git diff --git a/helm/software/matita/tests/a.ma b/helm/software/matita/tests/a.ma index 1061544d0..e6dac496c 100644 --- a/helm/software/matita/tests/a.ma +++ b/helm/software/matita/tests/a.ma @@ -18,13 +18,40 @@ axiom C : Prop. axiom a: A. axiom b: B. +definition xxx ≝ A. notation "#" non associative with precedence 90 for @{ 'sharp }. interpretation "a" 'sharp = a. -interpretation "b" 'sharp = b. +interpretation "b" 'sharp = b. -ntheorem prova : (A → B → C) → C. +definition k : A → A ≝ λx.a. +definition k1 : A → A ≝ λx.a. + +axiom P : A → Prop. + +include "nat/plus.ma". + +ntheorem pappo : ∀n:nat.n = S n + n → S n = (S (S n)). +#m; #H; napply (let pippo ≝ (S m) in ?); +nchange in match (S m) in ⊢ (?) with pippo; + +nletin pippo ≝ (S m) in H ⊢ (?); + +nwhd in H:(???%); +nchange in match (S ?) in H:% ⊢ (? → %) with (pred (S ?)); +ntaint; + +ngeneralize in match m in ⊢ %; in ⊢ (???% → ??%?); +STOP +ncases (O) in m : % (*H : (??%?)*) ⊢ (???%); +nelim (S m) in H : (??%?) ⊢ (???%); +STOP; + +ntheorem pippo : ∀x:A. P (k x). +nchange in match (k x) in ⊢ (∀_.%) with (k1 x); STOP + +ntheorem prova : (A → A → C) → C. napply (λH.?); -napply (H ? ?); +napply (H ? ?); nchange A xxx; napply #. nqed. \ No newline at end of file