src/HOL/Induct/Term.thy
changeset 5191 8ceaa19f7717
parent 3120 c58423c20740
child 5717 0d28dbe484b6
--- a/src/HOL/Induct/Term.thy	Fri Jul 24 13:36:49 1998 +0200
+++ b/src/HOL/Induct/Term.thy	Fri Jul 24 13:39:47 1998 +0200
@@ -6,7 +6,7 @@
 Terms over a given alphabet -- function applications; illustrates list functor
   (essentially the same type as in Trees & Forests)
 
-There is no constructor APP because it is simply cons ($) 
+There is no constructor APP because it is simply Scons
 *)
 
 Term = SList +
@@ -27,7 +27,7 @@
 
 inductive "term(A)"
   intrs
-    APP_I "[| M: A;  N : list(term(A)) |] ==> M$N : term(A)"
+    APP_I "[| M: A;  N : list(term(A)) |] ==> Scons M N : term(A)"
   monos   "[list_mono]"
 
 defs
@@ -36,7 +36,7 @@
   Abs_Tlist_def "Abs_Tlist == Abs_map(Abs_term)"
 
   (*defining the abstract constants*)
-  App_def       "App a ts == Abs_term(Leaf(a) $ Rep_Tlist(ts))"
+  App_def       "App a ts == Abs_term(Scons (Leaf a) (Rep_Tlist ts))"
 
   (*list recursion*)
   Term_rec_def