paulson [Mon, 23 Jan 2006 11:41:54 +0100] rev 18753
ResClasimp.get_clasimp_lemmas now takes all subgoals rather than only the first
paulson [Mon, 23 Jan 2006 11:38:43 +0100] rev 18752
Clausification now handles some IFs in rewrite rules (if-split did not work)
paulson [Mon, 23 Jan 2006 11:37:53 +0100] rev 18751
bugfix: induct_tac no longer raises THM "dest_state"
paulson [Mon, 23 Jan 2006 11:36:50 +0100] rev 18750
fixed the <<= notation
paulson [Mon, 23 Jan 2006 11:36:05 +0100] rev 18749
replacement of bool by a datatype (making problems first-order). More lemma names
mengj [Mon, 23 Jan 2006 10:34:38 +0100] rev 18748
Fixed a bug.
urbanc [Sun, 22 Jan 2006 22:16:34 +0100] rev 18747
no essential changes
urbanc [Sun, 22 Jan 2006 22:11:50 +0100] rev 18746
made the change for setup-functions not returning functions
anymore
urbanc [Sun, 22 Jan 2006 21:58:43 +0100] rev 18745
a fixme comments about abs_fun_if, which should be called perm_if
and moved to the "bool"-section
wenzelm [Sun, 22 Jan 2006 18:46:01 +0100] rev 18744
Local theory operations, with optional target locale.
wenzelm [Sun, 22 Jan 2006 18:46:00 +0100] rev 18743
added restore_body;
wenzelm [Sun, 22 Jan 2006 18:45:59 +0100] rev 18742
added the_params;
wenzelm [Sun, 22 Jan 2006 18:45:58 +0100] rev 18741
tuned order;
wenzelm [Sun, 22 Jan 2006 18:45:57 +0100] rev 18740
added Isar/local_theory.ML;
mengj [Sat, 21 Jan 2006 23:22:40 +0100] rev 18739
Ensure dereference is delayed.
wenzelm [Sat, 21 Jan 2006 23:07:26 +0100] rev 18738
tuned;
wenzelm [Sat, 21 Jan 2006 23:02:30 +0100] rev 18737
* ML: simplified type attribute;
wenzelm [Sat, 21 Jan 2006 23:02:29 +0100] rev 18736
simplified type attribute;
removed obsolete tcset operations -- clean data/attribute/method setup;
wenzelm [Sat, 21 Jan 2006 23:02:28 +0100] rev 18735
removed duplicate type_solver (cf. Tools/typechk.ML);
wenzelm [Sat, 21 Jan 2006 23:02:27 +0100] rev 18734
simplified type attribute;
removed rule/declaration (cf. thm.ML);
removed obsolete theory/proof/generic/common;
removed obsolete global/local/context_attribute(_i);
added attribute(_i);
renamed attribute to internal;
wenzelm [Sat, 21 Jan 2006 23:02:25 +0100] rev 18733
simplified type attribute;
added rule/declaration_attribute (from drule.ML);
added theory/proof_attributes;
removed apply(s)_attributes;
wenzelm [Sat, 21 Jan 2006 23:02:24 +0100] rev 18732
simplified type attribute;
moved rule/declaration_attribute to thm.ML;
wenzelm [Sat, 21 Jan 2006 23:02:23 +0100] rev 18731
rename map_theory/proof to theory/proof_map;
added separate map_theory/proof;
wenzelm [Sat, 21 Jan 2006 23:02:21 +0100] rev 18730
tuned proofs;
wenzelm [Sat, 21 Jan 2006 23:02:20 +0100] rev 18729
simplified type attribute;
tuned;
wenzelm [Sat, 21 Jan 2006 23:02:14 +0100] rev 18728
simplified type attribute;
mengj [Fri, 20 Jan 2006 04:53:59 +0100] rev 18727
type information is now also printed.
mengj [Fri, 20 Jan 2006 04:50:01 +0100] rev 18726
added some debugging code.
mengj [Fri, 20 Jan 2006 04:35:23 +0100] rev 18725
fixed a bug
wenzelm [Thu, 19 Jan 2006 21:22:30 +0100] rev 18724
quote "atom";
wenzelm [Thu, 19 Jan 2006 21:22:29 +0100] rev 18723
updated;
wenzelm [Thu, 19 Jan 2006 21:22:27 +0100] rev 18722
* ML/Isar: theory setup has type (theory -> theory);
wenzelm [Thu, 19 Jan 2006 21:22:26 +0100] rev 18721
use/use_thy: Output.toplevel_errors;
wenzelm [Thu, 19 Jan 2006 21:22:25 +0100] rev 18720
added basic syntax;
removed pure syntax;
wenzelm [Thu, 19 Jan 2006 21:22:24 +0100] rev 18719
moved pure syntax to Syntax/syntax.ML and pure_thy.ML;
wenzelm [Thu, 19 Jan 2006 21:22:23 +0100] rev 18718
keep: disable Output.toplevel_errors;
program: Output.ML_errors;
wenzelm [Thu, 19 Jan 2006 21:22:22 +0100] rev 18717
run_thy: removed Output.toplevel_errors;
wenzelm [Thu, 19 Jan 2006 21:22:21 +0100] rev 18716
added ML_errors;
wenzelm [Thu, 19 Jan 2006 21:22:20 +0100] rev 18715
use: Output.ML_errors;
wenzelm [Thu, 19 Jan 2006 21:22:19 +0100] rev 18714
Syntax.basic_syn;
wenzelm [Thu, 19 Jan 2006 21:22:18 +0100] rev 18713
setup: theory -> theory;
added syntax (from Syntax/mixfix.ML);
added HTML output syntax for _lambda;
wenzelm [Thu, 19 Jan 2006 21:22:17 +0100] rev 18712
tuned setmp;
wenzelm [Thu, 19 Jan 2006 21:22:16 +0100] rev 18711
setup: theory -> theory;
use_output: Output.ML_errors;
wenzelm [Thu, 19 Jan 2006 21:22:15 +0100] rev 18710
tuned comments;
wenzelm [Thu, 19 Jan 2006 21:22:14 +0100] rev 18709
setup: theory -> theory;
Syntax.appl(C)_syntax;
wenzelm [Thu, 19 Jan 2006 21:22:08 +0100] rev 18708
setup: theory -> theory;
berghofe [Thu, 19 Jan 2006 15:45:10 +0100] rev 18707
Use generic Simplifier.simp_add attribute instead
of Simplifier.simp_add_global.
berghofe [Thu, 19 Jan 2006 14:59:55 +0100] rev 18706
Re-inserted consts_code declaration accidentally deleted
during last commit.
paulson [Thu, 19 Jan 2006 10:22:13 +0100] rev 18705
strengthened some lemmas; simplified some proofs
haftmann [Wed, 18 Jan 2006 11:55:50 +0100] rev 18704
substantial improvement in serialization handling
urbanc [Wed, 18 Jan 2006 02:48:58 +0100] rev 18703
fixed one proof that broke because of the changes
Markus did on the rules ex1I
haftmann [Tue, 17 Jan 2006 16:36:57 +0100] rev 18702
substantial improvements in code generator
paulson [Tue, 17 Jan 2006 10:26:50 +0100] rev 18701
these hacks are no longer needed
paulson [Tue, 17 Jan 2006 10:26:36 +0100] rev 18700
improved SPASS support
wenzelm [Mon, 16 Jan 2006 21:55:17 +0100] rev 18699
case_result: drop_schematic, i.e. be permissive about illegal binds;
wenzelm [Mon, 16 Jan 2006 21:55:15 +0100] rev 18698
put_facts: do not pretend local thms were named;
wenzelm [Mon, 16 Jan 2006 21:55:14 +0100] rev 18697
declare the1_equality [elim?];
wenzelm [Sun, 15 Jan 2006 20:04:05 +0100] rev 18696
tuned;
wenzelm [Sun, 15 Jan 2006 20:00:59 +0100] rev 18695
tuned;
wenzelm [Sun, 15 Jan 2006 19:58:57 +0100] rev 18694
* Classical: optional weight for attributes;
* HOL: prefer ex1I over ex_ex1I in single-step reasoning;
wenzelm [Sun, 15 Jan 2006 19:58:56 +0100] rev 18693
guess: used fixed inferred_type of vars;
wenzelm [Sun, 15 Jan 2006 19:58:55 +0100] rev 18692
export add_args;
tuned;
wenzelm [Sun, 15 Jan 2006 19:58:54 +0100] rev 18691
attributes: optional weight;
tuned;
wenzelm [Sun, 15 Jan 2006 19:58:53 +0100] rev 18690
classical attributes: optional weight;
wenzelm [Sun, 15 Jan 2006 19:58:51 +0100] rev 18689
prefer ex1I over ex_ex1I in single-step reasoning;
wenzelm [Sat, 14 Jan 2006 22:25:34 +0100] rev 18688
generic attributes;
wenzelm [Sat, 14 Jan 2006 17:20:51 +0100] rev 18687
tuned;
wenzelm [Sat, 14 Jan 2006 17:15:24 +0100] rev 18686
* ML/Isar: simplified treatment of user-level errors;
wenzelm [Sat, 14 Jan 2006 17:14:18 +0100] rev 18685
sane ERROR vs. TOPLEVEL_ERROR handling;
added program;
wenzelm [Sat, 14 Jan 2006 17:14:17 +0100] rev 18684
added Isar.toplevel;
wenzelm [Sat, 14 Jan 2006 17:14:16 +0100] rev 18683
Output.error_msg;
wenzelm [Sat, 14 Jan 2006 17:14:15 +0100] rev 18682
removed special ERROR handling stuff (transform_error etc.);
moved plain ERROR/error to library.ML;
added toplevel_errors, exception TOPLEVEL_ERROR;
error_msg, panic, info, debug no longer pervasive;
wenzelm [Sat, 14 Jan 2006 17:14:14 +0100] rev 18681
added exception ERROR, error, cat_error, sys_error, assert, deny, assert_all;
added transform_failure;
added prefix;
wenzelm [Sat, 14 Jan 2006 17:14:13 +0100] rev 18680
Output.debug;
wenzelm [Sat, 14 Jan 2006 17:14:11 +0100] rev 18679
generated code: raise Match instead of ERROR;
wenzelm [Sat, 14 Jan 2006 17:14:06 +0100] rev 18678
sane ERROR handling;
paulson [Fri, 13 Jan 2006 17:39:41 +0100] rev 18677
blacklist experiments
paulson [Fri, 13 Jan 2006 17:39:19 +0100] rev 18676
more readable divide ops
paulson [Fri, 13 Jan 2006 17:39:03 +0100] rev 18675
more practical time limit
nipkow [Fri, 13 Jan 2006 14:43:09 +0100] rev 18674
*** empty log message ***
wenzelm [Fri, 13 Jan 2006 01:13:17 +0100] rev 18673
mixfix: added Structure;
wenzelm [Fri, 13 Jan 2006 01:13:16 +0100] rev 18672
uniform handling of fixes: read/cert_vars, add_fixes(_i), body flag;
mixfix: added Structure;
renamed type exporter to export;
removed obsolete sign_of;
tuned signature;
tuned;
wenzelm [Fri, 13 Jan 2006 01:13:15 +0100] rev 18671
uniform handling of fixes;
mixfix: added Structure;
tuned;
wenzelm [Fri, 13 Jan 2006 01:13:11 +0100] rev 18670
uniform handling of fixes;
wenzelm [Fri, 13 Jan 2006 01:13:08 +0100] rev 18669
uniform handling of fixes;
mixfix: added Structure;
wenzelm [Fri, 13 Jan 2006 01:13:06 +0100] rev 18668
uniform handling of fixes;
tuned;
wenzelm [Fri, 13 Jan 2006 01:13:05 +0100] rev 18667
tuned;
wenzelm [Fri, 13 Jan 2006 01:13:03 +0100] rev 18666
generic_setup: optional argument, defaults to Context.setup();
wenzelm [Fri, 13 Jan 2006 01:13:02 +0100] rev 18665
added map_theory, map_proof;
wenzelm [Fri, 13 Jan 2006 01:13:00 +0100] rev 18664
removed obsolete sign_of;
wenzelm [Fri, 13 Jan 2006 01:12:59 +0100] rev 18663
implicit setup, which admits exception_trace;
wenzelm [Fri, 13 Jan 2006 01:12:58 +0100] rev 18662
ProofContext.def_export;
urbanc [Wed, 11 Jan 2006 18:46:31 +0100] rev 18661
updated to new induction principle
urbanc [Wed, 11 Jan 2006 18:39:19 +0100] rev 18660
cahges to use the new induction-principle (now proved in
full glory)
urbanc [Wed, 11 Jan 2006 18:38:32 +0100] rev 18659
changes to make use of the new induction principle proved by
Stefan horay (hooraayyy)
berghofe [Wed, 11 Jan 2006 18:21:23 +0100] rev 18658
Implemented proof of (strong) induction rule.
berghofe [Wed, 11 Jan 2006 18:20:59 +0100] rev 18657
Added theorem at_finite_select.
urbanc [Wed, 11 Jan 2006 17:12:30 +0100] rev 18656
added lemmas perm_empty, perm_insert to do with
permutations on sets
urbanc [Wed, 11 Jan 2006 17:10:11 +0100] rev 18655
merged the silly lemmas into the eqvt proof of subtype
urbanc [Wed, 11 Jan 2006 17:07:57 +0100] rev 18654
tuned proofs
urbanc [Wed, 11 Jan 2006 14:00:11 +0100] rev 18653
tuned the eqvt-proof
urbanc [Wed, 11 Jan 2006 12:21:01 +0100] rev 18652
rolled back the last addition since these lemmas were already
in the simpset.
urbanc [Wed, 11 Jan 2006 12:14:25 +0100] rev 18651
added the thms-collection "pt_id" (collection of all pt_<ak>1 lemmas)
urbanc [Wed, 11 Jan 2006 12:11:53 +0100] rev 18650
tuned
paulson [Wed, 11 Jan 2006 11:00:26 +0100] rev 18649
tidied, and added missing thm divide_less_eq_1_neg
paulson [Wed, 11 Jan 2006 10:59:55 +0100] rev 18648
tidied, and giving theorems names
huffman [Wed, 11 Jan 2006 03:10:04 +0100] rev 18647
add transitivity rules
wenzelm [Wed, 11 Jan 2006 00:11:05 +0100] rev 18646
tuned;
wenzelm [Wed, 11 Jan 2006 00:11:02 +0100] rev 18645
updated;
wenzelm [Tue, 10 Jan 2006 19:36:59 +0100] rev 18644
tuned;
wenzelm [Tue, 10 Jan 2006 19:34:04 +0100] rev 18643
generic attributes;
wenzelm [Tue, 10 Jan 2006 19:33:42 +0100] rev 18642
* ML: generic context, data, attributes;
wenzelm [Tue, 10 Jan 2006 19:33:41 +0100] rev 18641
added context_of -- generic context;
wenzelm [Tue, 10 Jan 2006 19:33:39 +0100] rev 18640
generic attributes;
tuned;
wenzelm [Tue, 10 Jan 2006 19:33:38 +0100] rev 18639
print rules: generic context;
wenzelm [Tue, 10 Jan 2006 19:33:37 +0100] rev 18638
Specification.pretty_consts ctxt;
wenzelm [Tue, 10 Jan 2006 19:33:36 +0100] rev 18637
generic data and attributes;
tuned;
wenzelm [Tue, 10 Jan 2006 19:33:35 +0100] rev 18636
added rule, declaration;
support generic attributes: theory, context, generic, common, generic_attribute(_i);
added generic syntax;
basic attributes now generic;
tuned;
wenzelm [Tue, 10 Jan 2006 19:33:34 +0100] rev 18635
added generic syntax;
mk_attribute: generic;
wenzelm [Tue, 10 Jan 2006 19:33:33 +0100] rev 18634
tuned dependencies;
wenzelm [Tue, 10 Jan 2006 19:33:32 +0100] rev 18633
added declaration_attribute;
wenzelm [Tue, 10 Jan 2006 19:33:31 +0100] rev 18632
support for generic contexts with data;
wenzelm [Tue, 10 Jan 2006 19:33:30 +0100] rev 18631
fix_tac: no warning;
wenzelm [Tue, 10 Jan 2006 19:33:29 +0100] rev 18630
generic attributes;
added low-level modifiers from Pure/context_rules.ML;
wenzelm [Tue, 10 Jan 2006 19:33:27 +0100] rev 18629
Attrib.rule;
urbanc [Tue, 10 Jan 2006 15:23:31 +0100] rev 18628
tuned
urbanc [Tue, 10 Jan 2006 02:32:10 +0100] rev 18627
added the lemmas supp_char and supp_string
urbanc [Mon, 09 Jan 2006 15:55:15 +0100] rev 18626
added some lemmas to the collection "abs_fresh"
the lemmas are of the form
finite (supp x) ==> (b # [a].x) = (b=a \/ b # x)
previously only lemmas of the form
(b # [a].x) = (b=a \/ b # x)
with the type-constraint that x is finitely supported
were included.
paulson [Mon, 09 Jan 2006 13:29:08 +0100] rev 18625
_E suffix for compatibility with AddIffs
paulson [Mon, 09 Jan 2006 13:28:34 +0100] rev 18624
tidied
paulson [Mon, 09 Jan 2006 13:28:06 +0100] rev 18623
simplified the special-case simprules
paulson [Mon, 09 Jan 2006 13:27:44 +0100] rev 18622
theorems need names
urbanc [Mon, 09 Jan 2006 00:05:10 +0100] rev 18621
commented the transitivity and narrowing proof
wenzelm [Sat, 07 Jan 2006 23:28:01 +0100] rev 18620
Theory specifications --- with type-inference, but no internal polymorphism.
wenzelm [Sat, 07 Jan 2006 23:28:00 +0100] rev 18619
added infer_type, declared_type;
wenzelm [Sat, 07 Jan 2006 23:27:59 +0100] rev 18618
added param, spec, named_spec;
wenzelm [Sat, 07 Jan 2006 23:27:58 +0100] rev 18617
added init;
tuned signature;
wenzelm [Sat, 07 Jan 2006 23:27:56 +0100] rev 18616
added 'axiomatization';
wenzelm [Sat, 07 Jan 2006 23:27:55 +0100] rev 18615
Specification.pretty_consts;
wenzelm [Sat, 07 Jan 2006 23:27:53 +0100] rev 18614
gen_names: preserve empty names;
wenzelm [Sat, 07 Jan 2006 23:27:52 +0100] rev 18613
added Isar/specification.ML;
wenzelm [Sat, 07 Jan 2006 23:27:51 +0100] rev 18612
updated;
urbanc [Sat, 07 Jan 2006 13:50:38 +0100] rev 18611
another change for the new induct-method
wenzelm [Sat, 07 Jan 2006 12:28:25 +0100] rev 18610
RuleCases.make_nested;
wenzelm [Sat, 07 Jan 2006 12:26:35 +0100] rev 18609
support nested cases;
tuned apply_case;
wenzelm [Sat, 07 Jan 2006 12:26:33 +0100] rev 18608
support nested cases;
added apply_case;
replaced make/simple by make_common/nested/simple;
wenzelm [Sat, 07 Jan 2006 12:26:32 +0100] rev 18607
RuleCases.make_common;
wenzelm [Sat, 07 Jan 2006 12:26:31 +0100] rev 18606
pretty_locale: backquote notes;
wenzelm [Sat, 07 Jan 2006 12:26:29 +0100] rev 18605
RuleCases.make_simple;
wenzelm [Sat, 07 Jan 2006 12:26:28 +0100] rev 18604
tuned order;
wenzelm [Sat, 07 Jan 2006 12:26:27 +0100] rev 18603
added backquote;
wenzelm [Sat, 07 Jan 2006 12:26:25 +0100] rev 18602
RuleCases.make_common/nested;
wenzelm [Sat, 07 Jan 2006 12:26:23 +0100] rev 18601
* Provers/induct: improved simultaneous goals -- nested cases;
urbanc [Sat, 07 Jan 2006 11:43:42 +0100] rev 18600
added private datatype nprod (copy of prod) to be
used in the induction rule
urbanc [Sat, 07 Jan 2006 11:36:58 +0100] rev 18599
changed PRO_RED proof to conform with the new induction rules
wenzelm [Fri, 06 Jan 2006 18:18:16 +0100] rev 18598
prep_meta_eq: reuse mk_rews of local simpset;
adapted ML code to common conventions;
tuned;
wenzelm [Fri, 06 Jan 2006 18:18:15 +0100] rev 18597
removed obsolete eqrule_HOL_data.ML;
wenzelm [Fri, 06 Jan 2006 18:18:14 +0100] rev 18596
removed obsolete eqrule_FOL_data.ML;
wenzelm [Fri, 06 Jan 2006 18:18:13 +0100] rev 18595
simplified EqSubst setup;
wenzelm [Fri, 06 Jan 2006 18:18:12 +0100] rev 18594
obsolete, reuse mk_rews of local simpset;
wenzelm [Fri, 06 Jan 2006 15:18:22 +0100] rev 18593
Toplevel.theory_to_proof;
wenzelm [Fri, 06 Jan 2006 15:18:21 +0100] rev 18592
transactions now always see quasi-functional intermediate checkpoint;
removed obsolete theory_theory_to_proof;
added
wenzelm [Fri, 06 Jan 2006 15:18:20 +0100] rev 18591
tuned EqSubst setup;
wenzelm [Fri, 06 Jan 2006 15:18:19 +0100] rev 18590
Pure/Isar: Toplevel.theory_to_proof admits transactions that modify the theory;
wenzelm [Thu, 05 Jan 2006 22:30:00 +0100] rev 18589
hide type datatype node;
added theory_node, proof_node, is_theory, is_proof, proof_position_of, checkpoint, copy;
no_body_context: no history;
transaction: test save = true;
wenzelm [Thu, 05 Jan 2006 22:29:59 +0100] rev 18588
tuned print_theorems_theory;
wenzelm [Thu, 05 Jan 2006 22:29:58 +0100] rev 18587
Toplevel.proof_position_of;
wenzelm [Thu, 05 Jan 2006 22:29:57 +0100] rev 18586
store_thm: transfer to current context, i.e. the target theory;
wenzelm [Thu, 05 Jan 2006 22:29:55 +0100] rev 18585
replaced swap by contrapos_np;
wenzelm [Thu, 05 Jan 2006 22:29:53 +0100] rev 18584
added setminus;
tuned;
wenzelm [Thu, 05 Jan 2006 17:16:40 +0100] rev 18583
proper handling of simultaneous goals and mutual rules;
wenzelm [Thu, 05 Jan 2006 17:16:38 +0100] rev 18582
provide projections of induct_weak, induct_unsafe;
wenzelm [Thu, 05 Jan 2006 17:14:08 +0100] rev 18581
added strict_mutual_rule;
wenzelm [Thu, 05 Jan 2006 17:14:07 +0100] rev 18580
RuleCases.strict_mutual_rule;
export internalize;
urbanc [Thu, 05 Jan 2006 12:09:26 +0100] rev 18579
changed the name of the type "nOption" to "noption".
urbanc [Wed, 04 Jan 2006 20:20:25 +0100] rev 18578
added "fresh_singleton" lemma
urbanc [Wed, 04 Jan 2006 19:53:39 +0100] rev 18577
added more documentation; will now try out a modification
of the ok-predicate
nipkow [Wed, 04 Jan 2006 19:22:53 +0100] rev 18576
Reversed Larry's option/iff change.
haftmann [Wed, 04 Jan 2006 17:04:11 +0100] rev 18575
substantial additions using locales
haftmann [Wed, 04 Jan 2006 17:03:43 +0100] rev 18574
exported read|cert_arity interfaces
nipkow [Wed, 04 Jan 2006 16:38:40 +0100] rev 18573
trace_simp_depth_limit is 1 by default
nipkow [Wed, 04 Jan 2006 16:37:57 +0100] rev 18572
removed pointless trace msg.
paulson [Wed, 04 Jan 2006 16:14:15 +0100] rev 18571
preservation of names
paulson [Wed, 04 Jan 2006 16:13:53 +0100] rev 18570
a few more named lemmas
haftmann [Wed, 04 Jan 2006 10:28:31 +0100] rev 18569
fix: reintroduced pred_ctxt in gen_add_locale
wenzelm [Wed, 04 Jan 2006 01:04:59 +0100] rev 18568
tuned;
wenzelm [Wed, 04 Jan 2006 01:00:52 +0100] rev 18567
* Pure/Isar: Toplevel.theory_theory_to_proof;
wenzelm [Wed, 04 Jan 2006 00:52:49 +0100] rev 18566
added unlocalize_mfix;
wenzelm [Wed, 04 Jan 2006 00:52:48 +0100] rev 18565
added unlocalize_mixfix;
wenzelm [Wed, 04 Jan 2006 00:52:47 +0100] rev 18564
added theory_to_theory_to_proof, which may change theory before entering the proof;
added forget_proof (from isar_thy.ML);
wenzelm [Wed, 04 Jan 2006 00:52:45 +0100] rev 18563
tuned;
wenzelm [Wed, 04 Jan 2006 00:52:45 +0100] rev 18562
moved forget_proof to toplevel.ML;
wenzelm [Wed, 04 Jan 2006 00:52:43 +0100] rev 18561
Toplevel.forget_proof;
wenzelm [Wed, 04 Jan 2006 00:52:42 +0100] rev 18560
adapted Toplevel.Proof;
wenzelm [Wed, 04 Jan 2006 00:52:40 +0100] rev 18559
removed dead code;
wenzelm [Wed, 04 Jan 2006 00:52:38 +0100] rev 18558
more stuff;
paulson [Tue, 03 Jan 2006 15:44:39 +0100] rev 18557
Provers/classical: stricter checks to ensure that supplied intro, dest and
elim rules are well-formed
paulson [Tue, 03 Jan 2006 15:43:54 +0100] rev 18556
added explicit paths to required theories
wenzelm [Tue, 03 Jan 2006 14:07:17 +0100] rev 18555
added implementation manual;
wenzelm [Tue, 03 Jan 2006 13:59:55 +0100] rev 18554
more stuff;
wenzelm [Tue, 03 Jan 2006 11:57:33 +0100] rev 18553
fixed LaTeX source;
haftmann [Tue, 03 Jan 2006 11:33:18 +0100] rev 18552
class now a keyword
haftmann [Tue, 03 Jan 2006 11:32:55 +0100] rev 18551
class now an keyword, quoted where necessary
haftmann [Tue, 03 Jan 2006 11:32:16 +0100] rev 18550
add_local_context now yields imported and body elements seperatly; additional slight clenup in code
haftmann [Tue, 03 Jan 2006 11:31:15 +0100] rev 18549
rearranged burrow_split to fold_burrow to allow composition with fold_map
wenzelm [Tue, 03 Jan 2006 00:06:30 +0100] rev 18548
added unfolding(_i);
renamed using_thmss(_i) to using_i;
wenzelm [Tue, 03 Jan 2006 00:06:29 +0100] rev 18547
unparse String/AltString: escape quotes;
wenzelm [Tue, 03 Jan 2006 00:06:28 +0100] rev 18546
tuned;
wenzelm [Tue, 03 Jan 2006 00:06:26 +0100] rev 18545
avoid hardwired Trueprop;
local proof: static refererence to Pure.thy;
wenzelm [Tue, 03 Jan 2006 00:06:24 +0100] rev 18544
added 'using' command;
wenzelm [Tue, 03 Jan 2006 00:06:23 +0100] rev 18543
updated;
wenzelm [Tue, 03 Jan 2006 00:06:22 +0100] rev 18542
added IsarImplementation;
wenzelm [Tue, 03 Jan 2006 00:06:20 +0100] rev 18541
updated -- lost update!?
wenzelm [Tue, 03 Jan 2006 00:06:18 +0100] rev 18540
* Pure/Isar: new command 'unfolding';
* ML/Provers: more generic wrt. syntax of object-logics;
tuned;
wenzelm [Mon, 02 Jan 2006 20:50:17 +0100] rev 18539
ISABELLE_USER for remote cvs access;
wenzelm [Mon, 02 Jan 2006 20:42:12 +0100] rev 18538
outline;
wenzelm [Mon, 02 Jan 2006 20:16:52 +0100] rev 18537
"The Isabelle/Isar Implementation" manual;
wenzelm [Sat, 31 Dec 2005 21:49:44 +0100] rev 18536
* Provers/classical: removed obsolete classical version of elim_format;
wenzelm [Sat, 31 Dec 2005 21:49:43 +0100] rev 18535
tuned forall_intr_vars;
wenzelm [Sat, 31 Dec 2005 21:49:42 +0100] rev 18534
added classical_rule, which replaces Data.make_elim;
removed obsolete Data.make_elim and classical elim_format attribute;
tuned;
wenzelm [Sat, 31 Dec 2005 21:49:41 +0100] rev 18533
explicitly reject consts *Goal*, *False*;
wenzelm [Sat, 31 Dec 2005 21:49:40 +0100] rev 18532
elim rules: Classical.classical_rule;
wenzelm [Sat, 31 Dec 2005 21:49:39 +0100] rev 18531
removed obsolete cla_dist_concl;
wenzelm [Sat, 31 Dec 2005 21:49:38 +0100] rev 18530
removed classical elim_format;
wenzelm [Sat, 31 Dec 2005 21:49:36 +0100] rev 18529
removed obsolete Provers/make_elim.ML;
wenzelm [Sat, 31 Dec 2005 21:49:35 +0100] rev 18528
obsolete, see classical_rule in Provers/classical.ML;
wenzelm [Sat, 31 Dec 2005 13:03:55 +0100] rev 18527
more robust phantomsection;
wenzelm [Fri, 30 Dec 2005 16:57:00 +0100] rev 18526
require cla_dist_concl, avoid assumptions about concrete syntax;
wenzelm [Fri, 30 Dec 2005 16:56:59 +0100] rev 18525
avoid implicit assumptions about consts Not, op =, *Goal*, *False*;
wenzelm [Fri, 30 Dec 2005 16:56:58 +0100] rev 18524
provide equality_name, not_name;
wenzelm [Fri, 30 Dec 2005 16:56:57 +0100] rev 18523
fixed final_consts;
wenzelm [Fri, 30 Dec 2005 16:56:56 +0100] rev 18522
provide cla_dist_concl;
wenzelm [Fri, 30 Dec 2005 16:56:54 +0100] rev 18521
non-PDF: phantomsection;
haftmann [Thu, 29 Dec 2005 16:10:58 +0100] rev 18520
added atom keyword
haftmann [Thu, 29 Dec 2005 15:31:27 +0100] rev 18519
changes in code generator keywords
haftmann [Thu, 29 Dec 2005 15:31:10 +0100] rev 18518
adaptions to changes in code generator
haftmann [Thu, 29 Dec 2005 15:30:52 +0100] rev 18517
slight improvements
haftmann [Wed, 28 Dec 2005 21:14:23 +0100] rev 18516
slightly improved serialization
haftmann [Tue, 27 Dec 2005 15:24:40 +0100] rev 18515
substantial improvements in code generating
haftmann [Tue, 27 Dec 2005 15:24:23 +0100] rev 18514
added map_index