changeset 64850 | fc9265882329 |
parent 64786 | 340db65fd2c1 |
child 65919 | b6d458915f1b |
--- a/src/HOL/Codegenerator_Test/Generate_Efficient_Datastructures.thy Mon Jan 09 18:53:20 2017 +0100 +++ b/src/HOL/Codegenerator_Test/Generate_Efficient_Datastructures.thy Mon Jan 09 19:13:49 2017 +0100 @@ -34,6 +34,8 @@ Cardinality.finite' Cardinality.subset' Cardinality.eq_set + Gcd_fin + Lcm_fin "Gcd :: nat set \<Rightarrow> nat" "Lcm :: nat set \<Rightarrow> nat" "Gcd :: int set \<Rightarrow> int"