src/HOL/Library/EfficientNat.thy
changeset 23017 00c0e4c42396
parent 22928 1feef3b54ce1
child 23269 851b8ea067ac
equal deleted inserted replaced
23016:fd7cd1edc18d 23017:00c0e4c42396
   386 
   386 
   387 code_modulename OCaml
   387 code_modulename OCaml
   388   Nat Integer
   388   Nat Integer
   389   EfficientNat Integer
   389   EfficientNat Integer
   390 
   390 
       
   391 code_modulename Haskell
       
   392   Nat Integer
       
   393   EfficientNat Integer
       
   394 
   391 hide const nat_of_int
   395 hide const nat_of_int
   392 
   396 
   393 end
   397 end