src/FOL/FOL.thy
changeset 51687 3d8720271ebf
parent 48891 c0eafbd55de3
child 51717 9e7d1c139569
--- a/src/FOL/FOL.thy	Wed Apr 10 17:02:47 2013 +0200
+++ b/src/FOL/FOL.thy	Wed Apr 10 17:17:16 2013 +0200
@@ -181,24 +181,19 @@
 open Basic_Classical;
 *}
 
-setup {*
-  ML_Antiquote.value @{binding claset}
-    (Scan.succeed "Cla.claset_of ML_context")
-*}
-
 setup Cla.setup
 
 (*Propositional rules*)
 lemmas [intro!] = refl TrueI conjI disjCI impI notI iffI
   and [elim!] = conjE disjE impCE FalseE iffCE
-ML {* val prop_cs = @{claset} *}
+ML {* val prop_cs = claset_of @{context} *}
 
 (*Quantifier rules*)
 lemmas [intro!] = allI ex_ex1I
   and [intro] = exI
   and [elim!] = exE alt_ex1E
   and [elim] = allE
-ML {* val FOL_cs = @{claset} *}
+ML {* val FOL_cs = claset_of @{context} *}
 
 ML {*
   structure Blast = Blast