src/HOL/Calculation.thy
changeset 8855 ef4848bb0696
parent 8301 d9345bad5e5c
child 9035 371f023d3dbd
--- a/src/HOL/Calculation.thy	Wed May 10 21:03:12 2000 +0200
+++ b/src/HOL/Calculation.thy	Wed May 10 21:04:16 2000 +0200
@@ -6,7 +6,7 @@
 list below later rules have priority.
 *)
 
-theory Calculation = Int:;
+theory Calculation = IntArith:;
 
 theorems [trans] = rev_mp mp;