Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-300
-100
-96
+96
+100
+300
+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.
remove dead code
2010-02-27, by huffman
removed dead code
2010-02-27, by huffman
register match functions from domain_constructors.ML
2010-02-27, by huffman
move definition of match combinators to domain_constructors.ML
2010-02-27, by huffman
move proofs of dis_rews to domain_constructors.ML; change dis_defins to iff-style
2010-02-27, by huffman
move definition of discriminators to domain_constructors.ML
2010-02-27, by huffman
move proofs of when_rews intro domain_constructors.ML
2010-02-27, by huffman
moved proofs of dist_les and dist_eqs to domain_constructors.ML
2010-02-27, by huffman
move proofs of casedist into domain_constructors.ML
2010-02-27, by huffman
move proofs of injects and inverts to domain_constructors.ML
2010-02-26, by huffman
reuse vars_of function
2010-02-26, by huffman
remove unnecessary stuff from argument to add_constructors function
2010-02-26, by huffman
reorder sections
2010-02-26, by huffman
move proof of con_rews into domain_constructor.ML
2010-02-26, by huffman
don't bother returning con_defs
2010-02-26, by huffman
move constructor-specific stuff to a separate function
2010-02-26, by huffman
replace prove_thm function
2010-02-26, by huffman
move proof of compactness rules into domain_constructors.ML
2010-02-26, by huffman
add some convenience functions
2010-02-26, by huffman
rewrite domain package code for selector functions
2010-02-25, by huffman
add function beta_of_def
2010-02-24, by huffman
reorganizing domain package code (in progress)
2010-02-24, by huffman
change domain package's treatment of variable names in theorems to be like datatype package
2010-02-24, by huffman
remove redundant lemma real_minus_half_eq
2010-02-24, by huffman
polished and converted some proofs to Isar style
2010-02-24, by huffman
killed more recdefs
2010-03-02, by krauss
tuned comment
2010-03-01, by krauss
repaired subscripts broken in d8d7d1b785af
2010-03-02, by haftmann
repaired definition (cf. d8d7d1b785af)
2010-03-02, by haftmann
authentic syntax for *all* logical entities;
2010-03-03, by wenzelm
mark_atoms: more precise treatment of SynExt.standard_token_markers vs. syntax consts;
2010-03-03, by wenzelm
notation for xsymbols (cf. ad039d29e01c);
2010-03-03, by wenzelm
"_type_prop" is syntax const -- recovered printing of OFCLASS;
2010-03-03, by wenzelm
removed unused external_names;
2010-03-03, by wenzelm
cleanup type translations;
2010-03-03, by wenzelm
adapted to authentic syntax -- actual types are verbatim;
2010-03-03, by wenzelm
authentic syntax for classes and type constructors;
2010-03-03, by wenzelm
more systematic mark/unmark operations;
2010-03-03, by wenzelm
proper (type_)notation;
2010-03-02, by wenzelm
proper antiquotations;
2010-03-02, by wenzelm
standard convention for syntax consts;
2010-03-02, by wenzelm
more precise scope of exception handler;
2010-03-02, by wenzelm
eliminated hard tabs;
2010-03-01, by wenzelm
tuned final whitespace;
2010-03-01, by wenzelm
repaired 'definition' (cf. d8d7d1b785af);
2010-03-01, by wenzelm
merged
2010-03-01, by wenzelm
more recdef (and old primrec) hunting
2010-03-01, by krauss
killed recdefs in HOL-Auth
2010-03-01, by krauss
merged
2010-03-01, by haftmann
replaced a couple of constsdefs by definitions (also some old primrecs by modern ones)
2010-03-01, by haftmann
export add_quotient_type.
2010-03-01, by Cezary Kaliszyk
updated generated files;
2010-03-01, by wenzelm
added type_notation command;
2010-03-01, by wenzelm
more uniform treatment of syntax for types vs. consts;
2010-03-01, by wenzelm
made smlnj happy
2010-03-01, by bulwahn
more antiquotations;
2010-02-28, by wenzelm
more antiquotations;
2010-02-28, by wenzelm
modernized structure Term_Ord;
2010-02-27, by wenzelm
use existing Typ_Graph;
2010-02-27, by wenzelm
further standard instances of functor Graph;
2010-02-27, by wenzelm
code simplification by inlining;
2010-02-27, by wenzelm
just one copy of structure Term_Graph (in Pure);
2010-02-27, by wenzelm
modernized structure Int_Graph;
2010-02-27, by wenzelm
clarified @{const_name} vs. @{const_abbrev};
2010-02-27, by wenzelm
clarified @{const_name} (only logical consts) vs. @{const_abbrev};
2010-02-27, by wenzelm
type/const name: explicitly allow abbreviations as well;
2010-02-27, by wenzelm
clarified ProofContext.read_const(_proper)/Args.const(_proper) wrt. strict logical consts;
2010-02-27, by wenzelm
added at-poly-test, which is intended for performance tests of Poly/ML itself;
2010-02-27, by wenzelm
more precise syntax antiquotations;
2010-02-27, by wenzelm
ML antiquotations for type classes;
2010-02-27, by wenzelm
read_class: perform actual read, with source position;
2010-02-27, by wenzelm
parallel brute-force disambiguation;
2010-02-27, by wenzelm
degrade gracefully in CRITICAL section;
2010-02-27, by wenzelm
gen_dest_case: recovered @{const_name} from c8a6fae0ad0c, because of separate Syntax.mark_const in case_tr' -- avoid extra syntax markers in output;
2010-02-26, by wenzelm
tuned;
2010-02-26, by wenzelm
use simplified Syntax.escape;
2010-02-26, by wenzelm
tuned hyp_subst_tac';
2010-02-26, by wenzelm
use SAT4J for "Tests_Nits.thy" for safety (this should solve the Isatest failures) + minor changes
2010-02-26, by blanchet
merged
2010-02-26, by blanchet
more work on the new monotonicity stuff in Nitpick
2010-02-26, by blanchet
improved precision of infinite "shallow" datatypes in Nitpick;
2010-02-25, by blanchet
cosmetics
2010-02-25, by blanchet
merged
2010-02-26, by bulwahn
merged
2010-02-26, by bulwahn
adding no_topmost_reordering as new option to the code_pred command
2010-02-25, by bulwahn
adopting Mutabelle to quickcheck reporting; improving quickcheck reporting
2010-02-25, by bulwahn
added quiet option to quickcheck command
2010-02-25, by bulwahn
added basic reporting of test cases to quickcheck
2010-02-25, by bulwahn
merged
2010-02-26, by haftmann
use abstract code cerficates for bare code theorems
2010-02-26, by haftmann
implement quotient_of for odl SML code generator
2010-02-26, by haftmann
adjusted to cs. e4a7947e02b8
2010-02-26, by haftmann
bound argument for abstype proposition
2010-02-24, by haftmann
renamed theory Rational to Rat
2010-02-24, by haftmann
tuned whitespace
2010-02-24, by haftmann
more precise exception handler
2010-02-24, by haftmann
less
more
|
(0)
-30000
-10000
-3000
-1000
-300
-100
-96
+96
+100
+300
+1000
+3000
+10000
+30000
tip