--- a/Admin/Benchmarks/HOL-datatype/SML.thy Sun Nov 15 13:06:42 2009 +0100
+++ b/Admin/Benchmarks/HOL-datatype/SML.thy Sun Nov 15 15:13:31 2009 +0100
@@ -1,13 +1,10 @@
(* Title: Admin/Benchmarks/HOL-datatype/SML.thy
- ID: $Id$
+
+Example from Myra: part of the syntax of SML.
*)
theory SML imports Main begin
-(* ------------------------------------------------------------------------- *)
-(* Example from Myra: part of the syntax of SML. *)
-(* ------------------------------------------------------------------------- *)
-
datatype
string = EMPTY_STRING | CONS_STRING nat string