equal
deleted
inserted
replaced
615 val facts = |
615 val facts = |
616 map2 (fn ((a, atts), _) => fn thms => ((a, map (prep_att lthy) atts), [(thms, [])])) |
616 map2 (fn ((a, atts), _) => fn thms => ((a, map (prep_att lthy) atts), [(thms, [])])) |
617 args thmss; |
617 args thmss; |
618 val (res, lthy') = lthy |> Local_Theory.notes facts |
618 val (res, lthy') = lthy |> Local_Theory.notes facts |
619 val _ = |
619 val _ = |
620 Proof_Display.print_results |
620 Proof_Display.print_results {interactive = int, pos = Position.thread_data ()} |
621 {interactive = int, pos = Position.thread_data (), proof_state = false} |
|
622 lthy' ((Thm.theoremK, ""), res); |
621 lthy' ((Thm.theoremK, ""), res); |
623 in (res, lthy') end; |
622 in (res, lthy') end; |
624 |
623 |
625 val inductive_cases = gen_inductive_cases (K I) Syntax.check_prop; |
624 val inductive_cases = gen_inductive_cases (K I) Syntax.check_prop; |
626 val inductive_cases_cmd = gen_inductive_cases Attrib.check_src Syntax.read_prop; |
625 val inductive_cases_cmd = gen_inductive_cases Attrib.check_src Syntax.read_prop; |
678 val facts = args |> map (fn ((a, atts), props) => |
677 val facts = args |> map (fn ((a, atts), props) => |
679 ((a, map (prep_att lthy) atts), |
678 ((a, map (prep_att lthy) atts), |
680 map (Thm.no_attributes o single o mk_simp_eq lthy o prep_prop lthy) props)); |
679 map (Thm.no_attributes o single o mk_simp_eq lthy o prep_prop lthy) props)); |
681 val (res, lthy') = lthy |> Local_Theory.notes facts |
680 val (res, lthy') = lthy |> Local_Theory.notes facts |
682 val _ = |
681 val _ = |
683 Proof_Display.print_results |
682 Proof_Display.print_results {interactive = int, pos = Position.thread_data ()} |
684 {interactive = int, pos = Position.thread_data (), proof_state = false} |
|
685 lthy' ((Thm.theoremK, ""), res) |
683 lthy' ((Thm.theoremK, ""), res) |
686 in (res, lthy') end; |
684 in (res, lthy') end; |
687 |
685 |
688 val inductive_simps = gen_inductive_simps (K I) Syntax.check_prop; |
686 val inductive_simps = gen_inductive_simps (K I) Syntax.check_prop; |
689 val inductive_simps_cmd = gen_inductive_simps Attrib.check_src Syntax.read_prop; |
687 val inductive_simps_cmd = gen_inductive_simps Attrib.check_src Syntax.read_prop; |