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.
added Term and Tree_Forest (from converted ZF/ex);
2001-11-15, by wenzelm
TF and Term moved to ZF/Induct;
2001-11-15, by wenzelm
miniscoping of UN and INT
2001-11-15, by paulson
Added new entry
2001-11-15, by ehmety
New files
2001-11-15, by ehmety
new theories from Jacques Fleuriot
2001-11-15, by paulson
*** empty log message ***
2001-11-15, by ehmety
converted datatype examples moved from ZF/ex to ZF/Induct;
2001-11-14, by wenzelm
document setup;
2001-11-14, by wenzelm
removed BT, Data, Enum (see ZF/Induct);
2001-11-14, by wenzelm
case_names;
2001-11-14, by wenzelm
added Datatypes, Binary_Trees (from ZF/ex);
2001-11-14, by wenzelm
Isar attribute and method setup;
2001-11-14, by wenzelm
fix path prefix;
2001-11-14, by wenzelm
use proper intr_names (for required case_names);
2001-11-14, by wenzelm
added Induct/Binary_Trees.thy, Induct/Datatypes.thy;
2001-11-14, by wenzelm
tuned;
2001-11-14, by wenzelm
updated;
2001-11-14, by wenzelm
adapted primrec/datatype to Isar;
2001-11-14, by wenzelm
tuned;
2001-11-14, by wenzelm
store original simps for codegen;
2001-11-14, by wenzelm
inductive: removed con_defs;
2001-11-14, by wenzelm
updated;
2001-11-14, by wenzelm
updated;
2001-11-13, by wenzelm
* ZF: new-style theory commands 'inductive', 'inductive_cases', and
2001-11-13, by wenzelm
ZF specific keywords;
2001-11-13, by wenzelm
rearranged inductive package for Isar;
2001-11-13, by wenzelm
Generic inductive cases facility for (co)inductive definitions.
2001-11-13, by wenzelm
converted;
2001-11-13, by wenzelm
tuned;
2001-11-13, by wenzelm
tuned inductions;
2001-11-13, by wenzelm
prove: Envir.beta_norm;
2001-11-13, by wenzelm
new SList theory from Bu Wolff
2001-11-13, by paulson
induct: rule_versions produces localized variants;
2001-11-12, by wenzelm
empty rule_context for multiple goals;
2001-11-12, by wenzelm
added empty;
2001-11-12, by wenzelm
mutual rules declared as ``consumes 0'';
2001-11-12, by wenzelm
induct_atomize: include atomize_conj (for mutual induction);
2001-11-12, by wenzelm
Isar: 'induct' proper support for mutual induction involving
2001-11-12, by wenzelm
proper handling of mutual rules (esp. for sets);
2001-11-12, by wenzelm
lemmas induct_atomize = atomize_conj ...;
2001-11-12, by wenzelm
val local_imp_def = thm "induct_implies_def";
2001-11-12, by wenzelm
ZF/Induct,UNITY
2001-11-12, by paulson
Tidying necessitated by new simprules in equalities.ML
2001-11-12, by paulson
conditional miniscoping equalities now made unconditional
2001-11-12, by paulson
new-style numerals without leading #, along with generic 0 and 1
2001-11-12, by paulson
congc now returns None if congruence rule has no effect.
2001-11-12, by berghofe
Renamed some bound variables due to changes in simplifier.
2001-11-12, by berghofe
Fixed proof depending on strange behaviour of rename_bvs.
2001-11-12, by berghofe
Renamed some bound variables due to changes in simplifier.
2001-11-12, by berghofe
present multi_result;
2001-11-11, by wenzelm
added meta_conjunction_tr';
2001-11-11, by wenzelm
pure_syntax_output: "_meta_conjunction";
2001-11-11, by wenzelm
adapted to multiple results;
2001-11-11, by wenzelm
adapted auto_bind_goal, auto_bind_facts;
2001-11-11, by wenzelm
added multi_theorem(_i);
2001-11-11, by wenzelm
Proof.have_i: multiple statements;
2001-11-11, by wenzelm
added RAW_METHOD, RAW_METHOD_CASES;
2001-11-11, by wenzelm
added add_thmss;
2001-11-11, by wenzelm
"theorem" etc.: multiple statements;
2001-11-11, by wenzelm
theorem, have, show etc: multiple statements;
2001-11-11, by wenzelm
facts: multiple args;
2001-11-11, by wenzelm
added conjunction_tac;
2001-11-11, by wenzelm
renamed open_smart_store_thms to smart_store_thms_open;
2001-11-11, by wenzelm
added mk_conjunction;
2001-11-11, by wenzelm
added unflat;
2001-11-11, by wenzelm
added conj_elim_precise, conj_intr_thm;
2001-11-11, by wenzelm
use Tactic.prove;
2001-11-10, by wenzelm
tuned;
2001-11-09, by wenzelm
support co/inductive definitions in new-style theories;
2001-11-09, by wenzelm
adapted to add_inductive_x;
2001-11-09, by wenzelm
syntactic declaration of external *and* internal versions of fixes;
2001-11-09, by wenzelm
fixed print_records;
2001-11-09, by wenzelm
tuned;
2001-11-09, by wenzelm
theorems case_split = case_split_thm [case_names True False, cases type: o];
2001-11-09, by wenzelm
Theorems symmetric, reflexive and transitive are now stored with "open"
2001-11-09, by berghofe
Commands prf and full_prf can now also be used to display proof term
2001-11-09, by berghofe
eliminated old "symbols" syntax, use "xsymbols" instead;
2001-11-09, by wenzelm
theory data: finish method;
2001-11-09, by wenzelm
indexvar_ast_tr (for \<index> placeholder);
2001-11-09, by wenzelm
removed pure_sym_syntax;
2001-11-09, by wenzelm
File.use;
2001-11-09, by wenzelm
added impose_hyps_tac;
2001-11-09, by wenzelm
proper close_locale;
2001-11-09, by wenzelm
no longer support "isabelle_font" or "symbols";
2001-11-09, by wenzelm
got rid of obsolete input filtering;
2001-11-09, by wenzelm
back to normal;
2001-11-09, by wenzelm
eliminated old "symbols" syntax, use "xsymbols" instead;
2001-11-09, by wenzelm
updated;
2001-11-09, by wenzelm
got rid of obsolete input filtering and isabelle font encoding;
2001-11-09, by wenzelm
got rid of obsolete input filtering;
2001-11-09, by wenzelm
eliminated old "symbols" syntax, use "xsymbols" instead;
2001-11-09, by wenzelm
theory data: finish method;
2001-11-08, by wenzelm
removed needs_filtered_use;
2001-11-08, by wenzelm
\newcommand{\isasymindex}{\isamath{\i}};
2001-11-08, by wenzelm
* Isar/Pure: emulation of instantiation tactics (rule_tac, cut_tac,
2001-11-08, by wenzelm
tuned;
2001-11-08, by wenzelm
\bibliographystyle{abbrv};
2001-11-08, by wenzelm
updated;
2001-11-08, by wenzelm
make SML/XL of NJ happy;
2001-11-08, by wenzelm
ex/document/root.bib;
2001-11-08, by wenzelm
proper syntax for structs;
2001-11-08, by wenzelm
more explanations on advanced syntax;
2001-11-08, by wenzelm
use num_const of Pure;
2001-11-08, by wenzelm
\newcommand{\isasymstruct}{\isamath{\diamond}};
2001-11-08, by wenzelm
locale_prefix: Sign.base_name;
2001-11-07, by wenzelm
syntax for structs;
2001-11-07, by wenzelm
tuned;
2001-11-07, by wenzelm
syntax for structures;
2001-11-07, by wenzelm
tuned impose_hyps;
2001-11-07, by wenzelm
added structures;
2001-11-07, by wenzelm
\isasymstruct;
2001-11-07, by wenzelm
Sidi Ehmety's port of the fold_set operator and multisets to ZF.
2001-11-07, by paulson
reorganization of the ZF examples
2001-11-07, by paulson
tuned;
2001-11-07, by wenzelm
cert_def: proper check of args, improved msgs;
2001-11-06, by wenzelm
pretty_goals_local: observes context syntax;
2001-11-06, by wenzelm
defines: Thm.def_name, proper check of args;
2001-11-06, by wenzelm
separate "in" locale vs. ad-hoc context;
2001-11-06, by wenzelm
goals_limit moved to display.ML;
2001-11-06, by wenzelm
less
more
|
(0)
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip