src/HOL/HOL.thy
changeset 69216 1a52baa70aed
parent 68979 e2244e5707dd
child 69593 3dda49e08b9d
equal deleted inserted replaced
69215:ab94035ba6ea 69216:1a52baa70aed
  1229         eq $ lhs $ rhs =>
  1229         eq $ lhs $ rhs =>
  1230           (case find_first (is_neq eq lhs rhs) (Simplifier.prems_of ss) of
  1230           (case find_first (is_neq eq lhs rhs) (Simplifier.prems_of ss) of
  1231             SOME thm => SOME (thm RS neq_to_EQ_False)
  1231             SOME thm => SOME (thm RS neq_to_EQ_False)
  1232           | NONE => NONE)
  1232           | NONE => NONE)
  1233        | _ => NONE);
  1233        | _ => NONE);
  1234   in proc end;
  1234   in proc end
  1235 \<close>
  1235 \<close>
  1236 
  1236 
  1237 simproc_setup let_simp ("Let x f") = \<open>
  1237 simproc_setup let_simp ("Let x f") = \<open>
  1238   let
  1238   let
  1239     fun count_loose (Bound i) k = if i >= k then 1 else 0
  1239     fun count_loose (Bound i) k = if i >= k then 1 else 0