src/HOL/ex/Adder.thy
changeset 17388 495c799df31d
parent 16417 9bc16273c2d4
child 19736 d8d0f8f51d69
--- a/src/HOL/ex/Adder.thy	Wed Sep 14 22:04:38 2005 +0200
+++ b/src/HOL/ex/Adder.thy	Wed Sep 14 22:08:08 2005 +0200
@@ -1,11 +1,9 @@
 (*  Title:      HOL/ex/Adder.thy
     ID:         $Id$
     Author:     Sergey Tverdyshev (Universitaet des Saarlandes)
-
-Implementation of carry chain incrementor and adder.
 *)
 
-header{* Adder *}
+header {* Implementation of carry chain incrementor and adder *}
 
 theory Adder imports Main Word begin