src/HOL/Codegenerator_Test/Generate_Efficient_Datastructures.thy
changeset 63965 d510b816ea41
parent 63167 0909deb8059b
child 64786 340db65fd2c1
--- a/src/HOL/Codegenerator_Test/Generate_Efficient_Datastructures.thy	Thu Sep 29 11:24:36 2016 +0100
+++ b/src/HOL/Codegenerator_Test/Generate_Efficient_Datastructures.thy	Thu Sep 29 16:49:42 2016 +0200
@@ -76,6 +76,9 @@
 lemma [code, code del]:
   "permutations_of_set = permutations_of_set" ..
 
+lemma [code, code del]:
+  "permutations_of_multiset = permutations_of_multiset" ..
+
 (*
   If the code generation ends with an exception with the following message:
   '"List.set" is not a constructor, on left hand side of equation: ...',