equal
deleted
inserted
replaced
86 "print_interps" "print_attributes" |
86 "print_interps" "print_attributes" |
87 "print_simpset" "print_rules" "print_trans_rules" "print_methods" |
87 "print_simpset" "print_rules" "print_trans_rules" "print_methods" |
88 "print_antiquotations" "print_ML_antiquotations" "thy_deps" |
88 "print_antiquotations" "print_ML_antiquotations" "thy_deps" |
89 "locale_deps" "class_deps" "thm_deps" "thm_oracles" "print_term_bindings" |
89 "locale_deps" "class_deps" "thm_deps" "thm_oracles" "print_term_bindings" |
90 "print_facts" "print_cases" "print_statement" "thm" "prf" "full_prf" |
90 "print_facts" "print_cases" "print_statement" "thm" "prf" "full_prf" |
91 "prop" "term" "typ" "print_codesetup" "unused_thms" :: diag |
91 "prop" "term" "typ" "print_codesetup" "print_context_tracing" "unused_thms" :: diag |
92 and "print_state" :: diag |
92 and "print_state" :: diag |
93 and "welcome" :: diag |
93 and "welcome" :: diag |
94 and "end" :: thy_end |
94 and "end" :: thy_end |
95 and "realizers" :: thy_decl |
95 and "realizers" :: thy_decl |
96 and "realizability" :: thy_decl |
96 and "realizability" :: thy_decl |
1297 val _ = |
1297 val _ = |
1298 Outer_Syntax.command \<^command_keyword>\<open>print_codesetup\<close> "print code generator setup" |
1298 Outer_Syntax.command \<^command_keyword>\<open>print_codesetup\<close> "print code generator setup" |
1299 (Scan.succeed (Toplevel.keep (Code.print_codesetup o Toplevel.theory_of))); |
1299 (Scan.succeed (Toplevel.keep (Code.print_codesetup o Toplevel.theory_of))); |
1300 |
1300 |
1301 val _ = |
1301 val _ = |
|
1302 Outer_Syntax.command \<^command_keyword>\<open>print_context_tracing\<close> |
|
1303 "print result of context tracing from ML heap" |
|
1304 (Scan.succeed (Toplevel.keep (fn _ => Session.print_context_tracing (K true)))); |
|
1305 |
|
1306 val _ = |
1302 Outer_Syntax.command \<^command_keyword>\<open>print_state\<close> |
1307 Outer_Syntax.command \<^command_keyword>\<open>print_state\<close> |
1303 "print current proof state (if present)" |
1308 "print current proof state (if present)" |
1304 (opt_modes >> (fn modes => |
1309 (opt_modes >> (fn modes => |
1305 Toplevel.keep (Print_Mode.with_modes modes (Output.writeln o Toplevel.string_of_state)))); |
1310 Toplevel.keep (Print_Mode.with_modes modes (Output.writeln o Toplevel.string_of_state)))); |
1306 |
1311 |