src/HOL/Import/import_rule.ML
changeset 70303 502749883f53
parent 69829 3bfa28b3a5b2
child 74282 c2ee8d993d6a
equal deleted inserted replaced
70302:9ea7081c3f03 70303:502749883f53
   371           getth th1 tstate ||>> getth th2 |>> (fn (t1, t2) => deduct t1 t2) |-> setth
   371           getth th1 tstate ||>> getth th2 |>> (fn (t1, t2) => deduct t1 t2) |-> setth
   372       | process tstate (#"L", [t, th]) =
   372       | process tstate (#"L", [t, th]) =
   373           gettm t tstate ||>> (fn ti => getth th ti) |>> (fn (tm, th) => abs tm th) |-> setth
   373           gettm t tstate ||>> (fn ti => getth th ti) |>> (fn (tm, th) => abs tm th) |-> setth
   374       | process (thy, state) (#"M", [s]) =
   374       | process (thy, state) (#"M", [s]) =
   375           let
   375           let
   376             val ctxt = Variable.set_body false (Proof_Context.init_global thy)
   376             val ctxt = Proof_Context.init_global thy
   377             val thm = freezeT thy (Global_Theory.get_thm thy s)
   377             val thm = freezeT thy (Global_Theory.get_thm thy s)
   378             val ((_, [th']), _) = Variable.import true [thm] ctxt
   378             val ((_, [th']), _) = Variable.import true [thm] ctxt
   379           in
   379           in
   380             setth th' (thy, state)
   380             setth th' (thy, state)
   381           end
   381           end