src/ZF/UNITY/Constrains.thy
changeset 54742 7a86358a3c0b
parent 51717 9e7d1c139569
child 57945 cacb00a569e0
equal deleted inserted replaced
54741:010eefa0a4f3 54742:7a86358a3c0b
   477                       ORELSE
   477                       ORELSE
   478                       resolve_tac [@{thm StableI}, @{thm stableI},
   478                       resolve_tac [@{thm StableI}, @{thm stableI},
   479                                    @{thm constrains_imp_Constrains}] 1),
   479                                    @{thm constrains_imp_Constrains}] 1),
   480               rtac @{thm constrainsI} 1,
   480               rtac @{thm constrainsI} 1,
   481               (* Three subgoals *)
   481               (* Three subgoals *)
   482               rewrite_goal_tac [@{thm st_set_def}] 3,
   482               rewrite_goal_tac ctxt [@{thm st_set_def}] 3,
   483               REPEAT (force_tac ctxt 2),
   483               REPEAT (force_tac ctxt 2),
   484               full_simp_tac (ctxt addsimps (Program_Defs.get ctxt)) 1,
   484               full_simp_tac (ctxt addsimps (Program_Defs.get ctxt)) 1,
   485               ALLGOALS (clarify_tac ctxt),
   485               ALLGOALS (clarify_tac ctxt),
   486               REPEAT (FIRSTGOAL (etac @{thm disjE})),
   486               REPEAT (FIRSTGOAL (etac @{thm disjE})),
   487               ALLGOALS (clarify_tac ctxt),
   487               ALLGOALS (clarify_tac ctxt),