src/HOLCF/IOA/meta_theory/Pred.thy
changeset 36452 d37c6eed8117
parent 35355 613e133966ea
--- a/src/HOLCF/IOA/meta_theory/Pred.thy	Wed Apr 28 11:41:27 2010 +0200
+++ b/src/HOLCF/IOA/meta_theory/Pred.thy	Wed Apr 28 12:07:52 2010 +0200
@@ -8,7 +8,7 @@
 imports Main
 begin
 
-defaultsort type
+default_sort type
 
 types
   'a predicate = "'a => bool"