src/HOL/RealDef.thy
changeset 45051 c478d1876371
parent 44822 2690b6de5021
child 45184 426dbd896c9e
equal deleted inserted replaced
45050:f65593159ee8 45051:c478d1876371
  1047 
  1047 
  1048 declare Real_induct [induct del]
  1048 declare Real_induct [induct del]
  1049 declare Abs_real_induct [induct del]
  1049 declare Abs_real_induct [induct del]
  1050 declare Abs_real_cases [cases del]
  1050 declare Abs_real_cases [cases del]
  1051 
  1051 
  1052 subsection {* Legacy theorem names *}
       
  1053 
       
  1054 text {* TODO: Could we have a way to mark theorem names as deprecated,
       
  1055 and have Isabelle issue a warning and display the preferred name? *}
       
  1056 
       
  1057 lemmas real_diff_def = minus_real_def [of "r" "s", standard]
       
  1058 lemmas real_divide_def = divide_real_def [of "R" "S", standard]
       
  1059 lemmas real_less_def = less_le [of "x::real" "y", standard]
       
  1060 lemmas real_abs_def = abs_real_def [of "r", standard]
       
  1061 lemmas real_sgn_def = sgn_real_def [of "x", standard]
       
  1062 lemmas real_mult_commute = mult_commute [of "z::real" "w", standard]
       
  1063 lemmas real_mult_assoc = mult_assoc [of "z1::real" "z2" "z3", standard]
       
  1064 lemmas real_mult_1 = mult_1_left [of "z::real", standard]
       
  1065 lemmas real_add_mult_distrib = left_distrib [of "z1::real" "z2" "w", standard]
       
  1066 lemmas real_zero_not_eq_one = zero_neq_one [where 'a=real]
       
  1067 lemmas real_mult_inverse_left = left_inverse [of "x::real", standard]
       
  1068 lemmas INVERSE_ZERO = inverse_zero [where 'a=real]
       
  1069 lemmas real_le_refl = order_refl [of "w::real", standard]
       
  1070 lemmas real_le_antisym = order_antisym [of "z::real" "w", standard]
       
  1071 lemmas real_le_trans = order_trans [of "i::real" "j" "k", standard]
       
  1072 lemmas real_le_linear = linear [of "z::real" "w", standard]
       
  1073 lemmas real_le_eq_diff = le_iff_diff_le_0 [of "x::real" "y", standard]
       
  1074 lemmas real_add_left_mono = add_left_mono [of "x::real" "y" "z", standard]
       
  1075 lemmas real_mult_order = mult_pos_pos [of "x::real" "y", standard]
       
  1076 lemmas real_mult_less_mono2 =
       
  1077   mult_strict_left_mono [of "x::real" "y" "z", COMP swap_prems_rl, standard]
       
  1078 
       
  1079 subsection{*More Lemmas*}
  1052 subsection{*More Lemmas*}
  1080 
  1053 
  1081 text {* BH: These lemmas should not be necessary; they should be
  1054 text {* BH: These lemmas should not be necessary; they should be
  1082 covered by existing simp rules and simplification procedures. *}
  1055 covered by existing simp rules and simplification procedures. *}
  1083 
  1056