src/HOL/Rat.thy
changeset 80932 261cd8722677
parent 80061 4c1347e172b1
child 81124 6ce0c8d59f5a
equal deleted inserted replaced
80931:f6e595e4f608 80932:261cd8722677
   798 subsection \<open>The Set of Rational Numbers\<close>
   798 subsection \<open>The Set of Rational Numbers\<close>
   799 
   799 
   800 context field_char_0
   800 context field_char_0
   801 begin
   801 begin
   802 
   802 
   803 definition Rats :: "'a set" ("\<rat>")
   803 definition Rats :: "'a set" (\<open>\<rat>\<close>)
   804   where "\<rat> = range of_rat"
   804   where "\<rat> = range of_rat"
   805 
   805 
   806 end
   806 end
   807 
   807 
   808 lemma Rats_cases [cases set: Rats]:
   808 lemma Rats_cases [cases set: Rats]:
  1153   uminus_rat_inst.uminus_rat zero_rat_inst.zero_rat
  1153   uminus_rat_inst.uminus_rat zero_rat_inst.zero_rat
  1154 
  1154 
  1155 
  1155 
  1156 subsection \<open>Float syntax\<close>
  1156 subsection \<open>Float syntax\<close>
  1157 
  1157 
  1158 syntax "_Float" :: "float_const \<Rightarrow> 'a"    ("_")
  1158 syntax "_Float" :: "float_const \<Rightarrow> 'a"    (\<open>_\<close>)
  1159 
  1159 
  1160 parse_translation \<open>
  1160 parse_translation \<open>
  1161   let
  1161   let
  1162     fun mk_frac str =
  1162     fun mk_frac str =
  1163       let
  1163       let