src/HOL/IMP/Vars.thy
changeset 50303 5c4c35321e87
parent 50173 e014009fbd93
child 51698 c0af8bbc5825
--- a/src/HOL/IMP/Vars.thy	Thu Nov 29 23:12:50 2012 +0100
+++ b/src/HOL/IMP/Vars.thy	Fri Nov 30 17:12:01 2012 +0100
@@ -1,6 +1,6 @@
 (* Author: Tobias Nipkow *)
 
-header "Definite Assignment Analysis"
+header "Definite Initialization Analysis"
 
 theory Vars imports BExp
 begin