]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/library/nat/euler_theorem.ma
Towards chebyshev.
[helm.git] / matita / library / nat / euler_theorem.ma
index ab7d8242e1e5752573c61e187807a4aeeecfdbab..1e5988b35de64d1a9eba560dadd53e6929e98f15 100644 (file)
@@ -55,7 +55,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 +135,6 @@ elim (m)
 ]
 qed.
   
-
 lemma totient_card: \forall n.
 totient n = card n (\lambda i.eqb (gcd i n) (S O)).
 intros.