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