src/HOL/Orderings.thy
changeset 15622 4723248c982b
parent 15531 08c8dad8e399
child 15780 6744bba5561d
--- a/src/HOL/Orderings.thy	Thu Mar 24 10:59:21 2005 +0100
+++ b/src/HOL/Orderings.thy	Thu Mar 24 16:34:15 2005 +0100
@@ -287,7 +287,10 @@
    Quasi_Tac.quasi_tac are not of much use. *)
 
 fun decomp_gen sort sign (Trueprop $ t) =
-  let fun of_sort t = Sign.of_sort sign (type_of t, sort)
+  let fun of_sort t = let val T = type_of t in
+        (* exclude numeric types: linear arithmetic subsumes transitivity *)
+        T <> HOLogic.natT andalso T <> HOLogic.intT andalso
+        T <> HOLogic.realT andalso Sign.of_sort sign (T, sort) end
   fun dec (Const ("Not", _) $ t) = (
 	  case dec t of
 	    NONE => NONE