]> matita.cs.unibo.it Git - helm.git/blobdiff - helm/software/matita/tests/a.ma
test/a.ma => tests/ng_tactics.ma, with nassert here and there
[helm.git] / helm / software / matita / tests / a.ma
diff --git a/helm/software/matita/tests/a.ma b/helm/software/matita/tests/a.ma
deleted file mode 100644 (file)
index e6dac49..0000000
+++ /dev/null
@@ -1,57 +0,0 @@
-(**************************************************************************)
-(*       ___                                                              *)
-(*      ||M||                                                             *)
-(*      ||A||       A project by Andrea Asperti                           *)
-(*      ||T||                                                             *)
-(*      ||I||       Developers:                                           *)
-(*      ||T||         The HELM team.                                      *)
-(*      ||A||         http://helm.cs.unibo.it                             *)
-(*      \   /                                                             *)
-(*       \ /        This file is distributed under the terms of the       *)
-(*        v         GNU General Public License Version 2                  *)
-(*                                                                        *)
-(**************************************************************************)
-
-axiom A : Prop.
-axiom B : Prop.
-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.
-
-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 ? ?); nchange A xxx; 
-napply #.
-nqed. 
\ No newline at end of file