src/ZF/ArithSimp.thy
changeset 9548 15bee2731e43
child 13259 01fa0c8dbc92
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/src/ZF/ArithSimp.thy	Mon Aug 07 10:29:54 2000 +0200
@@ -0,0 +1,11 @@
+(*  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