src/HOL/Rings.thy
changeset 52435 6646bb548c6b
parent 51520 e9b361845809
child 54147 97a8ff4e4ac9
equal deleted inserted replaced
52434:cbb94074682b 52435:6646bb548c6b
  1147   "\<bar>x - a\<bar> < r \<longleftrightarrow> a - r < x \<and> x < a + r"
  1147   "\<bar>x - a\<bar> < r \<longleftrightarrow> a - r < x \<and> x < a + r"
  1148   by (auto simp add: diff_less_eq ac_simps abs_less_iff)
  1148   by (auto simp add: diff_less_eq ac_simps abs_less_iff)
  1149 
  1149 
  1150 end
  1150 end
  1151 
  1151 
  1152 code_modulename SML
  1152 code_identifier
  1153   Rings Arith
  1153   code_module Rings \<rightharpoonup> (SML) Arith and (OCaml) Arith and (Haskell) Arith
  1154 
  1154 
  1155 code_modulename OCaml
  1155 end
  1156   Rings Arith
  1156 
  1157 
       
  1158 code_modulename Haskell
       
  1159   Rings Arith
       
  1160 
       
  1161 end