src/CTT/ex/Synthesis.thy
changeset 69593 3dda49e08b9d
parent 65447 fae6051ec192
child 76377 2510e6f7b11c
equal deleted inserted replaced
69592:a80d8ec6c998 69593:3dda49e08b9d
    89   "?c : \<Sum>plus : ?A .
    89   "?c : \<Sum>plus : ?A .
    90          \<Prod>x:N. Eq(N, plus`0`x, x)
    90          \<Prod>x:N. Eq(N, plus`0`x, x)
    91                 \<times>  (\<Prod>y:N. Eq(N, plus`succ(y)`x, succ(plus`y`x)))"
    91                 \<times>  (\<Prod>y:N. Eq(N, plus`succ(y)`x, succ(plus`y`x)))"
    92 apply intr
    92 apply intr
    93 apply eqintr
    93 apply eqintr
    94 apply (tactic "resolve_tac @{context} [TSimp.split_eqn] 3")
    94 apply (tactic "resolve_tac \<^context> [TSimp.split_eqn] 3")
    95 apply (tactic "SELECT_GOAL (rew_tac @{context} []) 4")
    95 apply (tactic "SELECT_GOAL (rew_tac \<^context> []) 4")
    96 apply (tactic "resolve_tac @{context} [TSimp.split_eqn] 3")
    96 apply (tactic "resolve_tac \<^context> [TSimp.split_eqn] 3")
    97 apply (tactic "SELECT_GOAL (rew_tac @{context} []) 4")
    97 apply (tactic "SELECT_GOAL (rew_tac \<^context> []) 4")
    98 apply (rule_tac [3] p = "y" in NC_succ)
    98 apply (rule_tac [3] p = "y" in NC_succ)
    99   (**  by (resolve_tac @{context} comp_rls 3);  caused excessive branching  **)
    99   (**  by (resolve_tac @{context} comp_rls 3);  caused excessive branching  **)
   100 apply rew
   100 apply rew
   101 done
   101 done
   102 
   102