src/HOL/Tools/SMT/smt_normalize.ML
changeset 40162 7f58a9a843c2
parent 40161 539d07b00e5f
child 40274 6486c610a549
--- a/src/HOL/Tools/SMT/smt_normalize.ML	Tue Oct 26 11:39:26 2010 +0200
+++ b/src/HOL/Tools/SMT/smt_normalize.ML	Tue Oct 26 11:45:12 2010 +0200
@@ -17,7 +17,7 @@
 
 signature SMT_NORMALIZE =
 sig
-  type extra_norm = (int * thm) list -> Proof.context ->
+  type extra_norm = bool -> (int * thm) list -> Proof.context ->
     (int * thm) list * Proof.context
   val normalize: extra_norm -> bool -> (int * thm) list -> Proof.context ->
     (int * thm) list * Proof.context
@@ -480,7 +480,7 @@
 
 (* combined normalization *)
 
-type extra_norm = (int * thm) list -> Proof.context ->
+type extra_norm = bool -> (int * thm) list -> Proof.context ->
   (int * thm) list * Proof.context
 
 fun with_context f irules ctxt = (f ctxt irules, ctxt)
@@ -492,7 +492,7 @@
   |> normalize_numerals ctxt
   |> nat_as_int ctxt
   |> rpair ctxt
-  |-> extra_norm
+  |-> extra_norm with_datatypes
   |-> with_context (fn cx => map (apsnd (normalize_rule cx)))
   |-> SMT_Monomorph.monomorph
   |-> lift_lambdas