1
(* Title: ZF/ArithSimp.ML
2
ID: $Id$
3
Author: Lawrence C Paulson, Cambridge University Computer Laboratory
4
Copyright 2000 University of Cambridge
5
6
Arithmetic with simplification
7
*)
8
9
theory ArithSimp = Arith
10
files "arith_data.ML":
11
end