src/HOL/MicroJava/BV/Typing_Framework.thy
changeset 13224 6f0928a942d1
parent 13062 4b1edf2f6bd2
child 14653 0848ab6fe5fc
--- a/src/HOL/MicroJava/BV/Typing_Framework.thy	Wed Jun 19 11:48:01 2002 +0200
+++ b/src/HOL/MicroJava/BV/Typing_Framework.thy	Wed Jun 19 12:39:41 2002 +0200
@@ -9,7 +9,7 @@
 theory Typing_Framework = Listn:
 
 text {* 
-  The relationship between dataflow analysis and a welltyped-insruction predicate. 
+  The relationship between dataflow analysis and a welltyped-instruction predicate. 
 *}
 types
   's step_type = "nat \<Rightarrow> 's \<Rightarrow> (nat \<times> 's) list"