src/HOL/Codatatype/Tools/bnf_wrap.ML
changeset 49125 5fc5211cf104
parent 49123 263b0e330d8b
child 49129 b5413cb7d860
equal deleted inserted replaced
49124:968e1b7de057 49125:5fc5211cf104
   301           in
   301           in
   302             Skip_Proof.prove lthy [] [] goal (fn {context = ctxt, ...} =>
   302             Skip_Proof.prove lthy [] [] goal (fn {context = ctxt, ...} =>
   303               mk_not_other_disc_def_tac ctxt (nth disc_defs (2 - k)) (nth distinct_thms (2 - k))
   303               mk_not_other_disc_def_tac ctxt (nth disc_defs (2 - k)) (nth distinct_thms (2 - k))
   304                 exhaust_thm')
   304                 exhaust_thm')
   305             |> singleton (Proof_Context.export names_lthy lthy)
   305             |> singleton (Proof_Context.export names_lthy lthy)
       
   306             |> Thm.close_derivation
   306           end;
   307           end;
   307 
   308 
   308         val has_not_other_disc_def =
   309         val has_not_other_disc_def =
   309           exists (fn def => Thm.eq_thm_prop (def, missing_disc_def)) disc_defs;
   310           exists (fn def => Thm.eq_thm_prop (def, missing_disc_def)) disc_defs;
   310 
   311