src/ZF/ArithSimp.thy
author nipkow
Fri, 31 May 2002 07:53:37 +0200
changeset 13189 81ed5c6de890
parent 9548 15bee2731e43
child 13259 01fa0c8dbc92
permissions -rw-r--r--
Now arith can deal with div/mod arbitrary nat numerals.

(*  Title:      ZF/ArithSimp.ML
    ID:         $Id$
    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
    Copyright   2000  University of Cambridge

Arithmetic with simplification
*)

theory ArithSimp = Arith
files "arith_data.ML":
end