src/HOL/Library/RType.thy
changeset 28083 103d9282a946
parent 27487 c8a6ce181805
child 28084 a05ca48ef263
equal deleted inserted replaced
28082:37350f301128 28083:103d9282a946
    65     val eq = HOLogic.mk_Trueprop (HOLogic.mk_eq (lhs, rhs));
    65     val eq = HOLogic.mk_Trueprop (HOLogic.mk_eq (lhs, rhs));
    66   in
    66   in
    67     thy
    67     thy
    68     |> TheoryTarget.instantiation ([tyco], vs, @{sort rtype})
    68     |> TheoryTarget.instantiation ([tyco], vs, @{sort rtype})
    69     |> `(fn lthy => Syntax.check_term lthy eq)
    69     |> `(fn lthy => Syntax.check_term lthy eq)
    70     |-> (fn eq => Specification.definition (NONE, (("", []), eq)))
    70     |-> (fn eq => Specification.definition (NONE, ((Name.no_binding, []), eq)))
    71     |> snd
    71     |> snd
    72     |> Class.prove_instantiation_instance (K (Class.intro_classes_tac []))
    72     |> Class.prove_instantiation_instance (K (Class.intro_classes_tac []))
    73     |> LocalTheory.exit
    73     |> LocalTheory.exit
    74     |> ProofContext.theory_of
    74     |> ProofContext.theory_of
    75   end;
    75   end;