]> matita.cs.unibo.it Git - helm.git/blobdiff - helm/software/matita/contribs/assembly/freescale/extra.ma
nasty change in the lexer/parser:
[helm.git] / helm / software / matita / contribs / assembly / freescale / extra.ma
index 207a5a267d386b67af511cedf815e1c242114261..7da45c848e3a2aef8e3f012548998ea217c177ce 100644 (file)
@@ -208,7 +208,7 @@ axiom or_lt_le : ∀n,m. n < m ∨ m ≤ n.
 
 lemma le_to_lt: ∀n,m. n ≤ m → n < S m.
  intros;
- autobatch.
unfold;autobatch.
 qed.
 
 alias num (instance 0) = "natural number".
@@ -253,7 +253,7 @@ lemma leq_m_n_to_eq_div_n_m_S: ∀n,m:nat. 0 < m → m ≤ n → ∃z. n/m = S z
         ]
      | elim H1; autobatch
      ]
-  | autobatch
+  | exists;[apply (pred m);]autobatch
   ].
 qed.