src/HOL/Rat.thy
changeset 70347 e5cd5471c18a
parent 70345 80a1aa30e24d
child 70350 571ae57313a4
equal deleted inserted replaced
70346:408e15cbd2a6 70347:e5cd5471c18a
   527     done
   527     done
   528 qed
   528 qed
   529 
   529 
   530 end
   530 end
   531 
   531 
   532 text\<open>Lemmas \<open>sign_simps\<close> is a first attempt to automate proofs
       
   533 of positivity/negativity needed for \<open>field_simps\<close>. Have not added \<open>sign_simps\<close> to \<open>field_simps\<close> because the former can lead to case
       
   534 explosions.\<close>
       
   535 
       
   536 lemmas (in linordered_field) sign_simps [no_atp] = algebra_simps zero_less_mult_iff mult_less_0_iff
       
   537 lemmas sign_simps [no_atp] = algebra_simps zero_less_mult_iff mult_less_0_iff
       
   538 
       
   539 
       
   540 instantiation rat :: distrib_lattice
   532 instantiation rat :: distrib_lattice
   541 begin
   533 begin
   542 
   534 
   543 definition "(inf :: rat \<Rightarrow> rat \<Rightarrow> rat) = min"
   535 definition "(inf :: rat \<Rightarrow> rat \<Rightarrow> rat) = min"
   544 
   536