src/HOL/Library/Efficient_Nat.thy
changeset 39781 2053638a2bf2
parent 39302 d7728f65b353
child 40607 30d512bf47a7
--- a/src/HOL/Library/Efficient_Nat.thy	Wed Sep 29 09:21:26 2010 +0200
+++ b/src/HOL/Library/Efficient_Nat.thy	Wed Sep 29 10:05:44 2010 +0200
@@ -303,7 +303,7 @@
   def equals(that: Nat): 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)