src/HOL/Orderings.thy
changeset 25502 9200b36280c0
parent 25377 dcde128c84a2
child 25510 38c15efe603b
--- a/src/HOL/Orderings.thy	Thu Nov 29 07:55:46 2007 +0100
+++ b/src/HOL/Orderings.thy	Thu Nov 29 17:08:26 2007 +0100
@@ -930,7 +930,7 @@
 
 instance bool :: order 
   le_bool_def: "P \<le> Q \<equiv> P \<longrightarrow> Q"
-  less_bool_def: "P < Q \<equiv> P \<le> Q \<and> P \<noteq> Q"
+  less_bool_def: "(P\<Colon>bool) < Q \<equiv> P \<le> Q \<and> P \<noteq> Q"
   by intro_classes (auto simp add: le_bool_def less_bool_def)
 lemmas [code func del] = le_bool_def less_bool_def
 
@@ -968,7 +968,7 @@
 
 instance "fun" :: (type, ord) ord
   le_fun_def: "f \<le> g \<equiv> \<forall>x. f x \<le> g x"
-  less_fun_def: "f < g \<equiv> f \<le> g \<and> f \<noteq> g" ..
+  less_fun_def: "(f\<Colon>'a \<Rightarrow> 'b) < g \<equiv> f \<le> g \<and> f \<noteq> g" ..
 
 lemmas [code func del] = le_fun_def less_fun_def