src/HOL/Hyperreal/StarClasses.thy
changeset 25230 022029099a83
parent 25208 1a7318a04068
child 25304 7491c00f0915
equal deleted inserted replaced
25229:2673709fb8f7 25230:022029099a83
   401 apply (transfer, erule (1) mult_strict_left_mono)
   401 apply (transfer, erule (1) mult_strict_left_mono)
   402 apply (transfer, erule (1) mult_strict_right_mono)
   402 apply (transfer, erule (1) mult_strict_right_mono)
   403 done
   403 done
   404 
   404 
   405 instance star :: (pordered_comm_semiring) pordered_comm_semiring
   405 instance star :: (pordered_comm_semiring) pordered_comm_semiring
   406 by (intro_classes, transfer, rule mult_mono1_class.times_zero_less_eq_less.mult_mono)
   406 by (intro_classes, transfer, rule mult_mono1_class.times_zero_less_eq_less.mult_mono1)
   407 
   407 
   408 instance star :: (pordered_cancel_comm_semiring) pordered_cancel_comm_semiring ..
   408 instance star :: (pordered_cancel_comm_semiring) pordered_cancel_comm_semiring ..
   409 
   409 
   410 instance star :: (ordered_comm_semiring_strict) ordered_comm_semiring_strict
   410 instance star :: (ordered_comm_semiring_strict) ordered_comm_semiring_strict
   411 by (intro_classes, transfer, rule ordered_comm_semiring_strict_class.plus_times_zero_less_eq_less.mult_strict_mono)
   411 by (intro_classes, transfer, rule ordered_comm_semiring_strict_class.plus_times_zero_less_eq_less.mult_strict_mono)
   449 qed
   449 qed
   450 
   450 
   451 subsection {* Number classes *}
   451 subsection {* Number classes *}
   452 
   452 
   453 lemma star_of_nat_def [transfer_unfold]: "of_nat n = star_of (of_nat n)"
   453 lemma star_of_nat_def [transfer_unfold]: "of_nat n = star_of (of_nat n)"
   454 by (induct_tac n, simp_all)
   454 by (induct n, simp_all)
   455 
   455 
   456 lemma Standard_of_nat [simp]: "of_nat n \<in> Standard"
   456 lemma Standard_of_nat [simp]: "of_nat n \<in> Standard"
   457 by (simp add: star_of_nat_def)
   457 by (simp add: star_of_nat_def)
   458 
   458 
   459 lemma star_of_of_nat [simp]: "star_of (of_nat n) = of_nat n"
   459 lemma star_of_of_nat [simp]: "star_of (of_nat n) = of_nat n"