src/HOL/Library/Abstract_Rat.thy
changeset 33657 a4179bf442d1
parent 32960 69916a850301
child 35028 108662d50512
equal deleted inserted replaced
33648:555e5358b8c9 33657:a4179bf442d1
   204       apply algebra
   204       apply algebra
   205       apply algebra
   205       apply algebra
   206       apply simp
   206       apply simp
   207       apply algebra
   207       apply algebra
   208       done
   208       done
   209     from zdvd_dvd_eq[OF bz coprime_dvd_mult_int[OF gcd1(2) raw_dvd(2)]
   209     from zdvd_antisym_abs[OF coprime_dvd_mult_int[OF gcd1(2) raw_dvd(2)]
   210       coprime_dvd_mult_int[OF gcd1(4) raw_dvd(4)]]
   210       coprime_dvd_mult_int[OF gcd1(4) raw_dvd(4)]]
   211       have eq1: "b = b'" using pos by arith  
   211       have eq1: "b = b'" using pos by arith  
   212       with eq have "a = a'" using pos by simp
   212       with eq have "a = a'" using pos by simp
   213       with eq1 have ?rhs by simp}
   213       with eq1 have ?rhs by simp}
   214   ultimately show ?rhs by blast
   214   ultimately show ?rhs by blast