]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/dama/reals.ma
Notation is finally fully working everywhere.
[helm.git] / matita / dama / reals.ma
index c03fdf26bf6c4d6ef3a6eefecb57f5bdc4f41116..87bbee5fd0d2e84de0a9e49d8ee066f4d826e8b8 100644 (file)
@@ -147,7 +147,7 @@ lemma technical1: ∀R:real.lim R (to_zero R) (is_cauchy_seq_to_zero R) = 0.
  elim daemon.
 qed.
  
-lemma abs_x_ge_O: \forall R: real. \forall x:R. (zero R) ≤ abs R x.
+lemma abs_x_ge_O: ∀R:real.∀x:R. 0 ≤ abs ? x.
  intros;
  unfold abs;
  unfold max;