src/HOL/HOL.thy
changeset 39782 f75381bc46d2
parent 39722 4a4086908382
child 40222 cd6d2b0a4096
--- a/src/HOL/HOL.thy	Wed Sep 29 10:05:44 2010 +0200
+++ b/src/HOL/HOL.thy	Wed Sep 29 11:02:24 2010 +0200
@@ -834,8 +834,6 @@
   val subst = @{thm subst}
   val sym = @{thm sym}
   val thin_refl = @{thm thin_refl};
-  val prop_subst = @{lemma "PROP P t ==> PROP prop (x = t ==> PROP P x)"
-                     by (unfold prop_def) (drule eq_reflection, unfold)}
 end);
 open Hypsubst;