src/HOL/Word/Word.thy
changeset 29628 d9294387ab0e
parent 27137 d0070c32fdc1
child 35049 00f311c32444
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/src/HOL/Word/Word.thy	Mon Jan 26 22:14:16 2009 +0100
@@ -0,0 +1,13 @@
+(*  Title:      HOL/Word/Word.thy
+    Author:     Gerwin Klein, NICTA
+*)
+
+header {* Word Library interafce *}
+
+theory Word
+imports WordGenLib
+begin
+
+text {* see @{text "Examples/WordExamples.thy"} for examples *}
+
+end