use new-style class for po
authorhuffman
Mon, 14 Jan 2008 03:56:31 +0100
changeset 25897 e9d45709bece
parent 25896 b2d2f1ae5808
child 25898 d8f17d8cf9d4
use new-style class for po
src/HOLCF/Porder.thy
src/HOLCF/SetPcpo.thy
--- a/src/HOLCF/Porder.thy	Mon Jan 14 03:54:31 2008 +0100
+++ b/src/HOLCF/Porder.thy	Mon Jan 14 03:56:31 2008 +0100
@@ -20,10 +20,10 @@
 notation (xsymbols)
   sq_le (infixl "\<sqsubseteq>" 55)
 
-axclass po < sq_ord
-  refl_less [iff]: "x \<sqsubseteq> x"
-  antisym_less:    "\<lbrakk>x \<sqsubseteq> y; y \<sqsubseteq> x\<rbrakk> \<Longrightarrow> x = y"
-  trans_less:      "\<lbrakk>x \<sqsubseteq> y; y \<sqsubseteq> z\<rbrakk> \<Longrightarrow> x \<sqsubseteq> z"
+class po = sq_ord +
+  assumes refl_less [iff]: "x \<sqsubseteq> x"
+  assumes antisym_less: "\<lbrakk>x \<sqsubseteq> y; y \<sqsubseteq> x\<rbrakk> \<Longrightarrow> x = y"
+  assumes trans_less: "\<lbrakk>x \<sqsubseteq> y; y \<sqsubseteq> z\<rbrakk> \<Longrightarrow> x \<sqsubseteq> z"
 
 text {* minimal fixes least element *}
 
--- a/src/HOLCF/SetPcpo.thy	Mon Jan 14 03:54:31 2008 +0100
+++ b/src/HOLCF/SetPcpo.thy	Mon Jan 14 03:56:31 2008 +0100
@@ -9,17 +9,16 @@
 imports Adm
 begin
 
-instantiation set :: (type) sq_ord
+instantiation set :: (type) po
 begin
 
 definition
   less_set_def: "(op \<sqsubseteq>) = (op \<subseteq>)"
 
-instance ..
-end
+instance
+by (intro_classes, auto simp add: less_set_def)
 
-instance set :: (type) po
-by (intro_classes, auto simp add: less_set_def)
+end
 
 instance set :: (finite) finite_po ..