src/Pure/Thy/term_style.ML
changeset 42360 da8817d01e7c
parent 42016 3b6826b3ed37
child 43277 1fd31f859fc7
--- a/src/Pure/Thy/term_style.ML	Sat Apr 16 15:25:25 2011 +0200
+++ b/src/Pure/Thy/term_style.ML	Sat Apr 16 15:47:52 2011 +0200
@@ -45,7 +45,7 @@
 
 fun parse_single ctxt = Parse.position (Parse.xname -- Args.parse)
   >> (fn x as ((name, _), _) => fst (Args.context_syntax "style"
-       (Scan.lift (the_style (ProofContext.theory_of ctxt) name))
+       (Scan.lift (the_style (Proof_Context.theory_of ctxt) name))
          (Args.src x) ctxt |>> (fn f => f ctxt)));
 
 val parse = Args.context :|-- (fn ctxt => Scan.lift 
@@ -56,7 +56,7 @@
 val parse_bare = Args.context :|-- (fn ctxt => (Output.legacy_feature "Old-style antiquotation style.";
   Scan.lift Args.liberal_name
   >> (fn name => fst (Args.context_syntax "style"
-       (Scan.lift (the_style (ProofContext.theory_of ctxt) name))
+       (Scan.lift (the_style (Proof_Context.theory_of ctxt) name))
           (Args.src (("style", []), Position.none)) ctxt |>> (fn f => f ctxt)))));
 
 
@@ -65,7 +65,7 @@
 fun style_lhs_rhs proj = Scan.succeed (fn ctxt => fn t =>
   let
     val concl =
-      Object_Logic.drop_judgment (ProofContext.theory_of ctxt) (Logic.strip_imp_concl t)
+      Object_Logic.drop_judgment (Proof_Context.theory_of ctxt) (Logic.strip_imp_concl t)
   in
     case concl of (_ $ l $ r) => proj (l, r)
     | _ => error ("Binary operator expected in term: " ^ Syntax.string_of_term ctxt concl)