src/HOL/Bali/WellType.thy
changeset 46212 d86ef6b96097
parent 41778 5f79a9e42507
child 46714 a7ca72710dfe
--- a/src/HOL/Bali/WellType.thy	Sat Jan 14 16:12:09 2012 +0100
+++ b/src/HOL/Bali/WellType.thy	Sat Jan 14 16:14:22 2012 +0100
@@ -108,7 +108,7 @@
 
 definition
   --{* applicable methods, cf. 15.11.2.1 *}
-  appl_methds :: "prog \<Rightarrow> qtname \<Rightarrow>  ref_ty \<Rightarrow> sig \<Rightarrow> (emhead \<times> ty list)\<spacespace> set" where
+  appl_methds :: "prog \<Rightarrow> qtname \<Rightarrow>  ref_ty \<Rightarrow> sig \<Rightarrow> (emhead \<times> ty list) set" where
   "appl_methds G S rt = (\<lambda> sig. 
       {(mh,pTs') |mh pTs'. mh \<in> mheads G S rt \<lparr>name=name sig,parTs=pTs'\<rparr> \<and> 
                            G\<turnstile>(parTs sig)[\<preceq>]pTs'})"
@@ -121,7 +121,7 @@
 
 definition
   --{* maximally specific methods, cf. 15.11.2.2 *}
-  max_spec :: "prog \<Rightarrow> qtname \<Rightarrow> ref_ty \<Rightarrow> sig \<Rightarrow> (emhead \<times> ty list)\<spacespace> set" where
+  max_spec :: "prog \<Rightarrow> qtname \<Rightarrow> ref_ty \<Rightarrow> sig \<Rightarrow> (emhead \<times> ty list) set" where
   "max_spec G S rt sig = {m. m \<in>appl_methds G S rt sig \<and>
                           (\<forall>m'\<in>appl_methds G S rt sig. more_spec G m' m \<longrightarrow> m'=m)}"