src/HOL/HOL.thy
changeset 20741 c8fdad2dc6e6
parent 20713 823967ef47f1
child 20766 9913d3bc3d17
equal deleted inserted replaced
20740:5a103b43da5a 20741:c8fdad2dc6e6
   227 in
   227 in
   228   map (tr' o prefix Syntax.constN) ["HOL.one", "HOL.zero"]
   228   map (tr' o prefix Syntax.constN) ["HOL.one", "HOL.zero"]
   229 end;
   229 end;
   230 *} -- {* show types that are presumably too general *}
   230 *} -- {* show types that are presumably too general *}
   231 
   231 
   232 syntax
   232 const_syntax
   233   uminus :: "'a\<Colon>minus \<Rightarrow> 'a" ("- _" [81] 80)
   233   uminus  ("- _" [81] 80)
   234 
   234 
   235 syntax (xsymbols)
   235 const_syntax (xsymbols)
   236   abs :: "'a::minus => 'a"    ("\<bar>_\<bar>")
   236   abs  ("\<bar>_\<bar>")
   237 syntax (HTML output)
   237 const_syntax (HTML output)
   238   abs :: "'a::minus => 'a"    ("\<bar>_\<bar>")
   238   abs  ("\<bar>_\<bar>")
   239 
   239 
   240 
   240 
   241 subsection {*Equality*}
   241 subsection {*Equality*}
   242 
   242 
   243 lemma sym: "s = t ==> t = s"
   243 lemma sym: "s = t ==> t = s"