]> matita.cs.unibo.it Git - helm.git/blobdiff - helm/software/matita/library/nat/pi_p.ma
garbage removed
[helm.git] / helm / software / matita / library / nat / pi_p.ma
index e649f5f193ecdda0b0d9e7fc0c54b0d7355a233c..93f127372410610e5147fe02c5bf3fa59a08b2c7 100644 (file)
@@ -12,8 +12,6 @@
 (*                                                                        *)
 (**************************************************************************)
 
-set "baseuri" "cic:/matita/nat/pi_p".
-
 include "nat/primes.ma".
 (* include "nat/ord.ma". *)
 include "nat/generic_iter_p.ma".
@@ -257,6 +255,35 @@ elim n
   ]
 qed.
 
+theorem exp_sigma_p1: \forall n,a,p,f. 
+pi_p n p (\lambda x.(exp a (f x))) = (exp a (sigma_p n p f)).
+intros.
+elim n
+  [reflexivity
+  |apply (bool_elim ? (p n1))
+    [intro.
+     rewrite > true_to_pi_p_Sn
+      [rewrite > true_to_sigma_p_Sn
+        [simplify.
+         rewrite > H.
+         rewrite > exp_plus_times.
+         reflexivity.
+        |assumption
+        ]
+      |assumption
+      ]
+    |intro.
+     rewrite > false_to_pi_p_Sn
+      [rewrite > false_to_sigma_p_Sn
+        [simplify.assumption
+        |assumption
+        ]
+      |assumption
+      ]
+    ]
+  ]
+qed.
+
 theorem times_pi_p: \forall n,p,f,g. 
 pi_p n p (\lambda x.f x*g x) = pi_p n p f * pi_p n p  g. 
 intros.