Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-10000
-3000
-1000
-128
+128
+1000
+3000
+10000
+30000
tip
Find changesets by keywords (author, files, the commit message), revision number or hash, or
revset expression
.
The revision graph only works with JavaScript-enabled browsers.
moved atomize stuff to theory IFOL;
2001-10-04, by wenzelm
atomize stuff from theory FOL;
2001-10-04, by wenzelm
added Provers/induct_method.ML, document/root.tex, ex/Natural_Numbers.thy;
2001-10-04, by wenzelm
theory Natural_Numbers;
2001-10-04, by wenzelm
use "~~/src/Provers/induct_method.ML";
2001-10-04, by wenzelm
Theory of the natural numbers: Peano's axioms, primitive recursion.
2001-10-04, by wenzelm
full_rewrite_cterm_aux (see also tactic.ML);
2001-10-04, by wenzelm
added full_rewrite_cterm;
2001-10-04, by wenzelm
proof by cases and induction on types and sets (used to be specific for HOL);
2001-10-04, by wenzelm
qualify MetaSimplifier;
2001-10-04, by wenzelm
added dest_conj, dest_concls;
2001-10-04, by wenzelm
document setup;
2001-10-04, by wenzelm
added print_induct_rules;
2001-10-04, by wenzelm
tuned print operation;
2001-10-04, by wenzelm
tuned;
2001-10-04, by wenzelm
* moved induct/cases attributes to Pure, added 'print_induct_rules' command;
2001-10-04, by wenzelm
print_induct_rules;
2001-10-04, by wenzelm
updated;
2001-10-04, by wenzelm
Fixed bug in decompose.
2001-10-04, by berghofe
Tools/induct_attrib.ML now part of Pure;
2001-10-03, by wenzelm
Isar/induct_attrib.ML;
2001-10-03, by wenzelm
*** empty log message ***
2001-10-03, by wenzelm
moved HOL/Tools/induct_attrib.ML to Pure/Isar/induct_attrib.ML;
2001-10-03, by wenzelm
tuned parentheses in relational expressions;
2001-10-03, by wenzelm
moved linorder_cases to theory Ord;
2001-10-03, by wenzelm
linorder_cases supersedes linorder_less_split;
2001-10-03, by wenzelm
eta-expansion required for SML/NJ
2001-10-03, by paulson
support non-oriented infix;
2001-10-02, by wenzelm
tuned;
2001-10-01, by wenzelm
tuned;
2001-10-01, by wenzelm
*** empty log message ***
2001-10-01, by wenzelm
initial setup for chapter on document preparation;
2001-10-01, by wenzelm
updated output;
2001-10-01, by wenzelm
- declared wf_java_prog as syntax (previously: definition)
2001-10-01, by streckem
Removed some unfoldings of defs after declaring wf_java_prog as syntax
2001-10-01, by streckem
Added axiom e~=This to reflect strengthened precond. in rule LAss
2001-10-01, by streckem
Minor modifications
2001-10-01, by streckem
added Ordinals example;
2001-10-01, by wenzelm
Tuned indentation of abstractions.
2001-09-30, by berghofe
tuned;
2001-09-28, by wenzelm
inductive: no collective atts;
2001-09-28, by wenzelm
inductive: no collective atts;
2001-09-28, by wenzelm
oops;
2001-09-28, by wenzelm
tuned;
2001-09-28, by wenzelm
recdef (permissive);
2001-09-28, by wenzelm
*** empty log message ***
2001-09-28, by wenzelm
prove: ``strict'' argument;
2001-09-28, by wenzelm
internal thm numbering with ":" instead of "_";
2001-09-28, by wenzelm
avoid handle _;
2001-09-28, by wenzelm
permissive option;
2001-09-28, by wenzelm
inductive: no collective atts;
2001-09-28, by wenzelm
updated;
2001-09-28, by wenzelm
recdef (permissive);
2001-09-28, by wenzelm
Tuned section about parsing and printing proof terms.
2001-09-28, by berghofe
mksimps and mk_eq_True no longer raise THM exception.
2001-09-28, by berghofe
Added label for section on terms.
2001-09-28, by berghofe
Added documentation for proof terms.
2001-09-28, by berghofe
Added TYPE to Pure grammar.
2001-09-28, by berghofe
Added \ttlbrack and \ttrbrack.
2001-09-28, by berghofe
Added TPHOLs2000 paper about proof terms.
2001-09-28, by berghofe
updated;
2001-09-28, by wenzelm
tuned;
2001-09-28, by wenzelm
tuned;
2001-09-28, by wenzelm
- Exchanged % and %%.
2001-09-28, by berghofe
- Tuned syntax
2001-09-28, by berghofe
- Exchanged % and %%
2001-09-28, by berghofe
Exchanged % and %%.
2001-09-28, by berghofe
HOL: eliminated global items;
2001-09-27, by wenzelm
updated;
2001-09-27, by wenzelm
eliminated theories "equalities" and "mono" (made part of "Typedef",
2001-09-27, by wenzelm
renamed theory "subset" to "Typedef";
2001-09-27, by wenzelm
unsymbolize;
2001-09-27, by wenzelm
renamed "()" to Unity;
2001-09-27, by wenzelm
HOLogic.unit;
2001-09-27, by wenzelm
made unit type local;
2001-09-27, by wenzelm
tuned:
2001-09-27, by wenzelm
renamed "()" to Unity, made local;
2001-09-27, by wenzelm
added surjE;
2001-09-27, by wenzelm
prepared for Isabelle2001;
2001-09-27, by wenzelm
renamed real_of_nat_eq_cancel to real_of_nat_inject, and declared as iff rule;
2001-09-27, by wenzelm
updated;
2001-09-27, by wenzelm
renamed real_of_int_eq_iff to real_of_int_inject;
2001-09-27, by wenzelm
document setup;
2001-09-27, by wenzelm
new-style theory;
2001-09-27, by wenzelm
Square roots of primes are irrational;
2001-09-27, by wenzelm
AddXIs [dvdI]; AddXEs [dvdE];
2001-09-27, by wenzelm
tuned;
2001-09-27, by wenzelm
tuned;
2001-09-27, by wenzelm
tuned;
2001-09-27, by wenzelm
AddXEs [UnI1, UnI2];
2001-09-27, by wenzelm
AddXEs [disjI1, disjI2];
2001-09-27, by wenzelm
ex/Hilbert_Classical.thy ex/document/root.tex;
2001-09-27, by wenzelm
tuned;
2001-09-27, by wenzelm
document setup;
2001-09-27, by wenzelm
derive tertium-non-datur by means of Hilbert's choice operator;
2001-09-27, by wenzelm
obsolete;
2001-09-27, by wenzelm
updated;
2001-09-27, by wenzelm
-v option;
2001-09-27, by wenzelm
verbose option;
2001-09-27, by wenzelm
use_dir: verbose option;
2001-09-27, by wenzelm
removed option -d (now standard behaviour);
2001-09-27, by wenzelm
option -v;
2001-09-27, by wenzelm
activate default ISABELLE_USEDIR_OPTIONS for precompiled distribution;
2001-09-26, by wenzelm
updated;
2001-09-26, by wenzelm
tuned order;
2001-09-26, by wenzelm
bold symbols;
2001-09-26, by wenzelm
tuned;
2001-09-26, by wenzelm
turn bullet into bold cdot (looks much better in printed output);
2001-09-26, by wenzelm
use darkblue for all links;
2001-09-26, by wenzelm
updated;
2001-09-26, by wenzelm
updated;
2001-09-25, by wenzelm
*** empty log message ***
2001-09-25, by wenzelm
tuned;
2001-09-25, by wenzelm
Minor improvements, added Example
2001-09-21, by oheimb
tuned;
2001-09-17, by wenzelm
Fixed proof term bug in permute_prems.
2001-09-13, by berghofe
result_error_default: include msg;
2001-09-12, by wenzelm
*** empty log message ***
2001-09-11, by nipkow
marginally improved comments
2001-09-10, by oheimb
corrected antiquotations in comment
2001-09-10, by oheimb
simplified vnam/vname, introduced fname, improved comments
2001-09-10, by oheimb
tuned usage;
2001-09-10, by wenzelm
print_state: subgoals;
2001-09-08, by wenzelm
export pretty_goals;
2001-09-08, by wenzelm
result_error_default: output *single* error message;
2001-09-08, by wenzelm
tuned;
2001-09-08, by wenzelm
ISABELLE_INTERFACE=none by default (cannot expect X11 everywhere);
2001-09-08, by wenzelm
* system: support Poly/ML 4.1.1 (large heaps);
2001-09-08, by wenzelm
less
more
|
(0)
-10000
-3000
-1000
-128
+128
+1000
+3000
+10000
+30000
tip