src/HOL/Tools/SMT/smtlib_interface.ML
changeset 47155 ade3fc826af3
parent 41473 3717fc42ebe9
--- a/src/HOL/Tools/SMT/smtlib_interface.ML	Tue Mar 27 16:59:13 2012 +0300
+++ b/src/HOL/Tools/SMT/smtlib_interface.ML	Tue Mar 27 17:11:02 2012 +0200
@@ -32,16 +32,6 @@
   fun times _ _ ts =
     let val mk = Term.list_comb o pair @{const times (int)}
     in if is_linear ts then SOME ("*", 2, ts, mk) else NONE end
-
-  fun distinct _ T [t] =
-        (case try HOLogic.dest_list t of
-          SOME (ts as _ :: _) =>
-            let
-              val c = Const (@{const_name distinct}, T)
-              fun mk us = c $ HOLogic.mk_list T us
-            in SOME ("distinct", length ts, ts, mk) end
-        | _ => NONE)
-    | distinct _ _ _ = NONE
 in
 
 val setup_builtins =
@@ -63,9 +53,7 @@
     (@{const plus (int)}, "+"),
     (@{const minus (int)}, "-") ] #>
   SMT_Builtin.add_builtin_fun smtlibC
-    (Term.dest_Const @{const times (int)}, times) #>
-  SMT_Builtin.add_builtin_fun smtlibC
-    (Term.dest_Const @{const distinct ('a)}, distinct)
+    (Term.dest_Const @{const times (int)}, times)
 
 end