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