src/HOL/Num.thy
changeset 58512 dc4d76dfa8f0
parent 58421 37cbbd8eb460
child 58889 5b7a9633cfa8
equal deleted inserted replaced
58511:97aec08d6f28 58512:dc4d76dfa8f0
  1071   by simp
  1071   by simp
  1072 
  1072 
  1073 lemmas nat_1_add_1 = one_add_one [where 'a=nat] (* legacy *)
  1073 lemmas nat_1_add_1 = one_add_one [where 'a=nat] (* legacy *)
  1074 
  1074 
  1075 
  1075 
       
  1076 subsection {* Particular lemmas concerning @{term 2} *}
       
  1077 
       
  1078 context linordered_field_inverse_zero
       
  1079 begin
       
  1080 
       
  1081 lemma half_gt_zero_iff:
       
  1082   "0 < a / 2 \<longleftrightarrow> 0 < a" (is "?P \<longleftrightarrow> ?Q")
       
  1083   by (auto simp add: field_simps)
       
  1084 
       
  1085 lemma half_gt_zero [simp]:
       
  1086   "0 < a \<Longrightarrow> 0 < a / 2"
       
  1087   by (simp add: half_gt_zero_iff)
       
  1088 
       
  1089 end
       
  1090 
       
  1091 
  1076 subsection {* Numeral equations as default simplification rules *}
  1092 subsection {* Numeral equations as default simplification rules *}
  1077 
  1093 
  1078 declare (in numeral) numeral_One [simp]
  1094 declare (in numeral) numeral_One [simp]
  1079 declare (in numeral) numeral_plus_numeral [simp]
  1095 declare (in numeral) numeral_plus_numeral [simp]
  1080 declare (in numeral) add_numeral_special [simp]
  1096 declare (in numeral) add_numeral_special [simp]