src/ZF/Coind/Types.thy
changeset 6046 2c8a8be36c94
parent 3840 e0baea4d485a
child 6068 2d8f3e1f1151
--- a/src/ZF/Coind/Types.thy	Mon Dec 28 16:53:24 1998 +0100
+++ b/src/ZF/Coind/Types.thy	Mon Dec 28 16:54:01 1998 +0100
@@ -23,19 +23,17 @@
           | te_owr("te:TyEnv","x:ExVar","t:Ty") 
 
 consts
-  te_rec :: [i,i,[i,i,i,i]=>i] => i
-defs
-  te_rec_def
-    "te_rec(te,c,h) ==   
-    Vrec(te,%te g. TyEnv_case(c,%tem x t. h(tem,x,t,g`tem),te))"
-  
-consts
   te_dom :: i => i
   te_app :: [i,i] => i
-defs
-  te_dom_def "te_dom(te) == te_rec(te,0,% te x t r. r Un {x})"
-  te_app_def "te_app(te,x) == te_rec(te,0, % te y t r. if(x=y,t,r))"
-  
+
+
+primrec (*domain of the type environment*)
+  "te_dom (te_emp) = 0"
+  "te_dom(te_owr(te,x,v)) = te_dom(te) Un {x}"
+
+primrec (*lookup up identifiers in the type environment*)
+  "te_app (te_emp,x) = 0"
+  "te_app (te_owr(te,y,t),x) = if(x=y, t, te_app(te,x))"
 
 end