Skip to content
This repository has been archived by the owner on Oct 14, 2023. It is now read-only.

Releases: leanprover/lean3

v3.4.2

18 Jan 14:46
Compare
Choose a tag to compare

Patch release

Features

  • leanpkg: Allow specifying a branch to use for leanpkg upgrade (#1981)

Changes

  • Fix the definition of list.lt

  • Make leanpkg work when installed in a path containing spaces

  • io: Encode/decode UTF-8 for text-mode streams

  • Remove coinductive predicates and transfer. To be moved to mathlib instead.

  • Windows: Ignore file changes that only changed line endings

v3.4.1

28 Apr 22:17
Compare
Choose a tag to compare

Bugfix release: Fix a regression concerning type ascriptions in function position

v3.4.0

16 Apr 23:00
Compare
Choose a tag to compare

Features

  • Implement RFC #1820

  • Add string.iterator abstraction for traversing strings.
    The VM contains an efficient implementation of this type.

  • Add support for non-ASCII char literals. Example: 'α'.

  • Unicode escape characters in string and char literals. For example, '\u03B1' is equivalent to 'α'.

  • Predictable runtime cost model for recursive functions. The equation compiler uses
    different techniques for converting recursive equations into recursors and/or
    well-founded fixed points. The new approach used in the code generator ignores
    these encoding tricks when producing byte code. So, the runtime cost model
    is identical to the one in regular strict functional languages.

  • Add d_array n α (array type where value type may depend on index),
    where (α : fin n → Type u).

  • Add instance for decidable_eq (d_array n α) and decidable_eq (array n α).
    The new instance is more efficient than the one in mathlib because it doesn't
    convert the array into a list.

  • Add aliasing pattern syntax id@pat, which introduces the name id for the value matched by
    the pattern pat.

  • Add alternative syntax {..., ..s} for the structure update {s with ...}.
    Multiple fallback sources can be given: {..., ..s, ..t} will fall back to
    searching a field in s, then in t. The last component can also be ..,
    which will replace any missing fields with a placeholder.
    The old notation will be removed in the future.

  • Add support for structure instance notation {...} in patterns. Use .. to ignore
    unmatched fields.

  • Type class has_equiv for notation.

  • Add funext ids* tactic for applying the funext lemma.

  • Add iterate n { t } for applying tactic t n times.
    Remark: iterate { t } applies t until it fails.

  • Add with_cases { t }. This tactic applies t to the main goal,
    and reverts any new hypothesis in the resulting subgoals. with_cases also enable "goal tagging".
    Remark: induction and cases tag goals using constructor names. apply and constructor tag goals
    using parameter names. The case tactic can select goals using tags.

  • Add cases_matching p tactic for applying the cases tactic to a hypothesis h : t s.t.
    t matches the pattern p. Alternative versions: cases_matching* p and cases_matching [p_1, ..., p_n].
    Example: cases_matching* [_ ∨ _, _ ∧ _] destructs all conjunctions and disjunctions in the main goal.

  • Add cases_type I tactic for applying the cases tactic to a hypothesis h : I ....
    cases_type! I only succeeds when the number of resulting goals is <= 1.
    Alternative versions: cases_type I_1 ... I_n, cases_type* I, cases_type!* I.
    Example: cases_type* and or destructs all conjunctions and disjunctions in the main goal.

  • Add constructor_matching p tactic. It is syntax sugar for match_target p; constructor.
    The variant constructor_matching* p is more efficient than focus1 { repeat { match_target p; constructor } }
    because the patterns are compiled only once.

  • injection h now supports nested and mutually recursive datatypes.

  • Display number of goals in the *Lean Goal* buffer (if number of goals > 1).

  • hide id* command for hiding aliases.
    The following command hides the alias is_true for decidable.is_true.

    hide is_true
    
  • Add abbreviation declaration command. abbreviation d : t := v is equivalent to
    @[reducible, inline] def d : t := v and a kernel reducibility hint.
    Before this command, we had to use meta programming for setting the kernel reducibility hint.
    This was problematic because we could only define abbreviations after the meta programming
    framework was defined.

  • Add "smart unfolding". The idea is to prevent internal compilation details
    used by the equation compiler to "leak" during unification, tactic execution and
    reduction. With "smart unfolding", the term nat.add a (nat.succ b) reduces
    to nat.succ (nat.add a b) instead of nat.succ (... incomprehensible mess ...).
    This feature addresses a problem reported by many users.
    See issue #1794.
    The command set_option type_context.smart_unfolding false disables this feature.

  • Add support for "auto params" at simp tactic. Example: given

    @[simp] lemma fprop1 (x : nat) (h : x > 0 . tactic.assumption) : f x = x := ...
    

    The simplifier will try to use tactic assumption to synthesize parameter h.

  • Add interactive sorry tactic (alias for admit).

  • simp now reduces equalities c_1 ... = c_2 ... to false if c_1 and c_2 are distinct
    constructors. This feature can be disabled using simp {constructor_eq := ff}.

  • simp now reduces equalities c a_1 ... a_n = c b_1 ... b_n to a_1 = b_1 /\ ... /\ a_n = b_n if c is a constructor.
    This feature can be disabled using simp {constructor_eq := ff}.

  • subst and subst_vars now support heterogeneous equalities that are actually homogeneous
    (i.e., @heq α a β b where α and β are definitionally equal).

  • Add interactive subst_vars tactic.

  • Add leanpkg add foo/bar as a shorthand for leanpkg add https://github.com/foo/bar.

  • Add leanpkg help <command>.

  • Add [norm] simp set. It contains all lemmas tagged with [simp] plus any
    lemma tagged with [norm].
    These rules are used to produce normal forms and/or reduce the
    number of constants used in a goal. For example, we plan to
    add the lemma f <$> x = x >>= pure ∘ f to [norm].

  • Add iota_eqn : bool field to simp_config. simp {iota_eqn := tt} uses
    all non trivial equation lemmas generated by equation/pattern-matching compiler.
    A lemma is considered non trivial if it is not of the form forall x_1 ... x_n, f x_1 ... x_n = t and
    a proof by reflexivity. simp! is a shorthand for simp {iota_eqn := tt}.
    For example, given the goal ... |- [1,2].map nat.succ = t, simp! reduces the left-hand-side
    of the equation to [nat.succ 1, nat.succ 2]. In this example, simp! is equivalent to
    simp [list.map].

  • Allow the Script, Double-struck, and Fractur symbols from
    Mathematical Alphanumeric Symbols: https://unicode.org/charts/PDF/U1D400.pdf
    to be used as variables Example: variables 𝓞 : Prop.

  • Structure instance notation now allows explicitly setting implicit structure fields

  • Structure instance notation now falls back to type inference for inferring the
    value of a superclass. This change eliminates the need for most .. source specifiers
    in instance declarations.

  • The --profile flag will now print cumulative profiling times at the end of execution

  • do notation now uses the top-level, overloadable bind function instead of has_bind.bind,
    allowing binds with different type signatures

  • Structures fields can now be defined with an implicitness infer annotation and parameters.

    class has_pure (f : Type u → Type v) :=
    -- make f implicit
    (pure {} {α : Type u} : α → f α)
    
  • Add except_t and reader_t monad transformers

  • Add monad_{except,reader,state} classes for accessing effects anywhere in a monad stack
    without the need for explicit lifting. Add analogous monad_{except,reader,state}_adapter
    classes for translating a monad stack into another one with the same shape but different
    parameter types.

Changes

  • Command variable [io.interface] is not needed anymore to use the io monad.
    It is also easier to add new io primitives.

  • Replace inout modifier in type class declarations with out_param modifier.
    Reason: counterintuitive behavior in the type class resolution procedure.
    The result could depend on partial information available in the inout
    parameter. Now a parameter (R : inout α → β → Prop) should be written
    as (R : out_param (α → β → Prop)) or (R : out_param $ α → β → Prop).
    Remark: users may define their own notation for declaring out_params.
    Example:

    notation `out`:1024 a:0 := out_param a
    

    We did not include this notation in core lib because out is frequently used to
    name parameters, local variables, etc.

  • case tactic now supports the with_cases { t } tactic. See entry above about with_cases.
    The tag and new hypotheses are now separated with :. Example:

    • case pos { t }: execute tactic t to goal tagged pos
    • case pos neg { t }: execute tactic t to goal tagged pos neg
    • case : x y { t }: execute tactic t to main goal after renaming the first two hypotheses produced by preceding with_case { t' }.
    • case pos neg : x y { t } : execute tactic t to goal tagged pos neg after renaming the first two hypotheses produced by preceding with_case { t' }.
  • cases h now also tries to clear h when performing dependent elimination.

  • repeat { t } behavior changed. Now, it applies t to each goal. If the application succeeds,
    the tactic is applied recursively to all the generated subgoals until it eventually fails.
    The recursion stops in a subgoal when the tactic has failed to make progress.
    The previous repeat tactic was renamed to iterate.

  • The automatically generated recursor C.rec for an inductive datatype
    now uses ih to name induction hypotheses instead of ih_1 if there is only one.
    If there is more than one induction hypotheses, the name is generated by concatenating ih_
    before the constructor field name. For example, for the constructor

    | node (left right : tree) (val : A) : tree
    

    The induction hypotheses are now named: ih_left and ih_right.
    This change only affects tactical proofs where explicit names are not provided
    to induction and cases tactics.

  • induction h and `cases...

Read more

v3.3.0

15 Sep 06:34
Compare
Choose a tag to compare

Lean version 3.3.0

Features

  • In addition to user-defined notation parsers introduced in Lean 3.2.0, users may now also define top-level commands in Lean. For an example, see the coinductive command that has been ported to the new model.

  • Add new simplifier configuration option simp_config.single_pass. It is useful for simplification rules that may produce non-termination.
    Example: simp {single_pass := tt}

  • The rewrite tactic has support for equational lemmas. Example: Given a definition f, rw [f] will try to rewrite the goal using the equational lemmas for f.
    The tactic fails if none of the equational lemmas can be used.

  • Add simp * at * variant. It acts on all (non dependent propositional) hypotheses.
    Simplified hypotheses are automatically inserted into the simplification set
    as additional simplification rules.

  • Add «id» notation that can be used to declare and refer to identifiers containing prohibited characters.
    For example, a.«b.c» is a two-part identifier with parts a and b.c.

  • simp tactic now handles lemmas with metavariables. Example simp [add_comm _ b].

  • conv { ... } tactic for applying simplification and rewriting steps.
    In the block {...}, we can use tactics from conv.interactive.
    Examples:

    • conv at h in (f _ _) { simp } applies simp to first subterm matching f _ _ at hypothesis h.
    • conv in (_ = _) { to_lhs, whnf } replace the left-hand-side of the equality in target with its weak-head-normal-form.
    • conv at h in (0 + _) { rw [zero_add] }
    • conv { for (f _ _) [1, 3] {rw [h]}, simp }, first execute rw[h] to the first and third occurrences of an f-application,
      and then execute simp.
  • simp tactics in interactive mode have a new configuration parameter (discharger : tactic unit)
    a tactic for discharging subgoals created by the simplifier. If the tactic fails, the simplifier
    tries to discharge the subgoal by reducing it to true.
    Example: simp {discharger := assumption}.

  • simp and dsimp can be used to unfold projection applications when the argument is a type class instance.
    Example: simp [has_add.add] will replace @has_add.add nat nat.has_add a b with nat.add a b

  • dsimp has several new configuration options to control reduction (e.g., iota, beta, zeta, ...).

  • Non-exhaustive pattern matches now show missing cases.

  • induction e now also works on non-variable e. Unlike ginduction, it will not introduce equalities relating e to the inductive cases.

  • Add notation #[a, b, c, d] for bin_tree.node (bin_tree.node (bin_tree.leaf a) (bin_tree.leaf b)) (bin_tree.node (bin_tree.leaf c) (bin_tree.leaf d)).
    There is a coercion from bin_tree to list. The new notation allows to input long sequences efficiently.
    It also prevents system stack overflows.

  • Tactics that accept a location parameter, like rw thm at h, may now use or the ASCII version |-
    to select the goal as well as any hypotheses, for example rw thm at h1 h2 ⊢.

  • Add user_attribute.after_set/before_unset handlers that can be used for validation as well as side-effecting attributes.

  • Field notation can now be used to make recursive calls.

def list.append : list α → list α → list α
| []       l := l
| (h :: s) t := h :: s.append t
  • leanpkg now stores the intended Lean version in the leanpkg.toml file and reports a warning if the version does not match the installed Lean version.

  • simp and dsimp can now unfold let-bindings in the local context. Use dsimp [x] or simp [x] to unfold the let-binding x : nat := 3.

  • User-defined attributes can now take parameters parsed by a lean.parser. A [derive] attribute that can derive typeclasses such as decidable_eq and inhabited has been implemented on top of this.

Changes

  • We now have two type classes for converting to string: has_to_string and has_repr.
    The has_to_string type class in v3.2.0 is roughly equivalent to has_repr.
    For more details, see discussion here.

  • Merged assert and note tactics and renamed -> have.

  • Renamed pose tactic -> let

  • assume is now a real tactic that does not exit tactic mode.

  • Modified apply tactic configuration object, and implemented RFC #1342. It now has support for auto_param and opt_param. The new eapply tactic only creates subgoals for non dependent premises, and it simulates the behavior of the apply tactic in version 3.2.0.

  • Add configuration object rewrite_cfg to rw/rewrite tactic. It now has support for auto_param and opt_param.
    The new goals are ordered using the same strategies available for apply.

  • All dsimp tactics fail if they did not change anything.
    We can simulate the v3.2.0 using dsimp {fail_if_unchaged := ff} or try dsimp.

  • dsimp does not unfold reducible definitions by default anymore.
    Example: function.comp applications will not be unfolded by default.
    We should use dsimp [f] if we want to reduce a reducible definition f.
    Another option is to use the new configuration parameter unfold_reducible.
    Example dsimp {unfold_reducible := tt}

  • All dunfold and unfold tactics fail if they did not unfold anything.
    We can simulate the v3.2.0 using unfold f {fail_if_unchaged := ff} or try {unfold f}.

  • dunfold_occs was deleted, the new conv tactical should be used instead.

  • unfold tactic is now implemented on top of the simp tactics. So, we can use it to unfold
    declarations defined using well founded recursion. The unfold1 variant does not unfold recursively,
    and it is shorthand for unfold f {single_pass := tt}.
    Remark: in v3.2.0, unfold was just an alias for the dunfold tactic.

  • Deleted simph and simp_using_hs tactics. We should use simp [*] instead.

  • Use simp [-h] and dsimp [-h] instead of simp without h and dsimp without h.
    Moreover, simp [*, -h] if h is a hypothesis, we are adding all hypotheses but h
    as additional simplification lemmas.

  • Changed notation rw [-h] to rw [← h] to avoid confusion with the new simp [-h] notation.
    The ASCII version rw [<- h] is also supported.

  • rw [t] at * now skips any hypothesis used by t. See discussion here.

  • Removed the redundant keywords take (replace with assume) and suppose (replace with the new anonymous assume :)

  • Universes max u v + 1 and imax u v + 1 are now parsed as (max u v) + 1 and (imax u v) + 1.

  • Merged generalize and generalize2 tactics into new generalize id? : expr = id tactic

  • standard.lean has been removed. Any files that import standard can simply remove the line as
    most things that were once imported by this are now imported by default.

  • The type classes for orders have been refactored to combine both the (<)
    and (≤) operations. The new classes are preorder, partial_order, and
    linear_order. The partial_order class corresponds to weak_order,
    strict_order, order_pair, and strong_order_pair. The linear_order
    class corresponds to linear_order_pair, and linear_strong_order_pair.

  • injection and injections tactics generate fresh names when user does not provide names.
    The fresh names are of the form h_<idx>. See discussion here.

  • Use structure to declare and. This change allows us to use h.1 and h.2 as shorthand for h.left and h.right.

  • Add attribute [pp_using_anonymous_constructor] to and. Now, and.intro h1 h2 is pretty printed as
    ⟨h1, h2⟩. This change is motivated by the previous one. Without it, and.intro h1 h2 would be
    pretty printed as {left := h1, right := h2}.

  • User attributes can no longer be set with set_basic_attribute. You need to use user_attribute.set now.

API name changes

  • list.dropn => list.drop
  • list.taken => list.take
  • tactic.dsimp and tactic.dsimp_core => tactic.dsimp_target
  • tactic.dsimp_at_core and tactic.dsimp_at => tactic.dsimp_hyp
  • tactic.delta_expr => tactic.delta
  • tactic.delta => tactic.delta_target
  • tactic.delta_at => tactic.delta_hyp
  • tactic.simplify_goal => tactic.simp_target
  • tactic.unfold_projection => tactic.unfold_proj
  • tactic.unfold_projections_core => tactic.unfold_projs
  • tactic.unfold_projections => tactic.unfold_projs_target
  • tactic.unfold_projections_at => tactic.unfold_projs_hyp
  • tactic.simp_intros_using, tactic.simph_intros_using, tactic.simp_intro_lst_using, tactic.simph_intro_lst_using => tactic.simp_intros
  • tactic.simp_at => tactic.simp_hyp
  • deleted tactic.simp_at_using
  • deleted tactic.simph_at

v3.2.0

18 Jun 18:03
Compare
Choose a tag to compare

Lean release

v3.1.0

26 Feb 00:05
Compare
Choose a tag to compare

Lean release

v3.0.0

20 Jan 02:58
Compare
Choose a tag to compare

Lean release

popl_paris_2017

14 Jan 17:10
Compare
Choose a tag to compare

Lean release