src/HOL/ex/FinFunPred.thy
changeset 48034 1c5171abe5cc
parent 48029 9d9c9069abbc
child 48035 2f9584581cf2
--- a/src/HOL/ex/FinFunPred.thy	Wed May 30 08:34:14 2012 +0200
+++ b/src/HOL/ex/FinFunPred.thy	Wed May 30 08:48:14 2012 +0200
@@ -8,14 +8,14 @@
 
 text {* Instantiate FinFun predicates just like predicates *}
 
-type_synonym 'a pred\<^isub>f = "'a \<Rightarrow>\<^isub>f bool"
+type_synonym 'a pred\<^isub>f = "'a \<Rightarrow>f bool"
 
 instantiation "finfun" :: (type, ord) ord
 begin
 
 definition le_finfun_def [code del]: "f \<le> g \<longleftrightarrow> (\<forall>x. f\<^sub>f x \<le> g\<^sub>f x)"
 
-definition [code del]: "(f\<Colon>'a \<Rightarrow>\<^isub>f 'b) < g \<longleftrightarrow> f \<le> g \<and> \<not> f \<ge> g"
+definition [code del]: "(f\<Colon>'a \<Rightarrow>f 'b) < g \<longleftrightarrow> f \<le> g \<and> \<not> f \<ge> g"
 
 instance ..