src/HOL/Bali/Name.thy
changeset 12859 f63315dfffd4
parent 12858 6214f03d6d27
child 13688 a0b16d42d489
--- a/src/HOL/Bali/Name.thy	Mon Jan 28 18:51:48 2002 +0100
+++ b/src/HOL/Bali/Name.thy	Mon Jan 28 23:35:20 2002 +0100
@@ -71,8 +71,7 @@
 axclass has_pname < "type"
 consts pname::"'a::has_pname \<Rightarrow> pname"
 
-instance pname::has_pname
-by (intro_classes)
+instance pname::has_pname ..
 
 defs (overloaded)
 pname_pname_def: "pname (p::pname) \<equiv> p"
@@ -80,8 +79,7 @@
 axclass has_tname < "type"
 consts tname::"'a::has_tname \<Rightarrow> tname"
 
-instance tname::has_tname
-by (intro_classes)
+instance tname::has_tname ..
 
 defs (overloaded)
 tname_tname_def: "tname (t::tname) \<equiv> t"
@@ -90,8 +88,7 @@
 consts qtname:: "'a::has_qtname \<Rightarrow> qtname"
 
 (* Declare qtname as instance of has_qtname *)
-instance pid_field_type::(has_pname,"type") has_qtname
-by intro_classes 
+instance pid_field_type::(has_pname,"type") has_qtname ..
 
 defs (overloaded)
 qtname_qtname_def: "qtname (q::qtname) \<equiv> q"