src/HOL/Library/Euclidean_Space.thy
changeset 30510 4120fc59dd85
parent 30489 5d7d0add1741
child 30549 d2d7874648bd
--- a/src/HOL/Library/Euclidean_Space.thy	Fri Mar 13 19:53:09 2009 +0100
+++ b/src/HOL/Library/Euclidean_Space.thy	Fri Mar 13 19:58:26 2009 +0100
@@ -134,7 +134,7 @@
    (* THEN' TRY o clarify_tac HOL_cs  THEN' (TRY o rtac @{thm iffI}) *)
    THEN' asm_full_simp_tac (ss2 addsimps ths)
  in
-  Method.thms_args (Method.SIMPLE_METHOD' o vector_arith_tac)
+  Method.thms_args (SIMPLE_METHOD' o vector_arith_tac)
 end
 *} "Lifts trivial vector statements to real arith statements"
 
@@ -948,7 +948,7 @@
 
 use "normarith.ML"
 
-method_setup norm = {* Method.ctxt_args (Method.SIMPLE_METHOD' o NormArith.norm_arith_tac)
+method_setup norm = {* Method.ctxt_args (SIMPLE_METHOD' o NormArith.norm_arith_tac)
 *} "Proves simple linear statements about vector norms"