src/HOL/Statespace/state_space.ML
changeset 41270 dea60d052923
parent 39134 917b4b6ba3d2
child 41472 f6ab14e61604
equal deleted inserted replaced
41269:abe867c29e55 41270:dea60d052923
   143 
   143 
   144 val get_silent = #silent o NameSpaceData.get;
   144 val get_silent = #silent o NameSpaceData.get;
   145 
   145 
   146 fun prove_interpretation_in ctxt_tac (name, expr) thy =
   146 fun prove_interpretation_in ctxt_tac (name, expr) thy =
   147    thy
   147    thy
   148    |> Expression.sublocale_cmd name expr
   148    |> Expression.sublocale_cmd name expr []
   149    |> Proof.global_terminal_proof
   149    |> Proof.global_terminal_proof
   150          (Method.Basic (fn ctxt => SIMPLE_METHOD (ctxt_tac ctxt)), NONE)
   150          (Method.Basic (fn ctxt => SIMPLE_METHOD (ctxt_tac ctxt)), NONE)
   151    |> ProofContext.theory_of
   151    |> ProofContext.theory_of
   152 
   152 
   153 fun add_locale name expr elems thy =
   153 fun add_locale name expr elems thy =