diff -r c50db2128048 -r 766db3539859 src/HOL/Rat.thy --- a/src/HOL/Rat.thy Mon Jan 09 18:53:06 2017 +0100 +++ b/src/HOL/Rat.thy Mon Jan 09 18:53:20 2017 +0100 @@ -401,6 +401,9 @@ lemma quotient_of_denom_pos: "quotient_of r = (p, q) \ q > 0" by (cases r) (simp add: quotient_of_Fract normalize_denom_pos) +lemma quotient_of_denom_pos': "snd (quotient_of r) > 0" + using quotient_of_denom_pos [of r] by (simp add: prod_eq_iff) + lemma quotient_of_coprime: "quotient_of r = (p, q) \ coprime p q" by (cases r) (simp add: quotient_of_Fract normalize_coprime)