src/HOL/TLA/Action.thy
changeset 69597 ff784d5a5bfb
parent 62146 324bc1ffba12
equal deleted inserted replaced
69596:c8a2755bf220 69597:ff784d5a5bfb
   112 (* Turn  \<turnstile> A = B  into meta-level rewrite rule  A == B *)
   112 (* Turn  \<turnstile> A = B  into meta-level rewrite rule  A == B *)
   113 val action_rewrite = int_rewrite
   113 val action_rewrite = int_rewrite
   114 
   114 
   115 fun action_use ctxt th =
   115 fun action_use ctxt th =
   116     case Thm.concl_of th of
   116     case Thm.concl_of th of
   117       Const _ $ (Const (@{const_name Valid}, _) $ _) =>
   117       Const _ $ (Const (\<^const_name>\<open>Valid\<close>, _) $ _) =>
   118               (flatten (action_unlift ctxt th) handle THM _ => th)
   118               (flatten (action_unlift ctxt th) handle THM _ => th)
   119     | _ => th;
   119     | _ => th;
   120 \<close>
   120 \<close>
   121 
   121 
   122 attribute_setup action_unlift =
   122 attribute_setup action_unlift =