src/HOL/Rings.thy
changeset 61944 5d06ecfdb472
parent 61799 4cf66f21b764
child 62347 2230b7047376
equal deleted inserted replaced
61943:7fba644ed827 61944:5d06ecfdb472
  1557   by (auto simp add: mult_nonpos_nonpos)
  1557   by (auto simp add: mult_nonpos_nonpos)
  1558 
  1558 
  1559 lemma not_square_less_zero [simp]: "\<not> (a * a < 0)"
  1559 lemma not_square_less_zero [simp]: "\<not> (a * a < 0)"
  1560   by (simp add: not_less)
  1560   by (simp add: not_less)
  1561 
  1561 
  1562 proposition abs_eq_iff: "abs x = abs y \<longleftrightarrow> x = y \<or> x = -y"
  1562 proposition abs_eq_iff: "\<bar>x\<bar> = \<bar>y\<bar> \<longleftrightarrow> x = y \<or> x = -y"
  1563   by (auto simp add: abs_if split: split_if_asm)
  1563   by (auto simp add: abs_if split: split_if_asm)
  1564 
  1564 
  1565 end
  1565 end
  1566 
  1566 
  1567 class linordered_ring_strict = ring + linordered_semiring_strict
  1567 class linordered_ring_strict = ring + linordered_semiring_strict