src/HOL/Fun.thy
changeset 12338 de0f4a63baa5
parent 12258 5da24e7e9aba
child 12459 6978ab7cac64
--- a/src/HOL/Fun.thy	Sat Dec 01 18:51:46 2001 +0100
+++ b/src/HOL/Fun.thy	Sat Dec 01 18:52:32 2001 +0100
@@ -8,7 +8,7 @@
 
 Fun = Typedef +
 
-instance set :: (term) order
+instance set :: (type) order
                        (subset_refl,subset_trans,subset_antisym,psubset_eq)
 consts
   fun_upd  :: "('a => 'b) => 'a => 'b => ('a => 'b)"