src/Pure/Tools/class_package.ML
changeset 19585 70a1ce3b23ae
parent 19575 2d9940cd52d3
child 19648 702843484da6
equal deleted inserted replaced
19584:606d6a73e6d9 19585:70a1ce3b23ae
   299 
   299 
   300 fun gen_instance mk_prop add_thm after_qed inst thy =
   300 fun gen_instance mk_prop add_thm after_qed inst thy =
   301   thy
   301   thy
   302   |> ProofContext.init
   302   |> ProofContext.init
   303   |> Proof.theorem_i PureThy.internalK NONE (after_qed oo (fold o fold) add_thm) NONE ("", [])
   303   |> Proof.theorem_i PureThy.internalK NONE (after_qed oo (fold o fold) add_thm) NONE ("", [])
   304        (map (fn t => (("", []), [(t, ([], []))])) (mk_prop thy inst));
   304        (map (fn t => (("", []), [(t, [])])) (mk_prop thy inst));
   305 
   305 
   306 in
   306 in
   307 
   307 
   308 val axclass_instance_subclass =
   308 val axclass_instance_subclass =
   309   gen_instance (single oo (Logic.mk_classrel oo AxClass.read_classrel)) AxClass.add_classrel I;
   309   gen_instance (single oo (Logic.mk_classrel oo AxClass.read_classrel)) AxClass.add_classrel I;