]> matita.cs.unibo.it Git - helm.git/blobdiff - helm/software/matita/tests/decl.ma
changed auto_tac params type and all derivate tactics like applyS and
[helm.git] / helm / software / matita / tests / decl.ma
index 4b67f551ab6821646c7bda52a445f646504916b4..569a2f8ffa12cf96d24d095c7062c294b26f7ec0 100644 (file)
@@ -12,7 +12,7 @@
 (*                                                                        *)
 (**************************************************************************)
 
-set "baseuri" "cic:/matita/tests/decl".
+
 
 include "nat/times.ma".
 include "nat/orders.ma".
@@ -114,11 +114,7 @@ theorem easy3: ∀A:Prop. (A ∧ ∃n:nat.n ≠ n) → True.
  assume P: Prop.
  suppose (P ∧ ∃m:nat.m ≠ m) (H).
  by H we have P (H1) and (∃x:nat.x≠x) (H2).
- (*BUG:
  by H2 let q:nat such that (q ≠ q) (Ineq).
- *)
- (* the next line is wrong, but for the moment it does the job *)
- by H2 let q:nat such that False (Ineq).
  by I done.
 qed.
 
@@ -129,9 +125,9 @@ assume p:nat.
 suppose (n=m) (H).
 suppose (S m = S p) (K).
 suppose (n = S p) (L).
-conclude (S n) = (S m) by (eq_f ? ? ? ? ? H).
+conclude (S n) = (S m) by H.
              = (S p) by K.
-             = n by (sym_eq ? ? ? L)
+             = n by L
 done.
 qed.
 
@@ -142,9 +138,9 @@ assume p:nat.
 suppose (n=m) (H).
 suppose (S m = S p) (K).
 suppose (n = S p) (L).
-conclude (S n) = (S m) by _.
-             = (S p) by _.
-             = n by _
+conclude (S n) = (S m).
+             = (S p).
+             = n
 done.
 qed.