src/HOL/MiniML/MiniML.thy
changeset 1790 2f3694c50101
parent 1525 d127436567d0
child 2525 477c05586286
--- a/src/HOL/MiniML/MiniML.thy	Thu Jun 06 14:39:44 1996 +0200
+++ b/src/HOL/MiniML/MiniML.thy	Thu Jun 06 16:20:27 1996 +0200
@@ -21,7 +21,7 @@
 translations 
         "a |- e :: t" == "(a,e,t):has_type"
 
-inductive "has_type"
+inductive has_type
 intrs
         VarI "[| n < length a |] ==> a |- Var n :: nth n a"
         AbsI "[| t1#a |- e :: t2 |] ==> a |- Abs e :: t1 -> t2"