src/HOL/Real/RealDef.thy
changeset 25502 9200b36280c0
parent 25303 0699e20feabd
child 25546 4f8d7ac83c0b
--- a/src/HOL/Real/RealDef.thy	Thu Nov 29 07:55:46 2007 +0100
+++ b/src/HOL/Real/RealDef.thy	Thu Nov 29 17:08:26 2007 +0100
@@ -66,7 +66,7 @@
   real_abs_def:  "abs (r::real) == (if r < 0 then - r else r)" ..
 
 instance real :: sgn
-  real_sgn_def: "sgn x == (if x=0 then 0 else if 0<x then 1 else - 1)" ..
+  real_sgn_def: "sgn (x::real) == (if x=0 then 0 else if 0<x then 1 else - 1)" ..
 
 subsection {* Equivalence relation over positive reals *}
 
@@ -401,8 +401,8 @@
 done
 
 instance real :: distrib_lattice
-  "inf x y \<equiv> min x y"
-  "sup x y \<equiv> max x y"
+  "inf \<Colon> real \<Rightarrow> real \<Rightarrow> real \<equiv> min"
+  "sup \<Colon> real \<Rightarrow> real \<Rightarrow> real \<equiv> max"
   by default (auto simp add: inf_real_def sup_real_def min_max.sup_inf_distrib1)