src/HOL/Tools/Predicate_Compile/predicate_compile_aux.ML
changeset 45701 615da8b8d758
parent 45461 130c90bb80b4
child 45822 843dc212f69e
--- a/src/HOL/Tools/Predicate_Compile/predicate_compile_aux.ML	Wed Nov 30 21:14:01 2011 +0100
+++ b/src/HOL/Tools/Predicate_Compile/predicate_compile_aux.ML	Wed Nov 30 23:30:08 2011 +0100
@@ -932,13 +932,10 @@
 
 fun case_rewrites thy Tcon =
   let
-    val info = Datatype.the_info thy Tcon
-    val descr = #descr info
-    val sorts = #sorts info
-    val typ_names = the_default [Tcon] (#alt_names info)
+    val {descr, sorts, ...} = Datatype.the_info thy Tcon
   in
     map (Drule.export_without_context o Skip_Proof.make_thm thy o HOLogic.mk_Trueprop)
-      (make_case_distribs typ_names [descr] sorts thy)
+      (make_case_distribs [Tcon] [descr] sorts thy)
   end
 
 fun instantiated_case_rewrites thy Tcon =