src/HOL/Library/Code_Natural.thy
changeset 39781 2053638a2bf2
parent 39272 0b61951d2682
child 46547 d1dcb91a512e
--- a/src/HOL/Library/Code_Natural.thy	Wed Sep 29 09:21:26 2010 +0200
+++ b/src/HOL/Library/Code_Natural.thy	Wed Sep 29 10:05:44 2010 +0200
@@ -78,7 +78,7 @@
   def equals(that: Natural): Boolean = this.value == that.value
 
   def as_BigInt: BigInt = this.value
-  def as_Int: Int = if (this.value >= Int.MinValue && this.value <= Int.MaxValue)
+  def as_Int: Int = if (this.value >= scala.Int.MinValue && this.value <= scala.Int.MaxValue)
       this.value.intValue
     else error("Int value out of range: " + this.value.toString)