src/HOL/Statespace/state_space.ML
changeset 61669 27ca6147e3b3
parent 61606 6d5213bd9709
child 61673 fd4ac1530d63
equal deleted inserted replaced
61668:9a51e4dfc5d9 61669:27ca6147e3b3
   125 fun expression_no_pos (expr, fixes) : Expression.expression =
   125 fun expression_no_pos (expr, fixes) : Expression.expression =
   126   (map (fn (name, inst) => ((name, Position.none), inst)) expr, fixes);
   126   (map (fn (name, inst) => ((name, Position.none), inst)) expr, fixes);
   127 
   127 
   128 fun prove_interpretation_in ctxt_tac (name, expr) thy =
   128 fun prove_interpretation_in ctxt_tac (name, expr) thy =
   129    thy
   129    thy
   130    |> Expression.sublocale_global_cmd (name, Position.none) (expression_no_pos expr) []
   130    |> Interpretation.sublocale_global_cmd (name, Position.none) (expression_no_pos expr) []
   131    |> Proof.global_terminal_proof
   131    |> Proof.global_terminal_proof
   132          ((Method.Basic (fn ctxt => SIMPLE_METHOD (ctxt_tac ctxt)), Position.no_range), NONE)
   132          ((Method.Basic (fn ctxt => SIMPLE_METHOD (ctxt_tac ctxt)), Position.no_range), NONE)
   133    |> Proof_Context.theory_of
   133    |> Proof_Context.theory_of
   134 
   134 
   135 fun add_locale name expr elems thy =
   135 fun add_locale name expr elems thy =