src/HOL/MiniML/MiniML.thy
changeset 1476 608483c2122a
parent 1400 5d909faf0e04
child 1525 d127436567d0
--- a/src/HOL/MiniML/MiniML.thy	Mon Feb 05 21:27:16 1996 +0100
+++ b/src/HOL/MiniML/MiniML.thy	Mon Feb 05 21:29:06 1996 +0100
@@ -10,11 +10,11 @@
 
 (* expressions *)
 datatype
-	expr = Var nat | Abs expr | App expr expr
+        expr = Var nat | Abs expr | App expr expr
 
 (* type inference rules *)
 consts
-	has_type :: "(typ list * expr * typ)set"
+        has_type :: "(typ list * expr * typ)set"
 syntax
         "@has_type" :: [typ list, expr, typ] => bool
                        ("((_) |-/ (_) :: (_))" 60)
@@ -23,10 +23,10 @@
 
 inductive "has_type"
 intrs
-	VarI "[| n < length a |] ==> a |- Var n :: nth n a"
-	AbsI "[| t1#a |- e :: t2 |] ==> a |- Abs e :: t1 -> t2"
-	AppI "[| a |- e1 :: t2 -> t1; a |- e2 :: t2 |] 
-     	      ==> a |- App e1 e2 :: t1"
+        VarI "[| n < length a |] ==> a |- Var n :: nth n a"
+        AbsI "[| t1#a |- e :: t2 |] ==> a |- Abs e :: t1 -> t2"
+        AppI "[| a |- e1 :: t2 -> t1; a |- e2 :: t2 |] 
+              ==> a |- App e1 e2 :: t1"
 
 end