src/HOL/Topological_Spaces.thy
changeset 59582 0fbed69ff081
parent 59452 2538b2c51769
child 59970 e9f73d87d904
equal deleted inserted replaced
59580:cbc38731d42f 59582:0fbed69ff081
   449       val mp_thms = thms RL [@{thm eventually_rev_mp}]
   449       val mp_thms = thms RL [@{thm eventually_rev_mp}]
   450       val raw_elim_thm =
   450       val raw_elim_thm =
   451         (@{thm allI} RS @{thm always_eventually})
   451         (@{thm allI} RS @{thm always_eventually})
   452         |> fold (fn thm1 => fn thm2 => thm2 RS thm1) mp_thms
   452         |> fold (fn thm1 => fn thm2 => thm2 RS thm1) mp_thms
   453         |> fold (fn _ => fn thm => @{thm impI} RS thm) thms
   453         |> fold (fn _ => fn thm => @{thm impI} RS thm) thms
   454       val cases_prop = prop_of (raw_elim_thm RS st)
   454       val cases_prop = Thm.prop_of (raw_elim_thm RS st)
   455       val cases = (Rule_Cases.make_common (thy, cases_prop) [(("elim", []), [])])
   455       val cases = (Rule_Cases.make_common (thy, cases_prop) [(("elim", []), [])])
   456     in
   456     in
   457       CASES cases (rtac raw_elim_thm 1)
   457       CASES cases (rtac raw_elim_thm 1)
   458     end) 1
   458     end) 1
   459 *}
   459 *}