src/HOL/Arith.thy
author paulson
Fri, 15 Sep 2000 15:30:50 +0200
changeset 9970 dfe4747c8318
parent 9618 ff8238561394
permissions -rw-r--r--
the final renaming: selectI -> someI

(*  Title:      HOL/Arith.thy
    ID:         $Id$

Setup arithmetic proof procedures.
*)

theory Arith = Nat
files "arith_data.ML":

setup arith_setup

(*elimination of `-' on nat*)
lemma nat_diff_split:
    "P(a - b::nat) = (ALL d. (a<b --> P 0) & (a = b + d --> P d))"
  by (cases "a < b" rule: case_split) (auto simp add: diff_is_0_eq [THEN iffD2])

ML {* val nat_diff_split = thm "nat_diff_split" *}

lemmas [arith_split] = nat_diff_split split_min split_max

end