]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/contribs/lambdadelta/ground/arith/arith_2a.ma
update from master branch
[helm.git] / matita / matita / contribs / lambdadelta / ground / arith / arith_2a.ma
index b5ff26116ef36e2b41f8e3c4abd9a51fc374f45c..114eddb1e34837a19871dc0dffd802764e0abc54 100644 (file)
 (*                                                                        *)
 (**************************************************************************)
 
-include "ground/notation/functions/two_0.ma".
+include "ground/arith/pnat_two.ma".
 include "ground/arith/nat_le_minus_plus.ma".
 include "ground/arith/nat_lt.ma".
 
 (* ARITHMETICAL PROPERTIES FOR λδ-2A ****************************************)
 
-interpretation
-  "zero (non-negative integers)"
-  'Two = (ninj (psucc punit)).
-
 (* Equalities ***************************************************************)
 
 lemma plus_n_2: ∀n. (n + 𝟐) = n + 𝟏 + 𝟏.
 // qed.
 
 lemma arith_b1: ∀a,b,c1. c1 ≤ b → a - c1 - (b - c1) = a - b.
-#a #b #c1 #H >nminus_comm <nminus_assoc_comm_23 //
+#a #b #c1 #H >nminus_comm_21 <nminus_assoc_comm_23 //
 qed-.
 
 lemma arith_b2: ∀a,b,c1,c2. c1 + c2 ≤ b → a - c1 - c2 - (b - c1 - c2) = a - b.
@@ -87,7 +83,7 @@ lemma lt_plus_SO_to_le: ∀x,y. x < y + (𝟏) → x ≤ y.
 
 (* Iterators ****************************************************************)
 
-lemma iter_SO: ∀B:Type[0]. ∀f:B→B. ∀b,l. f^(l+𝟏) b = f (f^l b).
+lemma iter_SO: ∀B:Type[0]. ∀f:B→B. ∀b,l. (f^(l+𝟏)) b = f ((f^l) b).
 #B #f #b #l
 <niter_succ //
 qed.