src/HOL/Ring_and_Field.thy
changeset 15229 1eb23f805c06
parent 15228 4d332d10fa3d
child 15234 ec91a90c604e
equal deleted inserted replaced
15228:4d332d10fa3d 15229:1eb23f805c06
     3     Author:  Gertrud Bauer, Steven Obua, Lawrence C Paulson and Markus Wenzel
     3     Author:  Gertrud Bauer, Steven Obua, Lawrence C Paulson and Markus Wenzel
     4 *)
     4 *)
     5 
     5 
     6 header {* (Ordered) Rings and Fields *}
     6 header {* (Ordered) Rings and Fields *}
     7 
     7 
     8 theory Ring_and_Field 
     8 theory Ring_and_Field
     9 imports OrderedGroup
     9 imports OrderedGroup
    10 begin
    10 begin
    11 
    11 
    12 text {*
    12 text {*
    13   The theory of partially ordered rings is taken from the books:
    13   The theory of partially ordered rings is taken from the books:
  1368 
  1368 
  1369 subsection {* Absolute Value *}
  1369 subsection {* Absolute Value *}
  1370 
  1370 
  1371 lemma abs_one [simp]: "abs 1 = (1::'a::ordered_idom)"
  1371 lemma abs_one [simp]: "abs 1 = (1::'a::ordered_idom)"
  1372   by (simp add: abs_if zero_less_one [THEN order_less_not_sym]) 
  1372   by (simp add: abs_if zero_less_one [THEN order_less_not_sym]) 
       
  1373 
       
  1374 lemma abs_eq [simp]: "(0::'a::ordered_idom) \<le> a ==> abs a = a"
       
  1375 by (simp add: abs_if linorder_not_less [symmetric]) 
       
  1376 
       
  1377 lemma abs_minus_eq [simp]: "a < (0::'a::ordered_idom) ==> abs a = -a"
       
  1378 by (simp add: abs_if linorder_not_less [symmetric])
  1373 
  1379 
  1374 lemma abs_le_mult: "abs (a * b) \<le> (abs a) * (abs (b::'a::lordered_ring))" 
  1380 lemma abs_le_mult: "abs (a * b) \<le> (abs a) * (abs (b::'a::lordered_ring))" 
  1375 proof -
  1381 proof -
  1376   let ?x = "pprt a * pprt b - pprt a * nprt b - nprt a * pprt b + nprt a * nprt b"
  1382   let ?x = "pprt a * pprt b - pprt a * nprt b - nprt a * pprt b + nprt a * nprt b"
  1377   let ?y = "pprt a * pprt b + pprt a * nprt b + nprt a * pprt b + nprt a * nprt b"
  1383   let ?y = "pprt a * pprt b + pprt a * nprt b + nprt a * pprt b + nprt a * nprt b"