src/Doc/Implementation/Logic.thy
changeset 61962 9c8fc56032e3
parent 61854 38b049cd3aad
child 62363 7b5468422352
equal deleted inserted replaced
61961:c4cc05200337 61962:9c8fc56032e3
  1009   and sub-problems. Branches are closed either by resolving with a rule of 0
  1009   and sub-problems. Branches are closed either by resolving with a rule of 0
  1010   premises, or by producing a ``short-circuit'' within a solved situation
  1010   premises, or by producing a ``short-circuit'' within a solved situation
  1011   (again modulo unification):
  1011   (again modulo unification):
  1012   \[
  1012   \[
  1013   \infer[(@{inference_def assumption})]{\<open>C\<vartheta>\<close>}
  1013   \infer[(@{inference_def assumption})]{\<open>C\<vartheta>\<close>}
  1014   {\<open>(\<And>\<^vec>x. \<^vec>H \<^vec>x \<Longrightarrow> A \<^vec>x) \<Longrightarrow> C\<close> & \<open>A\<vartheta> = H\<^sub>i\<vartheta>\<close>~~\text{(for some~\<open>i\<close>)}}
  1014   {\<open>(\<And>\<^vec>x. \<^vec>H \<^vec>x \<Longrightarrow> A \<^vec>x) \<Longrightarrow> C\<close> & \<open>A\<vartheta> = H\<^sub>i\<vartheta>\<close>~~\mbox{(for some~\<open>i\<close>)}}
  1015   \]
  1015   \]
  1016 
  1016 
  1017   %FIXME @{inference_def elim_resolution}, @{inference_def dest_resolution}
  1017   %FIXME @{inference_def elim_resolution}, @{inference_def dest_resolution}
  1018 \<close>
  1018 \<close>
  1019 
  1019