src/HOL/Power.thy
changeset 71398 e0237f2eb49d
parent 70928 273fc913427b
child 71435 d8fb621fea02
equal deleted inserted replaced
71397:028edb1e5b99 71398:e0237f2eb49d
   375 qed (auto intro: unit_imp_dvd simp: is_unit_power_iff le_imp_power_dvd)
   375 qed (auto intro: unit_imp_dvd simp: is_unit_power_iff le_imp_power_dvd)
   376 
   376 
   377 
   377 
   378 end
   378 end
   379 
   379 
   380 context normalization_semidom
   380 context normalization_semidom_multiplicative
   381 begin
   381 begin
   382 
   382 
   383 lemma normalize_power: "normalize (a ^ n) = normalize a ^ n"
   383 lemma normalize_power: "normalize (a ^ n) = normalize a ^ n"
   384   by (induct n) (simp_all add: normalize_mult)
   384   by (induct n) (simp_all add: normalize_mult)
   385 
   385