src/HOL/Orderings.thy
changeset 30240 5b25fee0362c
parent 29823 0ab754d13ccd
child 30298 abefe1dfadbb
--- a/src/HOL/Orderings.thy	Wed Mar 04 10:43:39 2009 +0100
+++ b/src/HOL/Orderings.thy	Wed Mar 04 10:45:52 2009 +0100
@@ -331,7 +331,7 @@
 
 fun struct_tac ((s, [eq, le, less]), thms) prems =
   let
-    fun decomp thy (Trueprop $ t) =
+    fun decomp thy (@{const Trueprop} $ t) =
       let
         fun excluded t =
           (* exclude numeric types: linear arithmetic subsumes transitivity *)
@@ -350,7 +350,8 @@
 	      of NONE => NONE
 	       | SOME (t1, rel, t2) => SOME (t1, "~" ^ rel, t2))
           | dec x = rel x;
-      in dec t end;
+      in dec t end
+      | decomp thy _ = NONE;
   in
     case s of
       "order" => Order_Tac.partial_tac decomp thms prems