Admin/Benchmarks/HOL-datatype/Verilog.thy
changeset 33695 bec342db1bf4
parent 22875 9b21fa38a3cf
--- a/Admin/Benchmarks/HOL-datatype/Verilog.thy	Sun Nov 15 13:06:42 2009 +0100
+++ b/Admin/Benchmarks/HOL-datatype/Verilog.thy	Sun Nov 15 15:13:31 2009 +0100
@@ -1,13 +1,10 @@
 (*  Title:      Admin/Benchmarks/HOL-datatype/Verilog.thy
-    ID:         $Id$
+
+Example from Daryl: a Verilog grammar.
 *)
 
 theory Verilog imports Main begin
 
-(* ------------------------------------------------------------------------- *)
-(* Example from Daryl: a Verilog grammar.                                    *)
-(* ------------------------------------------------------------------------- *)
-
 datatype
   Source_text
      = module string "string list" "Module_item list"