X-Git-Url: http://matita.cs.unibo.it/gitweb/?a=blobdiff_plain;f=matita%2Fmatita%2Flib%2Farithmetics%2Fbinomial.ma;h=7ab00d4991c23408fc1dc76ec149a4d7f80c86a2;hb=ddc80515997a3f56085c6234d4db326141e189aa;hp=c31e15d112ea510955481ef32e059a7c5584cc83;hpb=fc7af5f9ea2cd4a876b8babc6b691136799e3c87;p=helm.git diff --git a/matita/matita/lib/arithmetics/binomial.ma b/matita/matita/lib/arithmetics/binomial.ma index c31e15d11..7ab00d499 100644 --- a/matita/matita/lib/arithmetics/binomial.ma +++ b/matita/matita/lib/arithmetics/binomial.ma @@ -44,12 +44,12 @@ theorem bc2 : ∀n. cut (m-(m-(S c)) = S c) [@plus_to_minus @plus_minus_m_m //] #eqSc lapply (Hind c (le_S_S_to_le … lec)) #Hc lapply (Hind (m - (S c)) ?) [@le_plus_to_minus //] >eqSc #Hmc - >(plus_minus_m_m m c) in ⊢ (??(??(?%))) [|@le_S_S_to_le //] + >(plus_minus_m_m m c) {⊢ (??(??(?%)))} [|@le_S_S_to_le //] >commutative_plus >(distributive_times_plus ? (S c)) @divides_plus [>associative_times >(commutative_times (S c)) commutative_times @Hmc ] @@ -61,18 +61,18 @@ qed. theorem bc1: ∀n.∀k. k < n → bc (S n) (S k) = (bc n k) + (bc n (S k)). #n #k #ltkn > bceq >(bceq n) >(bceq n (S k)) ->(div_times_times ?? (S k)) in ⊢ (???(?%?)) +>(div_times_times ?? (S k)) {⊢ (???(?%?))} [|>(times_n_O 0) @lt_times // | //] ->associative_times in ⊢ (???(?(??%)?)) ->commutative_times in ⊢ (???(?(??(??%))?)) -(div_times_times ?? (n - k)) in ⊢ (???(??%)) +>associative_times {⊢ (???(?(??%)?))} +>commutative_times {⊢ (???(?(??(??%))?))} +(div_times_times ?? (n - k)) {⊢ (???(??%))} [|>(times_n_O 0) @lt_times // |@(le_plus_to_le_r k ??) associative_times in ⊢ (???(??(??%))) +>associative_times {⊢ (???(??(??%)))} >fact_minus // commutative_plus in ⊢ (???%) commutative_plus {⊢ (???%)} associative_times >(commutative_times (S k))