src/HOL/Library/Efficient_Nat.thy
changeset 37050 4a021f6be77c
parent 36603 d5d6111761a6
child 37223 5226259b6fa2
--- a/src/HOL/Library/Efficient_Nat.thy	Thu May 20 21:19:38 2010 -0700
+++ b/src/HOL/Library/Efficient_Nat.thy	Fri May 21 11:50:34 2010 +0200
@@ -252,7 +252,7 @@
 *}
 
 code_include Haskell "Nat" {*
-newtype Nat = Nat Integer deriving (Show, Eq);
+newtype Nat = Nat Integer deriving (Eq, Show, Read);
 
 instance Num Nat where {
   fromInteger k = Nat (if k >= 0 then k else 0);