src/HOL/Bali/Basis.thy
changeset 21314 6d709b9bea1a
parent 19323 ec5cd5b1804c
child 22578 b0eb5652f210
--- a/src/HOL/Bali/Basis.thy	Sun Nov 12 21:14:49 2006 +0100
+++ b/src/HOL/Bali/Basis.thy	Sun Nov 12 21:14:51 2006 +0100
@@ -185,12 +185,6 @@
 
 section "quantifiers"
 
-(*###to be phased out *)
-ML {* 
-fun noAll_simpset () = simpset() setmksimps 
-	mksimps (List.filter (fn (x,_) => x<>"All") mksimps_pairs)
-*}
-
 lemma All_Ex_refl_eq2 [simp]: 
  "(!x. (? b. x = f b & Q b) \<longrightarrow> P x) = (!b. Q b --> P (f b))"
 apply auto