src/ZF/equalities.thy
changeset 42793 88bee9f6eec7
parent 35762 af3ff2ba4c54
child 45602 2a858377c3d2
--- a/src/ZF/equalities.thy	Fri May 13 16:03:03 2011 +0200
+++ b/src/ZF/equalities.thy	Fri May 13 22:55:00 2011 +0200
@@ -970,17 +970,14 @@
                     Un_upper1 Un_upper2 Int_lower1 Int_lower2
 
 ML {*
-val subset_cs = @{claset} 
+val subset_cs =
+  claset_of (@{context}
     delrules [@{thm subsetI}, @{thm subsetCE}]
     addSIs @{thms subset_SIs}
     addIs  [@{thm Union_upper}, @{thm Inter_lower}]
-    addSEs [@{thm cons_subsetE}];
-*}
-(*subset_cs is a claset for subset reasoning*)
+    addSEs [@{thm cons_subsetE}]);
 
-ML
-{*
-val ZF_cs = @{claset} delrules [@{thm equalityI}];
+val ZF_cs = claset_of (@{context} delrules [@{thm equalityI}]);
 *}
  
 end