src/CCL/Wfd.thy
changeset 74375 ba880f3a4e52
parent 74298 45a77ee63e57
child 74563 042041c0ebeb
equal deleted inserted replaced
74374:e585e5a906ba 74375:ba880f3a4e52
   439             tac [((("g", 0), Position.none), x)] (nth rls (y - 1)) i ORELSE (try_IHs xs)
   439             tac [((("g", 0), Position.none), x)] (nth rls (y - 1)) i ORELSE (try_IHs xs)
   440   in try_IHs rnames end)
   440   in try_IHs rnames end)
   441 
   441 
   442 fun is_rigid_prog t =
   442 fun is_rigid_prog t =
   443   (case (Logic.strip_assums_concl t) of
   443   (case (Logic.strip_assums_concl t) of
   444     \<^Const_>\<open>Trueprop for \<open>\<^Const_>\<open>mem _ for a _\<close>\<close>\<close> => null (Term.add_vars a [])
   444     \<^Const_>\<open>Trueprop for \<^Const_>\<open>mem _ for a _\<close>\<close> => null (Term.add_vars a [])
   445   | _ => false)
   445   | _ => false)
   446 
   446 
   447 in
   447 in
   448 
   448 
   449 fun rcall_tac ctxt i =
   449 fun rcall_tac ctxt i =