src/HOL/Library/Formal_Power_Series.thy
changeset 64786 340db65fd2c1
parent 64784 5cb5e7ecb284
child 65396 b42167902f57
equal deleted inserted replaced
64785:ae0bbc8e45ad 64786:340db65fd2c1
  1419 
  1419 
  1420 end
  1420 end
  1421 
  1421 
  1422 instantiation fps :: (field) euclidean_ring_gcd
  1422 instantiation fps :: (field) euclidean_ring_gcd
  1423 begin
  1423 begin
  1424 definition fps_gcd_def: "(gcd :: 'a fps \<Rightarrow> _) = gcd_eucl"
  1424 definition fps_gcd_def: "(gcd :: 'a fps \<Rightarrow> _) = Euclidean_Algorithm.gcd"
  1425 definition fps_lcm_def: "(lcm :: 'a fps \<Rightarrow> _) = lcm_eucl"
  1425 definition fps_lcm_def: "(lcm :: 'a fps \<Rightarrow> _) = Euclidean_Algorithm.lcm"
  1426 definition fps_Gcd_def: "(Gcd :: 'a fps set \<Rightarrow> _) = Gcd_eucl"
  1426 definition fps_Gcd_def: "(Gcd :: 'a fps set \<Rightarrow> _) = Euclidean_Algorithm.Gcd"
  1427 definition fps_Lcm_def: "(Lcm :: 'a fps set \<Rightarrow> _) = Lcm_eucl"
  1427 definition fps_Lcm_def: "(Lcm :: 'a fps set \<Rightarrow> _) = Euclidean_Algorithm.Lcm"
  1428 instance by standard (simp_all add: fps_gcd_def fps_lcm_def fps_Gcd_def fps_Lcm_def)
  1428 instance by standard (simp_all add: fps_gcd_def fps_lcm_def fps_Gcd_def fps_Lcm_def)
  1429 end
  1429 end
  1430 
  1430 
  1431 lemma fps_gcd:
  1431 lemma fps_gcd:
  1432   assumes [simp]: "f \<noteq> 0" "g \<noteq> 0"
  1432   assumes [simp]: "f \<noteq> 0" "g \<noteq> 0"