src/ZF/UNITY/GenPrefix.thy
changeset 24893 b8ef7afe3a6b
parent 24892 c663e675e177
child 26056 6a0801279f4c
--- a/src/ZF/UNITY/GenPrefix.thy	Sun Oct 07 15:49:25 2007 +0200
+++ b/src/ZF/UNITY/GenPrefix.thy	Sun Oct 07 21:19:31 2007 +0200
@@ -15,8 +15,8 @@
 imports Main
 begin
 
-constdefs (*really belongs in ZF/Trancl*)
-  part_order :: "[i, i] => o"
+definition (*really belongs in ZF/Trancl*)
+  part_order :: "[i, i] => o"  where
   "part_order(A, r) == refl(A,r) & trans[A](r) & antisym(r)"
 
 consts
@@ -37,11 +37,12 @@
 	      ==> <xs, ys@zs>:gen_prefix(A, r)"
     type_intros app_type list.Nil list.Cons
 
-constdefs
-   prefix :: "i=>i"
+definition
+  prefix :: "i=>i"  where
   "prefix(A) == gen_prefix(A, id(A))"
 
-   strict_prefix :: "i=>i"
+definition
+  strict_prefix :: "i=>i"  where
   "strict_prefix(A) == prefix(A) - id(list(A))"