src/HOL/ex/InductiveInvariant.thy
changeset 17388 495c799df31d
parent 16417 9bc16273c2d4
child 19736 d8d0f8f51d69
--- a/src/HOL/ex/InductiveInvariant.thy	Wed Sep 14 22:04:38 2005 +0200
+++ b/src/HOL/ex/InductiveInvariant.thy	Wed Sep 14 22:08:08 2005 +0200
@@ -1,12 +1,15 @@
+(*  ID:         $Id$
+    Author:	Sava Krsti\'{c} and John Matthews
+*)
+
+header {* Some of the results in Inductive Invariants for Nested Recursion *}
+
 theory InductiveInvariant imports Main begin
 
-(** Authors: Sava Krsti\'{c} and John Matthews **)
-(**    Date: Sep 12, 2003                      **)
-
-text {* A formalization of some of the results in
-        \emph{Inductive Invariants for Nested Recursion},
-        by Sava Krsti\'{c} and John Matthews.
-        Appears in the proceedings of TPHOLs 2003, LNCS vol. 2758, pp. 253-269. *}
+text {* A formalization of some of the results in \emph{Inductive
+  Invariants for Nested Recursion}, by Sava Krsti\'{c} and John
+  Matthews.  Appears in the proceedings of TPHOLs 2003, LNCS
+  vol. 2758, pp. 253-269. *}
 
 
 text "S is an inductive invariant of the functional F with respect to the wellfounded relation r."
@@ -86,4 +89,4 @@
  ==> S x (f x)"
 by (simp add: indinv_on_wfrec)
 
-end
\ No newline at end of file
+end