src/HOL/HOL.thy
changeset 24506 020db6ec334a
parent 24462 d66cd8668a91
child 24553 9b19da7b2b08
equal deleted inserted replaced
24505:9e6d91f8bb73 24506:020db6ec334a
   230   fixes inverse :: "'a \<Rightarrow> 'a"
   230   fixes inverse :: "'a \<Rightarrow> 'a"
   231     and divide :: "'a \<Rightarrow> 'a \<Rightarrow> 'a"  (infixl "\<^loc>'/" 70)
   231     and divide :: "'a \<Rightarrow> 'a \<Rightarrow> 'a"  (infixl "\<^loc>'/" 70)
   232 
   232 
   233 class abs = type +
   233 class abs = type +
   234   fixes abs :: "'a \<Rightarrow> 'a"
   234   fixes abs :: "'a \<Rightarrow> 'a"
       
   235 
       
   236 class sgn = type +
       
   237   fixes sgn :: "'a \<Rightarrow> 'a"
   235 
   238 
   236 notation
   239 notation
   237   uminus  ("- _" [81] 80)
   240   uminus  ("- _" [81] 80)
   238 
   241 
   239 notation (xsymbols)
   242 notation (xsymbols)