Skip to content
Snippets Groups Projects

various cleanups and simplifications in util

Merged Björn Brandenburg requested to merge MathComp-PR-cleanups-and-simplifications into master
1 file
+ 3
3
Compare changes
  • Side-by-side
  • Inline
+ 3
3
@@ -6,9 +6,9 @@ Require Export prosa.util.tactics.
(** Additional lemmas about natural numbers. *)
Section NatLemmas.
(** First, we show that, given [m1 >= m2] and [n1 >= n2], an
expression [(m1 + n1) - (m2 + n2)] can be transformed into
expression [(m1 - m2) + (n1 - n2)]. *)
(** First, we show that, given [m >= p] and [n >= q], an
expression [(m + n) - (p + q)] can be transformed into
expression [(m - p) + (n - q)]. *)
Lemma subnACA m n p q : p <= m -> q <= n ->
(m + n) - (p + q) = (m - p) + (n - q).
Proof. by move=> plem qlen; rewrite subnDA addnBAC// addnBA// subnAC. Qed.
Loading