src/HOL/IntDef.thy
changeset 25230 022029099a83
parent 25193 e2e1a4b00de3
child 25349 0d46bea01741
--- a/src/HOL/IntDef.thy	Mon Oct 29 17:08:01 2007 +0100
+++ b/src/HOL/IntDef.thy	Tue Oct 30 08:45:54 2007 +0100
@@ -429,6 +429,8 @@
 context ring_1
 begin
 
+term of_nat
+
 definition
   of_int :: "int \<Rightarrow> 'a"
 where
@@ -518,10 +520,15 @@
     by (cases z) (simp add: of_int add minus int_def diff_minus)
 qed
 
+context ring_1
+begin
+
 lemma of_nat_nat: "0 \<le> z \<Longrightarrow> of_nat (nat z) = of_int z"
-by (cases z rule: eq_Abs_Integ)
+  by (cases z rule: eq_Abs_Integ)
    (simp add: nat le of_int Zero_int_def of_nat_diff)
 
+end
+
 
 subsection{*The Set of Integers*}