src/HOL/Library/Efficient_Nat.thy
changeset 38774 567b94f8bb6e
parent 38771 f9cd27cbe8a4
child 38857 97775f3e8722
--- a/src/HOL/Library/Efficient_Nat.thy	Thu Aug 26 12:19:49 2010 +0200
+++ b/src/HOL/Library/Efficient_Nat.thy	Thu Aug 26 12:19:50 2010 +0200
@@ -242,8 +242,8 @@
   and @{typ int}.
 *}
 
-code_include Haskell "Nat" {*
-newtype Nat = Nat Integer deriving (Eq, Show, Read);
+code_include Haskell "Nat"
+{*newtype Nat = Nat Integer deriving (Eq, Show, Read);
 
 instance Num Nat where {
   fromInteger k = Nat (if k >= 0 then k else 0);
@@ -280,8 +280,8 @@
 
 code_reserved Haskell Nat
 
-code_include Scala "Nat" {*
-import scala.Math
+code_include Scala "Nat"
+{*import scala.Math
 
 object Nat {