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.
HOL-Complex with proof terms
2008-06-30, by haftmann
code generator setup for "int" also works under eta-contraction
2008-06-30, by haftmann
added ML/ml_thms.ML;
2008-06-28, by wenzelm
tuned;
2008-06-28, by wenzelm
tuned;
2008-06-28, by wenzelm
additional ML antiquotations;
2008-06-28, by wenzelm
moved theorem values to ml_thms.ML;
2008-06-28, by wenzelm
Isar theorem values within ML.
2008-06-28, by wenzelm
added ML/ml_thms.ML;
2008-06-28, by wenzelm
updated generated file;
2008-06-28, by wenzelm
allow overlap of minor keywords and commands;
2008-06-28, by wenzelm
include HOL-Plain;
2008-06-28, by wenzelm
tuned args parser (cf. args.ML);
2008-06-28, by wenzelm
replaced simple_text by fully-featured parse_args;
2008-06-28, by wenzelm
tuned nested args parser;
2008-06-28, by wenzelm
@{lemma}: 'by' keyword;
2008-06-28, by wenzelm
ML: improved antiquotations;
2008-06-28, by wenzelm
added macro interface;
2008-06-28, by wenzelm
tuned;
2008-06-28, by wenzelm
added thm_name, opt_thm_name;
2008-06-28, by wenzelm
adjusted import
2008-06-27, by haftmann
adjusted import
2008-06-27, by haftmann
added a lemma to at_swap_simps
2008-06-27, by urbanc
remove cset theory; define ideal completions using typedef instead of cpodef
2008-06-26, by huffman
Args.theory;
2008-06-26, by wenzelm
added context/theory scanner;
2008-06-26, by wenzelm
Args.context;
2008-06-26, by wenzelm
fix: need to beta/eta normalize
2008-06-26, by krauss
established Plain theory and image
2008-06-26, by haftmann
added dummy citiation
2008-06-26, by haftmann
dropped recdef
2008-06-26, by haftmann
class theory name lookup improved
2008-06-26, by haftmann
modernized specifications;
2008-06-25, by wenzelm
tuned proofs;
2008-06-25, by wenzelm
modernized specifications;
2008-06-25, by wenzelm
modernized specifications;
2008-06-25, by wenzelm
typo
2008-06-25, by urbanc
re-use official outer keywords;
2008-06-25, by wenzelm
scan: prefer command over keyword, allowing lexicons to overlap;
2008-06-25, by wenzelm
moved global keywords from OuterSyntax to OuterKeyword, tuned interfaces;
2008-06-25, by wenzelm
moved global keywords from OuterSyntax to OuterKeyword, tuned interfaces;
2008-06-25, by wenzelm
antiquote: need to quote outer keywords;
2008-06-25, by wenzelm
tuned;
2008-06-25, by wenzelm
moved global keywords from OuterSyntax to OuterKeyword, tuned interfaces;
2008-06-25, by wenzelm
- Equivariance simpset used in proofs of strong induction and inversion
2008-06-25, by berghofe
pprint: back to proper output of markup, with workaround for Poly/ML crash;
2008-06-25, by wenzelm
back to 1.36 (Poly/ML crash!?);
2008-06-24, by wenzelm
updated generated file;
2008-06-24, by wenzelm
YXML: no special treatment of white space;
2008-06-24, by wenzelm
pprint: proper output of markup (important for token translation);
2008-06-24, by wenzelm
ml_code_antiq: proper scanner combinators;
2008-06-24, by wenzelm
moved concrete antiquotations to ml_antiquote.ML;
2008-06-24, by wenzelm
Antiquote.Open/Close;
2008-06-24, by wenzelm
add_antiq: more general notion of ML antiquotation;
2008-06-24, by wenzelm
added Open/Close -- checked blocks;
2008-06-24, by wenzelm
added pprint_thy_ref;
2008-06-24, by wenzelm
Common ML antiquotations.
2008-06-24, by wenzelm
added ML/ml_antiquote.ML;
2008-06-24, by wenzelm
ML_Antiquote.value;
2008-06-24, by wenzelm
added isaantiqopen/close;
2008-06-24, by wenzelm
Logic.all/mk_equals/mk_implies;
2008-06-23, by wenzelm
moved implies to logic.ML;
2008-06-23, by wenzelm
added all, is_all;
2008-06-23, by wenzelm
Logic.implies;
2008-06-23, by wenzelm
Logic.is_all;
2008-06-23, by wenzelm
Term.all;
2008-06-23, by wenzelm
Logic.all/mk_equals/mk_implies;
2008-06-23, by wenzelm
session name: empty for Pure and by default;
2008-06-23, by wenzelm
induct_tac: allow omission of arguments;
2008-06-23, by wenzelm
info: default name is "", not "Pure";
2008-06-23, by wenzelm
moved src/HOL/Tools/induct_tacs.ML to src/Tools/induct_tacs.ML;
2008-06-23, by wenzelm
removed obsolete dest_concls;
2008-06-23, by wenzelm
induct_tac: mutual rules work as for method "induct";
2008-06-23, by wenzelm
tuned get_inductT: *all* rules for missing instantiation;
2008-06-23, by wenzelm
induct_tac: infer mutual rule from types, as for proper induct method;
2008-06-23, by wenzelm
induct_tac/case_tac: nested tuples are split as expected;
2008-06-23, by wenzelm
induct_tac: old conjunctive rules no longer supported;
2008-06-23, by wenzelm
updated generated file;
2008-06-23, by wenzelm
induct_tac: rule is inferred from types;
2008-06-23, by wenzelm
cleaned up some proofs;
2008-06-22, by huffman
use new-style abbreviation/notation for fix syntax
2008-06-22, by huffman
import_export_proof: simplified thm definition -- PureThy.name_thm does the job;
2008-06-21, by wenzelm
added query_type/const/class (meta data);
2008-06-21, by wenzelm
the_tags: explicit error message;
2008-06-21, by wenzelm
activate_context: strict the_context, no fallback on theory context;
2008-06-21, by wenzelm
remove unused constant liftpair
2008-06-20, by huffman
simplify profinite class axioms
2008-06-20, by huffman
clean up and rename some profinite lemmas
2008-06-20, by huffman
move at-sml-dev-e to macbroy23
2008-06-20, by isatest
replace SetPcpo.thy with Cset.thy
2008-06-20, by huffman
updated for 2008;
2008-06-20, by wenzelm
(removed non-present change)
2008-06-20, by haftmann
explicit thm context for error messages
2008-06-20, by haftmann
using tages to find theory names
2008-06-20, by haftmann
type constructors now with markup
2008-06-20, by haftmann
fixed bind error for malformed primrec specifications
2008-06-20, by haftmann
DatatypeProp.make_distincts: only one half of each symmetric pair is constructed
2008-06-20, by haftmann
streamlined definitions
2008-06-20, by haftmann
moved Float.thy to Library
2008-06-20, by haftmann
removed SetPcpo.thy and cpo instance for type bool;
2008-06-20, by huffman
moved Abs_image to Typedef.thy; prove finite_UNIV outside the locale
2008-06-20, by huffman
add lemma Abs_image
2008-06-20, by huffman
added some lemmas; reorganized into sections; tuned proofs
2008-06-20, by huffman
added some lemmas; tuned proofs
2008-06-20, by huffman
tuned
2008-06-20, by huffman
replace less_lift with flat_less_iff
2008-06-20, by huffman
tweak lemmas adm_all and adm_ball
2008-06-20, by huffman
move lemmas into locales;
2008-06-19, by huffman
add lemmas take_chain_less and take_chain_le
2008-06-19, by huffman
disposed Sign.read_typ etc;
2008-06-19, by wenzelm
renamed is_abbrev_mode to abbrev_mode;
2008-06-19, by wenzelm
ProofContext.abbrev_mode;
2008-06-19, by wenzelm
moved get_sort to Isar/proof_context.ML;
2008-06-19, by wenzelm
tuned signature;
2008-06-19, by wenzelm
private add_used (from drule.ML);
2008-06-19, by wenzelm
Variable.declare_typ;
2008-06-19, by wenzelm
added declare_typ;
2008-06-19, by wenzelm
moved add_used to Isar/rule_insts.ML;
2008-06-19, by wenzelm
export read_typ/cert_typ -- version with regular context operations;
2008-06-19, by wenzelm
export read_typ/cert_typ -- version with regular context operations;
2008-06-19, by wenzelm
less
more
|
(0)
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip