wenzelm [Tue, 09 Oct 2001 18:11:07 +0200] rev 11714
added global modes ref;
wenzelm [Mon, 08 Oct 2001 15:23:20 +0200] rev 11713
sane numerals (stage 3): provide generic "1" on all number types;
wenzelm [Mon, 08 Oct 2001 14:30:28 +0200] rev 11712
* added default LaTeX bindings for \<tturnstile> and \<TTurnstile>;
note that these symbols are unavailable in Proof General / X-Symbol;
wenzelm [Mon, 08 Oct 2001 14:29:02 +0200] rev 11711
fixed numerals;
wenzelm [Mon, 08 Oct 2001 14:19:42 +0200] rev 11710
added tturnstile, TTurnstile;
wenzelm [Mon, 08 Oct 2001 14:19:22 +0200] rev 11709
*** empty log message ***
wenzelm [Mon, 08 Oct 2001 12:28:43 +0200] rev 11708
*** empty log message ***
wenzelm [Mon, 08 Oct 2001 12:27:19 +0200] rev 11707
replace 0r/1r by 0/1;
wenzelm [Mon, 08 Oct 2001 12:13:56 +0200] rev 11706
*** empty log message ***
wenzelm [Mon, 08 Oct 2001 12:13:34 +0200] rev 11705
fixed numerals;
wenzelm [Sat, 06 Oct 2001 00:02:46 +0200] rev 11704
* sane numerals (stage 2): plain "num" syntax (removed "#");
wenzelm [Fri, 05 Oct 2001 23:58:52 +0200] rev 11703
tuned;
wenzelm [Fri, 05 Oct 2001 23:58:17 +0200] rev 11702
*** empty log message ***
wenzelm [Fri, 05 Oct 2001 21:52:39 +0200] rev 11701
sane numerals (stage 1): added generic 1, removed 1' and 2 on nat,
"num" syntax (still with "#"), Numeral0, Numeral1;
wenzelm [Fri, 05 Oct 2001 21:50:37 +0200] rev 11700
*** empty log message ***
wenzelm [Fri, 05 Oct 2001 21:49:59 +0200] rev 11699
"num" syntax;
wenzelm [Fri, 05 Oct 2001 21:49:15 +0200] rev 11698
added axclass "one" and polymorphic const "1";
print consts "0" and "1" with type constraints;
wenzelm [Fri, 05 Oct 2001 21:48:04 +0200] rev 11697
added "num" token;
wenzelm [Fri, 05 Oct 2001 21:42:10 +0200] rev 11696
induct: case names;
wenzelm [Fri, 05 Oct 2001 21:37:33 +0200] rev 11695
sane spacing of "-";
wenzelm [Fri, 05 Oct 2001 16:04:56 +0200] rev 11694
tuned;
wenzelm [Thu, 04 Oct 2001 23:27:42 +0200] rev 11693
Thm.major_prem_of part of Logic.strip_assums_concl;
wenzelm [Thu, 04 Oct 2001 23:27:01 +0200] rev 11692
major_prem_of: Logic.strip_assums_concl;
wenzelm [Thu, 04 Oct 2001 16:09:12 +0200] rev 11691
induct/cases made generic, removed simplified/stripped options;
wenzelm [Thu, 04 Oct 2001 16:07:43 +0200] rev 11690
improved proof by cases and induction;
wenzelm [Thu, 04 Oct 2001 16:07:20 +0200] rev 11689
removed obsolete comment;
wenzelm [Thu, 04 Oct 2001 15:43:17 +0200] rev 11688
generic induct_method.ML;
tuned;
wenzelm [Thu, 04 Oct 2001 15:42:48 +0200] rev 11687
non-oriented infix = and ~= (output only);
added case_split (with case names);
wenzelm [Thu, 04 Oct 2001 15:41:43 +0200] rev 11686
$(SRC)/Provers/induct_method.ML replaces Tools/induct_method.ML;
wenzelm [Thu, 04 Oct 2001 15:40:52 +0200] rev 11685
use "~~/src/Provers/induct_method.ML";
wenzelm [Thu, 04 Oct 2001 15:40:31 +0200] rev 11684
removed hol_rewrite_cterm (use full_rewrite_cterm from Pure);
wenzelm [Thu, 04 Oct 2001 15:40:05 +0200] rev 11683
added dest_concls;
wenzelm [Thu, 04 Oct 2001 15:39:43 +0200] rev 11682
simp_case_tac is back again from induct_method.ML;
tuned;
wenzelm [Thu, 04 Oct 2001 15:39:00 +0200] rev 11681
made generic (see Provers/induct_method.ML);
wenzelm [Thu, 04 Oct 2001 15:29:37 +0200] rev 11680
qualify MetaSimplifier;
wenzelm [Thu, 04 Oct 2001 15:29:22 +0200] rev 11679
unsymbolized;
wenzelm [Thu, 04 Oct 2001 15:28:26 +0200] rev 11678
moved atomize stuff to theory IFOL;
added induct/cases setup;
wenzelm [Thu, 04 Oct 2001 15:28:00 +0200] rev 11677
atomize stuff from theory FOL;
tuned;
wenzelm [Thu, 04 Oct 2001 15:27:13 +0200] rev 11676
added Provers/induct_method.ML, document/root.tex, ex/Natural_Numbers.thy;
wenzelm [Thu, 04 Oct 2001 15:26:14 +0200] rev 11675
theory Natural_Numbers;
wenzelm [Thu, 04 Oct 2001 15:25:51 +0200] rev 11674
use "~~/src/Provers/induct_method.ML";
wenzelm [Thu, 04 Oct 2001 15:25:31 +0200] rev 11673
Theory of the natural numbers: Peano's axioms, primitive recursion.
(Modernized version of Larry Paulson's theory "Nat".)
wenzelm [Thu, 04 Oct 2001 15:21:47 +0200] rev 11672
full_rewrite_cterm_aux (see also tactic.ML);
no longer open MetaSimplifier;
wenzelm [Thu, 04 Oct 2001 15:21:17 +0200] rev 11671
added full_rewrite_cterm;
wenzelm [Thu, 04 Oct 2001 15:20:40 +0200] rev 11670
proof by cases and induction on types and sets (used to be specific for HOL);
wenzelm [Thu, 04 Oct 2001 15:19:56 +0200] rev 11669
qualify MetaSimplifier;
wenzelm [Thu, 04 Oct 2001 14:49:38 +0200] rev 11668
added dest_conj, dest_concls;
wenzelm [Thu, 04 Oct 2001 14:49:10 +0200] rev 11667
document setup;
wenzelm [Thu, 04 Oct 2001 11:29:46 +0200] rev 11666
added print_induct_rules;
wenzelm [Thu, 04 Oct 2001 11:29:25 +0200] rev 11665
tuned print operation;
wenzelm [Thu, 04 Oct 2001 11:29:02 +0200] rev 11664
tuned;
wenzelm [Thu, 04 Oct 2001 11:28:30 +0200] rev 11663
* moved induct/cases attributes to Pure, added 'print_induct_rules' command;
wenzelm [Thu, 04 Oct 2001 11:28:12 +0200] rev 11662
print_induct_rules;
wenzelm [Thu, 04 Oct 2001 11:22:10 +0200] rev 11661
updated;
berghofe [Thu, 04 Oct 2001 00:53:27 +0200] rev 11660
Fixed bug in decompose.
wenzelm [Wed, 03 Oct 2001 21:03:05 +0200] rev 11659
Tools/induct_attrib.ML now part of Pure;
wenzelm [Wed, 03 Oct 2001 21:01:53 +0200] rev 11658
Isar/induct_attrib.ML;
wenzelm [Wed, 03 Oct 2001 20:58:27 +0200] rev 11657
*** empty log message ***
wenzelm [Wed, 03 Oct 2001 20:55:31 +0200] rev 11656
moved HOL/Tools/induct_attrib.ML to Pure/Isar/induct_attrib.ML;
wenzelm [Wed, 03 Oct 2001 20:54:16 +0200] rev 11655
tuned parentheses in relational expressions;
wenzelm [Wed, 03 Oct 2001 20:54:05 +0200] rev 11654
moved linorder_cases to theory Ord;
wenzelm [Wed, 03 Oct 2001 20:53:02 +0200] rev 11653
linorder_cases supersedes linorder_less_split;
tuned parentheses in relational expressions;
paulson [Wed, 03 Oct 2001 11:45:24 +0200] rev 11652
eta-expansion required for SML/NJ
wenzelm [Tue, 02 Oct 2001 20:23:33 +0200] rev 11651
support non-oriented infix;
wenzelm [Mon, 01 Oct 2001 21:53:50 +0200] rev 11650
tuned;
wenzelm [Mon, 01 Oct 2001 15:46:35 +0200] rev 11649
tuned;
wenzelm [Mon, 01 Oct 2001 14:47:02 +0200] rev 11648
*** empty log message ***
wenzelm [Mon, 01 Oct 2001 14:44:00 +0200] rev 11647
initial setup for chapter on document preparation;
wenzelm [Mon, 01 Oct 2001 14:42:47 +0200] rev 11646
updated output;
streckem [Mon, 01 Oct 2001 13:39:17 +0200] rev 11645
- declared wf_java_prog as syntax (previously: definition)
- in wf_java_mdecl: added preconditions for 'This'
- rule LAss: precondition v ~=This
streckem [Mon, 01 Oct 2001 13:36:25 +0200] rev 11644
Removed some unfoldings of defs after declaring wf_java_prog as syntax
streckem [Mon, 01 Oct 2001 13:33:49 +0200] rev 11643
Added axiom e~=This to reflect strengthened precond. in rule LAss
streckem [Mon, 01 Oct 2001 13:32:11 +0200] rev 11642
Minor modifications
wenzelm [Mon, 01 Oct 2001 11:56:40 +0200] rev 11641
added Ordinals example;
berghofe [Sun, 30 Sep 2001 13:42:00 +0200] rev 11640
Tuned indentation of abstractions.
wenzelm [Fri, 28 Sep 2001 21:45:40 +0200] rev 11639
tuned;
wenzelm [Fri, 28 Sep 2001 21:45:11 +0200] rev 11638
inductive: no collective atts;
wenzelm [Fri, 28 Sep 2001 20:09:10 +0200] rev 11637
inductive: no collective atts;
wenzelm [Fri, 28 Sep 2001 20:08:28 +0200] rev 11636
oops;
wenzelm [Fri, 28 Sep 2001 20:08:05 +0200] rev 11635
tuned;
wenzelm [Fri, 28 Sep 2001 19:24:25 +0200] rev 11634
recdef (permissive);
inductive: no collective atts;
wenzelm [Fri, 28 Sep 2001 19:23:58 +0200] rev 11633
*** empty log message ***
wenzelm [Fri, 28 Sep 2001 19:23:35 +0200] rev 11632
prove: ``strict'' argument;
wenzelm [Fri, 28 Sep 2001 19:23:07 +0200] rev 11631
internal thm numbering with ":" instead of "_";
wenzelm [Fri, 28 Sep 2001 19:22:40 +0200] rev 11630
avoid handle _;
wenzelm [Fri, 28 Sep 2001 19:21:26 +0200] rev 11629
permissive option;
wenzelm [Fri, 28 Sep 2001 19:19:26 +0200] rev 11628
inductive: no collective atts;
wenzelm [Fri, 28 Sep 2001 19:18:46 +0200] rev 11627
updated;
wenzelm [Fri, 28 Sep 2001 19:17:01 +0200] rev 11626
recdef (permissive);
berghofe [Fri, 28 Sep 2001 18:55:37 +0200] rev 11625
Tuned section about parsing and printing proof terms.
berghofe [Fri, 28 Sep 2001 17:19:46 +0200] rev 11624
mksimps and mk_eq_True no longer raise THM exception.
berghofe [Fri, 28 Sep 2001 16:45:03 +0200] rev 11623
Added label for section on terms.
berghofe [Fri, 28 Sep 2001 16:44:27 +0200] rev 11622
Added documentation for proof terms.
berghofe [Fri, 28 Sep 2001 16:43:50 +0200] rev 11621
Added TYPE to Pure grammar.
berghofe [Fri, 28 Sep 2001 16:42:58 +0200] rev 11620
Added \ttlbrack and \ttrbrack.
berghofe [Fri, 28 Sep 2001 16:42:26 +0200] rev 11619
Added TPHOLs2000 paper about proof terms.
wenzelm [Fri, 28 Sep 2001 16:15:26 +0200] rev 11618
updated;
wenzelm [Fri, 28 Sep 2001 14:10:01 +0200] rev 11617
tuned;
wenzelm [Fri, 28 Sep 2001 14:04:14 +0200] rev 11616
tuned;
berghofe [Fri, 28 Sep 2001 11:08:53 +0200] rev 11615
- Exchanged % and %%.
- Fixed bug in shrink.
berghofe [Fri, 28 Sep 2001 11:07:40 +0200] rev 11614
- Tuned syntax
- proof_of_term: fixed problems with dummy patterns and typing information
berghofe [Fri, 28 Sep 2001 11:05:37 +0200] rev 11613
- Exchanged % and %%
- Renamed reconstruct_prf to reconstruct_proof
berghofe [Fri, 28 Sep 2001 11:04:44 +0200] rev 11612
Exchanged % and %%.
wenzelm [Thu, 27 Sep 2001 22:30:09 +0200] rev 11611
HOL: eliminated global items;
wenzelm [Thu, 27 Sep 2001 22:29:57 +0200] rev 11610
updated;
wenzelm [Thu, 27 Sep 2001 22:28:16 +0200] rev 11609
eliminated theories "equalities" and "mono" (made part of "Typedef",
which supercedes "subset");
wenzelm [Thu, 27 Sep 2001 22:26:00 +0200] rev 11608
renamed theory "subset" to "Typedef";
wenzelm [Thu, 27 Sep 2001 22:25:12 +0200] rev 11607
unsymbolize;
wenzelm [Thu, 27 Sep 2001 22:24:28 +0200] rev 11606
renamed "()" to Unity;
wenzelm [Thu, 27 Sep 2001 22:24:09 +0200] rev 11605
HOLogic.unit;
wenzelm [Thu, 27 Sep 2001 22:23:40 +0200] rev 11604
made unit type local;
wenzelm [Thu, 27 Sep 2001 22:23:20 +0200] rev 11603
tuned:
wenzelm [Thu, 27 Sep 2001 22:22:58 +0200] rev 11602
renamed "()" to Unity, made local;
wenzelm [Thu, 27 Sep 2001 22:22:08 +0200] rev 11601
added surjE;
wenzelm [Thu, 27 Sep 2001 18:56:39 +0200] rev 11600
prepared for Isabelle2001;
wenzelm [Thu, 27 Sep 2001 18:46:32 +0200] rev 11599
renamed real_of_nat_eq_cancel to real_of_nat_inject, and declared as iff rule;
wenzelm [Thu, 27 Sep 2001 18:45:40 +0200] rev 11598
updated;
wenzelm [Thu, 27 Sep 2001 18:45:23 +0200] rev 11597
renamed real_of_int_eq_iff to real_of_int_inject;
wenzelm [Thu, 27 Sep 2001 18:44:30 +0200] rev 11596
document setup;
wenzelm [Thu, 27 Sep 2001 18:44:12 +0200] rev 11595
new-style theory;