]> matita.cs.unibo.it Git - helm.git/blobdiff - helm/software/matita/library/nat/euler_theorem.ma
...
[helm.git] / helm / software / matita / library / nat / euler_theorem.ma
index ab7d8242e1e5752573c61e187807a4aeeecfdbab..9396d444ed4b5a93db0e074e200c451f082cf5aa 100644 (file)
@@ -12,8 +12,6 @@
 (*                                                                        *)
 (**************************************************************************)
 
-set "baseuri" "cic:/matita/nat/euler_theorem".
-
 include "nat/map_iter_p.ma".
 include "nat/totient.ma".
 
@@ -55,7 +53,6 @@ intro.apply (nat_case n)
 qed.
 *)
 
-
 (*this obvious property is useful because simplify, sometimes,
   "simplifies too much", and doesn't allow to obtain this simple result.
  *)
@@ -136,7 +133,6 @@ elim (m)
 ]
 qed.
   
-
 lemma totient_card: \forall n.
 totient n = card n (\lambda i.eqb (gcd i n) (S O)).
 intros.