Theory Number_Toolkit

section ‹ Number Toolkit ›

theory Number_Toolkit
  imports Function_Toolkit
begin

text ‹ The numeric operators are all implemented in HOL (@{const "plus"}, @{const "minus"}, 
  @{const times}, etc.), and there seems little to be gained by repackaging them. However,
  we do make some syntactic additions. ›

subsection ‹ Successor ›

abbreviation (input) "succ n  n + 1"

subsection ‹ Integers ›

type_notation int ("")

subsection ‹ Natural numbers ›

type_notation nat ("")

subsection ‹ Rational numbers ›

type_notation rat ("")

subsection ‹ Real numbers ›

type_notation real ("")

subsection ‹ Strictly positive natural numbers ›

definition Nats1 ("1") where "1 = {x  . ¬ x = 0}"

subsection ‹ Non-zero integers ›

definition Ints1 ("1") where "1 = {x  . ¬ x = 0}"

end