src/HOL/Statespace/state_fun.ML
changeset 45740 132a3e1c0fe5
parent 45661 ec6ba4b1f6d5
child 46218 ecf6375e2abb
--- a/src/HOL/Statespace/state_fun.ML	Fri Dec 02 14:37:25 2011 +0100
+++ b/src/HOL/Statespace/state_fun.ML	Fri Dec 02 14:54:25 2011 +0100
@@ -309,7 +309,7 @@
               val (eq, eT, nT, swap) = mkeq (dest_sel_eq t) 0;
               val prop =
                 list_all ([("n", nT), ("x", eT)],
-                  Logic.mk_equals (Const (@{const_name Ex}, Tex) $ Abs (s, T, eq), HOLogic.true_const));
+                  Logic.mk_equals (Const (@{const_name Ex}, Tex) $ Abs (s, T, eq), @{term True}));
               val thm = Drule.export_without_context (prove prop);
               val thm' = if swap then swap_ex_eq OF [thm] else thm
             in SOME thm' end handle TERM _ => NONE)