Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-10000
-3000
-1000
-120
+120
+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.
removed vars_of, concls_of;
2001-10-12, by wenzelm
declare impE iffD1 iffD2 ad elim of Pure;
2001-10-12, by wenzelm
removed lookups count;
2001-10-12, by wenzelm
added make_thm (sort-of);
2001-10-12, by wenzelm
added trace_rules, trace;
2001-10-12, by wenzelm
removed get_cases, get_induct;
2001-10-12, by wenzelm
removed read_inst', no longer export insts';
2001-10-12, by wenzelm
fixed typid;
2001-10-12, by wenzelm
test: use SkipProof.make_thm instead of Thm.assume;
2001-10-12, by wenzelm
tuned;
2001-10-12, by wenzelm
HOLogic.dest_concls, InductAttrib.vars_of;
2001-10-12, by wenzelm
declare impE iffD1 iffD2 as elim of Pure;
2001-10-12, by wenzelm
moved trace_rules to Pure/Isar/method.ML;
2001-10-12, by wenzelm
* Isar/Pure: fixed 'token_translation' command;
2001-10-11, by wenzelm
added try;
2001-10-11, by wenzelm
added certify_tyname;
2001-10-11, by wenzelm
Exported output_symbols.
2001-10-10, by berghofe
Removed unnecessary application of Drule.standard.
2001-10-10, by berghofe
Fixed erroneous type constraint in token_translation function.
2001-10-10, by berghofe
Exported output_with.
2001-10-10, by berghofe
Tuned several functions to improve sharing of unchanged subproofs.
2001-10-10, by berghofe
added global modes ref;
2001-10-09, by wenzelm
sane numerals (stage 3): provide generic "1" on all number types;
2001-10-08, by wenzelm
* added default LaTeX bindings for \<tturnstile> and \<TTurnstile>;
2001-10-08, by wenzelm
fixed numerals;
2001-10-08, by wenzelm
added tturnstile, TTurnstile;
2001-10-08, by wenzelm
*** empty log message ***
2001-10-08, by wenzelm
*** empty log message ***
2001-10-08, by wenzelm
replace 0r/1r by 0/1;
2001-10-08, by wenzelm
*** empty log message ***
2001-10-08, by wenzelm
fixed numerals;
2001-10-08, by wenzelm
* sane numerals (stage 2): plain "num" syntax (removed "#");
2001-10-06, by wenzelm
tuned;
2001-10-05, by wenzelm
*** empty log message ***
2001-10-05, by wenzelm
sane numerals (stage 1): added generic 1, removed 1' and 2 on nat,
2001-10-05, by wenzelm
*** empty log message ***
2001-10-05, by wenzelm
"num" syntax;
2001-10-05, by wenzelm
added axclass "one" and polymorphic const "1";
2001-10-05, by wenzelm
added "num" token;
2001-10-05, by wenzelm
induct: case names;
2001-10-05, by wenzelm
sane spacing of "-";
2001-10-05, by wenzelm
tuned;
2001-10-05, by wenzelm
Thm.major_prem_of part of Logic.strip_assums_concl;
2001-10-04, by wenzelm
major_prem_of: Logic.strip_assums_concl;
2001-10-04, by wenzelm
induct/cases made generic, removed simplified/stripped options;
2001-10-04, by wenzelm
improved proof by cases and induction;
2001-10-04, by wenzelm
removed obsolete comment;
2001-10-04, by wenzelm
generic induct_method.ML;
2001-10-04, by wenzelm
non-oriented infix = and ~= (output only);
2001-10-04, by wenzelm
$(SRC)/Provers/induct_method.ML replaces Tools/induct_method.ML;
2001-10-04, by wenzelm
use "~~/src/Provers/induct_method.ML";
2001-10-04, by wenzelm
removed hol_rewrite_cterm (use full_rewrite_cterm from Pure);
2001-10-04, by wenzelm
added dest_concls;
2001-10-04, by wenzelm
simp_case_tac is back again from induct_method.ML;
2001-10-04, by wenzelm
made generic (see Provers/induct_method.ML);
2001-10-04, by wenzelm
qualify MetaSimplifier;
2001-10-04, by wenzelm
unsymbolized;
2001-10-04, by wenzelm
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
less
more
|
(0)
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip