src/Pure/Isar/local_defs.ML
changeset 10464 b7b916a82dca
parent 9467 52fb37876254
child 11718 92706a69dacc
equal deleted inserted replaced
10463:474263d29057 10464:b7b916a82dca
    61     val lhs = ProofContext.bind_skolem ctxt [x] (Free (x, T));
    61     val lhs = ProofContext.bind_skolem ctxt [x] (Free (x, T));
    62   in
    62   in
    63     state
    63     state
    64     |> fix [([x], None)]
    64     |> fix [([x], None)]
    65     |> Proof.match_bind_i [(pats, rhs)]
    65     |> Proof.match_bind_i [(pats, rhs)]
    66     |> Proof.assm_i export_defs [(name, atts, [(Logic.mk_equals (lhs, rhs), ([], []))])]
    66     |> Proof.assm_i export_defs [((name, atts), [(Logic.mk_equals (lhs, rhs), ([], []))])]
    67   end;
    67   end;
    68 
    68 
    69 val def = gen_def Proof.fix ProofContext.read_term ProofContext.read_term_pats;
    69 val def = gen_def Proof.fix ProofContext.read_term ProofContext.read_term_pats;
    70 val def_i = gen_def Proof.fix_i ProofContext.cert_term ProofContext.cert_term_pats;
    70 val def_i = gen_def Proof.fix_i ProofContext.cert_term ProofContext.cert_term_pats;
    71 
    71