src/HOL/Tools/SMT/smt_normalize.ML
changeset 47155 ade3fc826af3
parent 47108 2a1953f0d20d
child 47207 9368aa814518
--- a/src/HOL/Tools/SMT/smt_normalize.ML	Tue Mar 27 16:59:13 2012 +0300
+++ b/src/HOL/Tools/SMT/smt_normalize.ML	Tue Mar 27 17:11:02 2012 +0200
@@ -346,32 +346,6 @@
 
 (* unfolding of definitions and theory-specific rewritings *)
 
-(** unfold trivial distincts **)
-
-local
-  fun is_trivial_distinct (Const (@{const_name distinct}, _) $ t) =
-        (case try HOLogic.dest_list t of
-          SOME [] => true
-        | SOME [_] => true
-        | _ => false)
-    | is_trivial_distinct _ = false
-
-  val thms = map mk_meta_eq @{lemma
-    "distinct [] = True"
-    "distinct [x] = True"
-    "distinct [x, y] = (x ~= y)"
-    by simp_all}
-  fun distinct_conv _ =
-    SMT_Utils.if_true_conv is_trivial_distinct (Conv.rewrs_conv thms)
-in
-
-fun trivial_distinct_conv ctxt =
-  SMT_Utils.if_exists_conv is_trivial_distinct
-    (Conv.top_conv distinct_conv ctxt)
-
-end
-
-
 (** rewrite bool case expressions as if expressions **)
 
 local
@@ -573,7 +547,6 @@
 (** combined unfoldings and rewritings **)
 
 fun unfold_conv ctxt =
-  trivial_distinct_conv ctxt then_conv
   rewrite_bool_case_conv ctxt then_conv
   unfold_abs_min_max_conv ctxt then_conv
   nat_as_int_conv ctxt then_conv