src/Pure/Isar/class.ML
changeset 51551 88d1d19fb74f
parent 51510 b4f7e6734acc
child 51578 969ad6538b8f
equal deleted inserted replaced
51550:cec08df2c030 51551:88d1d19fb74f
   249   let
   249   let
   250     val intros = (snd o rules thy) sup :: map_filter I
   250     val intros = (snd o rules thy) sup :: map_filter I
   251       [Option.map (Drule.export_without_context_open o Element.conclude_witness) some_wit,
   251       [Option.map (Drule.export_without_context_open o Element.conclude_witness) some_wit,
   252         (fst o rules thy) sub];
   252         (fst o rules thy) sub];
   253     val classrel =
   253     val classrel =
   254       Skip_Proof.prove_global thy [] [] (Logic.mk_classrel (sub, sup))
   254       Goal.prove_sorry_global thy [] [] (Logic.mk_classrel (sub, sup))
   255         (K (EVERY (map (TRYALL o Tactic.rtac) intros)));
   255         (K (EVERY (map (TRYALL o Tactic.rtac) intros)));
   256     val diff_sort = Sign.complete_sort thy [sup]
   256     val diff_sort = Sign.complete_sort thy [sup]
   257       |> subtract (op =) (Sign.complete_sort thy [sub])
   257       |> subtract (op =) (Sign.complete_sort thy [sub])
   258       |> filter (is_class thy);
   258       |> filter (is_class thy);
   259     val add_dependency =
   259     val add_dependency =